def
Lean.Elab.Tactic.Do.ProofMode.mIntroForall
{m : Type → Type u_1}
{α : Type}
[Monad m]
[MonadControlT MetaM m]
[MonadLiftT MetaM m]
(goal : MGoal)
(ident : TSyntax `Lean.binderIdent)
(k : MGoal → m (α × Expr))
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Elab.Tactic.Do.ProofMode.mIntroForallN
{m : Type → Type u_1}
{α : Type}
[Monad m]
[MonadControlT MetaM m]
[MonadLiftT MetaM m]
(goal : MGoal)
(n : Nat)
(k : MGoal → m (α × Expr))
:
Equations
- One or more equations did not get rendered due to their size.
- Lean.Elab.Tactic.Do.ProofMode.mIntroForallN goal 0 k = k goal
Instances For
Equations
- One or more equations did not get rendered due to their size.