grind parameter elaboration
def
Lean.Elab.Tactic.addEMatchTheorem
(params : Meta.Grind.Params)
(id : Ident)
(declName : Name)
(kind : Meta.Grind.EMatchTheoremKind)
(minIndexable : Bool)
(suggest : Bool := false)
(warn : Bool := true)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.Tactic.elabGrindParams
(params : Meta.Grind.Params)
(ps : TSyntaxArray `Lean.Parser.Tactic.grindParam)
(only : Bool)
(lax incremental : Bool := false)
:
Elaborates grind parameters.
incremental = true for tactics such as finish, in this case, we disable some kinds of parameters
such as - ident.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.Tactic.Grind.withParams
{α : Type}
(params : Meta.Grind.Params)
(ps : TSyntaxArray `Lean.Parser.Tactic.grindParam)
(only : Bool)
(k : GrindTacticM α)
:
Helper method for processing parameters in tactics such as finish and finish?
Equations
- One or more equations did not get rendered due to their size.