Equations
@[reducible, inline]
Instances For
@[reducible, inline]
Instances For
Instances For
Instances For
Equations
- Lean.Meta.Linear.Nat.instToExprLinearCnstr = { toExpr := fun (a : Lean.Meta.Linear.Nat.LinearCnstr) => a.toExpr, toTypeExpr := Lean.mkConst `Nat.Linear.ExprCnstr }
def
Lean.Meta.Linear.Nat.LinearExpr.toArith
(ctx : Array Lean.Expr)
(e : Lean.Meta.Linear.Nat.LinearExpr)
:
Instances For
def
Lean.Meta.Linear.Nat.LinearCnstr.toArith
(ctx : Array Lean.Expr)
(c : Lean.Meta.Linear.Nat.LinearCnstr)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
- varMap : Lean.Meta.KExprMap Nat
Instances For
@[reducible, inline]
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Meta.Linear.Nat.ToLinear.run
{α : Type}
(x : Lean.Meta.Linear.Nat.ToLinear.M α)
:
Lean.MetaM (α × Array Lean.Expr)
Instances For
Equations
- Lean.Meta.Linear.Nat.reflTrue = Lean.mkApp2 (Lean.mkConst `Eq.refl [Lean.levelOne]) (Lean.mkConst `Bool) (Lean.mkConst `Bool.true)