Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.PrettyPrinter.Delaborator.unfoldMDatas (Lean.Expr.mdata a e a_1) = Lean.PrettyPrinter.Delaborator.unfoldMDatas e
- Lean.PrettyPrinter.Delaborator.unfoldMDatas _fun_discr = _fun_discr
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.
def
Lean.PrettyPrinter.Delaborator.unresolveNameGlobal.unresolveNameCore
(n₀ : Lean.Name)
(n : Lean.Name)
:
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.
def
Lean.PrettyPrinter.Delaborator.withMDataOptions
{α : Type}
[inst : Inhabited α]
(x : Lean.PrettyPrinter.Delaborator.DelabM α)
:
Equations
- One or more equations did not get rendered due to their size.
partial def
Lean.PrettyPrinter.Delaborator.withMDatasOptions
{α : Type}
[inst : Inhabited α]
(x : Lean.PrettyPrinter.Delaborator.DelabM α)
:
Equations
- One or more equations did not get rendered due to their size.
- name : Lean.Name
- bInfo : Lean.BinderInfo
- isAutoParam : Bool
def
Lean.PrettyPrinter.Delaborator.ParamKind.isRegularExplicit
(param : Lean.PrettyPrinter.Delaborator.ParamKind)
:
Equations
- Lean.PrettyPrinter.Delaborator.ParamKind.isRegularExplicit param = (Lean.BinderInfo.isExplicit param.bInfo && !param.isAutoParam && Option.isNone param.defVal)
Return array with n-th element set to kind of n-th parameter of e
.
Equations
- One or more equations did not get rendered due to their size.
partial def
Lean.PrettyPrinter.Delaborator.getParamKinds.forallTelescopeArgs
(f : Lean.Expr)
(args : Array Lean.Expr)
(k : Array Lean.Expr → Lean.Expr → Lean.PrettyPrinter.Delaborator.DelabM (Array Lean.PrettyPrinter.Delaborator.ParamKind))
:
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.
- info : Lean.Meta.MatcherInfo
- matcherTy : Lean.Expr
- motiveNamed : Bool
State for delabAppMatch
and helpers.
Delaborate applications of the form (fun x => b) v
as let_fun x := v; b
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.
Check for a Syntax.ident
of the given name anywhere in the tree.
This is usually a bad idea since it does not check for shadowing bindings,
but in the delaborator we assume that bindings are never shadowed.
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.
Delaborate a projection primitive. These do not usually occur in
user code, but are pretty-printed when e.g. #print
ing a projection
function.
Equations
- One or more equations did not get rendered due to their size.
Delaborate a call to a projection function such as Prod.fst
.
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.
Equations
- One or more equations did not get rendered due to their size.