Documentation

Lean.Elab.Tactic.Do.Spec

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 : TypeType u_1} [Monad n] [MonadControlT MetaM n] [MonadLiftT MetaM n] (α ps Q Q' : Expr) (goalTag : Name) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          partial def Lean.Elab.Tactic.Do.dischargeFailEntails {n : TypeType u_1} [Monad n] [MonadControlT MetaM n] [MonadLiftT MetaM n] (ps Q Q' : Expr) (goalTag : Name) :
          def Lean.Elab.Tactic.Do.dischargeMGoal {n : TypeType u_1} [Monad n] [MonadLiftT MetaM n] (goal : ProofMode.MGoal) (goalTag : Name) :
          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 : TypeType u_1} [Monad n] [MonadControlT MetaM n] [MonadLiftT MetaM n] (goal : ProofMode.MGoal) (elabSpecAtWP : Exprn SpecAttr.SpecTheorem) (goalTag : Name) (mkPreTag : NameName := 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.
                Instances For