Documentation

Lean.Compiler.ConstFolding

Equations
  • One or more equations did not get rendered due to their size.
@[export lean_get_num_lit]
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Compiler.foldBinUInt (fn : Lean.Compiler.NumScalarTypeInfoBoolNatNatNat) (beforeErasure : Bool) (a₁ : Lean.Expr) (a₂ : Lean.Expr) :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Compiler.foldUIntSub (beforeErasure : Bool) (a₁ : Lean.Expr) (a₂ : Lean.Expr) :
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
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Compiler.toDecidableExpr (beforeErasure : Bool) (pred : Lean.Expr) (r : Bool) :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Compiler.foldNatBinPred (mkPred : Lean.ExprLean.ExprLean.Expr) (fn : NatNatBool) (beforeErasure : Bool) (a₁ : Lean.Expr) (a₂ : Lean.Expr) :
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.
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.
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_fold_bin_op]
def Lean.Compiler.foldBinOp (beforeErasure : Bool) (f : Lean.Expr) (a : Lean.Expr) (b : Lean.Expr) :
Equations
@[export lean_fold_un_op]
def Lean.Compiler.foldUnOp (beforeErasure : Bool) (f : Lean.Expr) (a : Lean.Expr) :
Equations