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
- Lean.PrettyPrinter.ppExpr e = Lean.PrettyPrinter.ppUsing e fun e => Lean.PrettyPrinter.delab e ∅
def
Lean.PrettyPrinter.ppExprWithInfos
(e : Lean.Expr)
(optsPerPos : optParam Lean.PrettyPrinter.Delaborator.OptionsPerPos ∅)
:
Lean.MetaM (Lean.Format × Std.RBMap Nat Lean.Elab.Info compare)
Return a fmt
representing pretty-printed e
together with a map from tags in fmt
to Elab.Info
nodes produced by the delaborator at various subexpressions of e
.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.PrettyPrinter.ppConst e = Lean.PrettyPrinter.ppUsing e fun e => do let a ← Lean.PrettyPrinter.delabCore e ∅ Lean.PrettyPrinter.Delaborator.delabConst pure a.fst
@[export lean_pp_expr]
def
Lean.PrettyPrinter.ppExprLegacy
(env : Lean.Environment)
(mctx : Lean.MetavarContext)
(lctx : Lean.LocalContext)
(opts : Lean.Options)
(e : 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.