Documentation

Lean.Elab.Tactic.Do.ProofMode.Intro

def Lean.Elab.Tactic.Do.ProofMode.mIntro {m : TypeType u_1} {α : Type} [Monad m] [MonadControlT MetaM m] (goal : MGoal) (ident : TSyntax `Lean.binderIdent) (k : MGoalm (α × Expr)) :
m (α × Expr)
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def Lean.Elab.Tactic.Do.ProofMode.mIntroForall {m : TypeType u_1} {α : Type} [Monad m] [MonadControlT MetaM m] [MonadLiftT MetaM m] (goal : MGoal) (ident : TSyntax `Lean.binderIdent) (k : MGoalm (α × Expr)) :
    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 : TypeType u_1} {α : Type} [Monad m] [MonadControlT MetaM m] [MonadLiftT MetaM m] (goal : MGoal) (n : Nat) (k : MGoalm (α × Expr)) :
      m (α × Expr)
      Equations
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For