Documentation

Lean.Meta.AbstractNestedProofs

def Lean.Meta.abstractProof {m : TypeType} [Monad m] [MonadLiftT MetaM m] [MonadEnv m] [MonadOptions m] [MonadFinally m] (proof : Expr) (cache : Bool := true) (postprocessType : Exprm Expr := pure) :

Abstracts the given proof into an auxiliary theorem, suitably pre-processing its type.

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

      Replace proofs nested in e with new lemmas. The new lemmas are named using getDeclNGen.

      Equations
      Instances For