Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Meta.Grind.GrindM.run
{α : Type}
(x : GrindM α)
(mainDeclName : Name)
(config : Grind.Config)
(fallback : Fallback)
:
MetaM α
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Meta.Grind.all goals f = List.foldlM (fun (acc : List Lean.Meta.Grind.Goal) (goal : Lean.Meta.Grind.Goal) => do let __do_lift ← f goal pure (acc ++ __do_lift)) [] goals
Instances For
def
Lean.Meta.Grind.main
(mvarId : MVarId)
(config : Grind.Config)
(mainDeclName : Name)
(fallback : Fallback)
:
Equations
- One or more equations did not get rendered due to their size.