Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.withPPInaccessibleNames
{m : Type → Type u_1}
{α : Type}
[inst : MonadControlT Lean.MetaM m]
[inst : Monad m]
(x : m α)
(flag : optParam Bool true)
:
m α
Equations
- Lean.Meta.withPPInaccessibleNames x flag = Lean.Meta.mapMetaM (fun {α} => Lean.Meta.withPPInaccessibleNamesImp flag) x
@[inline]
Equations
- Lean.Meta.ToHide.isMarked fvarId = do let s ← get pure (Std.RBTree.contains s.hiddenInaccessible fvarId || Std.RBTree.contains s.hiddenInaccessibleProp fvarId)
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
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.Meta.getGoalPrefix mvarDecl = if Option.isSome (Lean.isLHSGoal? mvarDecl.type) = true then "| " else "⊢ "
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.ppGoal.pushPending
(indent : Int)
(ids : List Lean.Name)
(type? : Option Lean.Expr)
(fmt : Lean.Format)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.ppGoal.ppVars
(indent : Int)
(hiddenProp : Lean.FVarIdSet)
(varNames : List Lean.Name)
(prevType? : Option Lean.Expr)
(fmt : Lean.Format)
(localDecl : Lean.LocalDecl)
:
Equations
- One or more equations did not get rendered due to their size.