@[match_pattern]
Equations
Instances For
@[match_pattern]
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Lean.Elab.Tactic.Do.ProofMode.parseHyp? x✝ = none
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
Equations
- One or more equations did not get rendered due to their size.
- Lean.Elab.Tactic.Do.ProofMode.parseEmptyHyp? x✝ = none
Instances For
Equations
Instances For
Equations
Instances For
Combine two hypotheses into a conjunction.
Precondition: Neither lhs
nor rhs
is empty (parseEmptyHyp?
).
Equations
- Lean.Elab.Tactic.Do.ProofMode.mkAnd! σs lhs rhs = Lean.mkApp3 (Lean.mkConst `Std.Do.SPred.and) σs lhs rhs
Instances For
Equations
Instances For
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- goal.strip = Lean.mkApp3 (Lean.mkConst `Std.Do.SPred.entails) goal.σs goal.hyps goal.target
Instances For
Roundtrips with parseMGoal?
.
Equations
- goal.toExpr = Lean.mkApp3 (Lean.mkConst `Std.Tactic.Do.MGoalEntails) goal.σs goal.hyps goal.target
Instances For
Equations
- goal.findHyp? name = Lean.Elab.Tactic.Do.ProofMode.MGoal.findHyp?.go name goal.hyps Lean.SubExpr.Pos.root
Instances For
partial def
Lean.Elab.Tactic.Do.ProofMode.MGoal.findHyp?.go
(name : Name)
(e : Expr)
(p : SubExpr.Pos)
: