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.
Instances For
def
Lean.Elab.Tactic.Do.dischargePostEntails
{n : Type → Type u_1}
[Monad n]
[MonadControlT MetaM n]
[MonadLiftT MetaM n]
(α ps Q Q' : Expr)
(goalTag : Name)
:
n Expr
Equations
- One or more equations did not get rendered due to their size.
Instances For
partial def
Lean.Elab.Tactic.Do.dischargeFailEntails
{n : Type → Type u_1}
[Monad n]
[MonadControlT MetaM n]
[MonadLiftT MetaM n]
(ps Q Q' : Expr)
(goalTag : Name)
:
n Expr
def
Lean.Elab.Tactic.Do.dischargeMGoal
{n : Type → Type u_1}
[Monad n]
[MonadLiftT MetaM n]
(goal : ProofMode.MGoal)
(goalTag : Name)
:
n 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.
Instances For
def
Lean.Elab.Tactic.Do.mSpec
{n : Type → Type u_1}
[Monad n]
[MonadControlT MetaM n]
[MonadLiftT MetaM n]
(goal : ProofMode.MGoal)
(elabSpecAtWP : Expr → n SpecAttr.SpecTheorem)
(goalTag : Name)
(mkPreTag : Name → Name := mkPreTag)
:
Returns the proof and the list of new unassigned MVars.
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.