- config : Grind.Config
- ematch : EMatchTheorems
- inj : InjectiveTheorems
- symPrios : SymbolPriorities
- casesTypes : CasesTypes
- extra : PArray EMatchTheorem
- norm : Simp.Context
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Meta.Grind.GrindM.run
{α : Type}
(x : GrindM α)
(params : Params)
(evalTactic? : Option EvalTactic := none)
:
MetaM α
Equations
- One or more equations did not get rendered due to their size.
Instances For
- issues : List MessageData
- config : Grind.Config
- trace : Trace
- counters : Counters
- simp : Simp.Stats
- splitDiags : PArray SplitDiagInfo
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Meta.Grind.GrindM.runAtGoal
{α : Type}
(mvarId : MVarId)
(params : Params)
(k : Goal → GrindM α)
(evalTactic? : Option EvalTactic := none)
:
MetaM α
Equations
- Lean.Meta.Grind.GrindM.runAtGoal mvarId params k evalTactic? = (Lean.Meta.withReducible do let goal ← Lean.Meta.Grind.initCore✝ mvarId params k goal).run params evalTactic?