Documentation

Lean.Exception

Equations
  • One or more equations did not get rendered due to their size.
Equations
instance Lean.instAddErrorMessageContext (m : TypeType) [inst : Lean.AddMessageContext m] [inst : Monad m] :
Equations
def Lean.throwError {m : TypeType} {α : Type} [inst : Monad m] [inst : Lean.MonadError m] (msg : Lean.MessageData) :
m α
Equations
def Lean.throwUnknownConstant {m : TypeType} {α : Type} [inst : Monad m] [inst : Lean.MonadError m] (constName : Lean.Name) :
m α
Equations
def Lean.throwErrorAt {m : TypeType} {α : Type} [inst : Monad m] [inst : Lean.MonadError m] (ref : Lean.Syntax) (msg : Lean.MessageData) :
m α
Equations
def Lean.ofExcept {m : TypeType} {ε : Type u_1} {α : Type} [inst : Monad m] [inst : Lean.MonadError m] [inst : ToString ε] (x : Except ε α) :
m α
Equations
def Lean.throwKernelException {m : TypeType} {α : Type} [inst : Monad m] [inst : Lean.MonadError m] [inst : Lean.MonadOptions m] (ex : Lean.KernelException) :
m α
Equations
instance Lean.instMonadRecDepthReaderT {m : TypeType} {ρ : Type} [inst : Monad m] [inst : Lean.MonadRecDepth m] :
Equations
  • One or more equations did not get rendered due to their size.
instance Lean.instMonadRecDepthStateRefT' {m : TypeType} {ω : Type} {σ : Type} [inst : Monad m] [inst : Lean.MonadRecDepth m] :
Equations
instance Lean.instMonadRecDepthMonadCacheT {α : Type} {m : TypeType} {ω : Type} {β : Type} [inst : BEq α] [inst : Hashable α] [inst : Monad m] [inst : STWorld ω m] [inst : Lean.MonadRecDepth m] :
Equations

Return true if ex was generated by throwMaxRecDepthAt. This function is a bit hackish. The max rec depth exception should probably be an internal exception, but it is also produced by MacroM which implemented in the prelude, and internal exceptions have not been defined yet.

Equations
@[inline]
def Lean.withIncRecDepth {m : TypeType} {α : Type} [inst : Monad m] [inst : Lean.MonadError m] [inst : Lean.MonadRecDepth m] (x : m α) :
m α
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.
Equations
  • One or more equations did not get rendered due to their size.