Documentation

Lean.Elab.Tactic.Do.ProofMode.Revert

def Lean.Elab.Tactic.Do.ProofMode.mRevert {m : TypeType u} [Monad m] [MonadLiftT MetaM m] (goal : MGoal) (ref : TSyntax `ident) (k : MGoalm Expr) :
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def Lean.Elab.Tactic.Do.ProofMode.mRevertForallN {m : TypeType u} [Monad m] [MonadControlT MetaM m] [MonadLiftT MetaM m] (goal : MGoal) (n : Nat) (hypName : Name) (k : MGoalm Expr) :

    Turn goal hᵢ : Hᵢ ⊢ₛ T e₁ ... eₙ into hᵢ : fun sₙ ... s₁ => Hᵢ h : fun sₙ ... s₁ => ⌜s₁ = e₁ ∧ ... ∧ sₙ = eₙ⌝ ⊢ₛ T

    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