def
Lean.Elab.Tactic.Do.ProofMode.patAsTerm
(pat : Parser.Tactic.MRefinePat)
(expected : Option Expr := none)
:
Equations
- One or more equations did not get rendered due to their size.
- Lean.Elab.Tactic.Do.ProofMode.patAsTerm (Lean.Parser.Tactic.MRefinePat.pure t) expected = liftM (Lean.Elab.Tactic.elabTerm t.raw expected)
- Lean.Elab.Tactic.Do.ProofMode.patAsTerm pat expected = failure
Instances For
partial def
Lean.Elab.Tactic.Do.ProofMode.mRefineCore
(goal : MGoal)
(pat : Parser.Tactic.MRefinePat)
(k : MGoal → TSyntax `Lean.binderIdent → TacticM Expr)
:
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.