Documentation

Lean.Level

def Nat.imax (n : Nat) (m : Nat) :
Equations

Cached hash code, cached results, and other data for Level. hash : 32-bits hasMVar : 1-bit hasParam : 1-bit depth : 24-bits

Equations
Equations
def Lean.Level.mkData (h : UInt64) (depth : optParam Nat 0) (hasMVar : optParam Bool false) (hasParam : optParam Bool false) :
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
structure Lean.MVarId:
Type
Equations
Equations
Equations
instance Lean.instForInMVarIdSetMVarId {m : Type u_1Type u_2} :
Equations
def Lean.MVarIdMap (α : Type) :
Type
Equations
Equations
instance Lean.instForInMVarIdMapProdMVarId {m : Type u_1Type u_2} {α : Type} :
Equations
Equations
  • Lean.instInhabitedMVarIdMap = { default := }
@[inline]
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_level_hash]
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_level_mk_zero]
Equations
Equations
Equations
Equations
Equations
Equations
Equations
Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
@[extern lean_level_eq]

occurs u l return true iff u occurs in l.

Equations
Equations
  • One or more equations did not get rendered due to their size.

A total order on level expressions that has the following properties

  • succ l is an immediate successor of l.
  • zero is the minimal element. This total order is used in the normalization procedure.
Equations

Reduce (if possible) universe level by 1

Equations
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_level_mk_max_simp]
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_level_mk_imax_simp]
Equations
  • One or more equations did not get rendered due to their size.
@[extern lean_level_update_succ]
Equations
@[inline]
Equations
  • One or more equations did not get rendered due to their size.
@[extern lean_level_update_max]
Equations
@[inline]
Equations
  • One or more equations did not get rendered due to their size.
@[extern lean_level_update_imax]
Equations
@[inline]
Equations
  • One or more equations did not get rendered due to their size.
@[specialize]
Equations
@[inline]
abbrev Lean.LevelMap (α : Type) :
Type
Equations
@[inline]
abbrev Lean.PersistentLevelMap (α : Type) :
Type
Equations
Equations
@[inline]
abbrev Nat.toLevel (n : Nat) :
Equations