Instances
- Lean.instToExprDeclarationRanges
- Lean.Position.instToExprPosition
- Lean.instToExprUnit
- Lean.instToExprOption
- Lean.Meta.Linear.Nat.instToExprLinearExpr
- Lean.Meta.Linear.Nat.instToExprLinearCnstr
- Lean.instToExprList
- Lean.instToExprNat
- Lean.instToExprArray
- Lean.instToExprProd
- Lean.instToExprDeclarationRange
- Lean.instToExprBool
- Lean.instToExprName
- Lean.instToExprString
- Lean.instToExprChar
Equations
- Lean.instToExprNat = { toExpr := Lean.mkNatLit, toTypeExpr := Lean.mkConst `Nat }
Equations
- Lean.instToExprBool = { toExpr := fun b => if b = true then Lean.mkConst `Bool.true else Lean.mkConst `Bool.false, toTypeExpr := Lean.mkConst `Bool }
Equations
- Lean.instToExprChar = { toExpr := fun c => Lean.mkApp (Lean.mkConst `Char.ofNat) (Lean.toExpr (Char.toNat c)), toTypeExpr := Lean.mkConst `Char }
Equations
- Lean.instToExprString = { toExpr := Lean.mkStrLit, toTypeExpr := Lean.mkConst `String }
Equations
- Lean.instToExprUnit = { toExpr := fun x => Lean.mkConst `Unit.unit, toTypeExpr := Lean.mkConst `Unit }
Equations
- Lean.Name.toExprAux Lean.Name.anonymous = Lean.mkConst `Lean.Name.anonymous
- Lean.Name.toExprAux (Lean.Name.str p s a) = Lean.mkAppB (Lean.mkConst `Lean.Name.mkStr) (Lean.Name.toExprAux p) (Lean.toExpr s)
- Lean.Name.toExprAux (Lean.Name.num p n a) = Lean.mkAppB (Lean.mkConst `Lean.Name.mkNum) (Lean.Name.toExprAux p) (Lean.toExpr n)
Equations
- Lean.instToExprName = { toExpr := Lean.Name.toExprAux, toTypeExpr := Lean.mkConst `Lean.Name }
Equations
- One or more equations did not get rendered due to their size.
def
Lean.List.toExprAux
{α : Type u_1}
[inst : Lean.ToExpr α]
(nilFn : Lean.Expr)
(consFn : Lean.Expr)
:
Equations
- Lean.List.toExprAux nilFn consFn [] = nilFn
- Lean.List.toExprAux nilFn consFn (a :: as) = Lean.mkApp2 consFn (Lean.toExpr a) (Lean.List.toExprAux nilFn consFn as)
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.
instance
Lean.instToExprProd
{α : Type}
{β : Type}
[inst : Lean.ToExpr α]
[inst : Lean.ToExpr β]
:
Lean.ToExpr (α × β)
Equations
- One or more equations did not get rendered due to their size.