Documentation

Lean.Elab.Tactic.Do.ProofMode.Frame

If P' is a conjunction of unnamed hypotheses that are a subset of the named hypotheses of P, transfer the names of the hypotheses of P to the hypotheses of P'.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def Lean.Elab.Tactic.Do.ProofMode.mFrameCore {m : TypeType u_1} {α : Type} [Monad m] [MonadControlT MetaM m] [MonadLiftT MetaM m] (goal : MGoal) (kFail : m (α × Expr)) (kSuccess : ExprExprMGoalm (α × Expr)) :
    m (α × Expr)
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      def Lean.Elab.Tactic.Do.ProofMode.mTryFrame {m : TypeType u_1} {α : Type} [Monad m] [MonadControlT MetaM m] [MonadLiftT MetaM m] (goal : MGoal) (k : MGoalm (α × Expr)) :
      m (α × Expr)
      Equations
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For