Documentation

Lean.Elab.Util

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.
def Lean.Elab.addMacroStack {m : TypeType} [inst : Monad m] [inst : Lean.MonadOptions m] (msgData : Lean.MessageData) (macroStack : Lean.Elab.MacroStack) :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.checkSyntaxNodeKind {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] [inst : Lean.MonadError m] (k : Lean.Name) :
Equations
Equations
  • One or more equations did not get rendered due to their size.
@[implementedBy _private.Lean.Elab.Util.0.Lean.Elab.evalSyntaxConstantUnsafe]
unsafe def Lean.Elab.mkElabAttribute (γ : Type) (attrDeclName : Lean.Name) (attrBuiltinName : Lean.Name) (attrName : Lean.Name) (parserNamespace : Lean.Name) (typeName : Lean.Name) (kind : String) :
Equations
  • One or more equations did not get rendered due to their size.
@[implementedBy Lean.Elab.mkMacroAttributeUnsafe]

Try to expand macro at syntax tree root and return macro declaration name and new syntax if successful. Return none if all macros threw Macro.Exception.unsupportedSyntax.

Equations
  • One or more equations did not get rendered due to their size.
instance Lean.Elab.instMonadMacroAdapter (m : TypeType) (n : TypeType) [inst : MonadLift m n] [inst : Lean.Elab.MonadMacroAdapter m] :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.liftMacroM {α : Type} {m : TypeType} [inst : Monad m] [inst : Lean.Elab.MonadMacroAdapter m] [inst : Lean.MonadEnv m] [inst : Lean.MonadRecDepth m] [inst : Lean.MonadError m] [inst : Lean.MonadResolveName m] [inst : Lean.MonadTrace m] [inst : Lean.MonadOptions m] [inst : Lean.AddMessageContext m] (x : Lean.MacroM α) :
m α
Equations
  • One or more equations did not get rendered due to their size.
@[inline]
def Lean.Elab.adaptMacro {m : TypeType} [inst : Monad m] [inst : Lean.Elab.MonadMacroAdapter m] [inst : Lean.MonadEnv m] [inst : Lean.MonadRecDepth m] [inst : Lean.MonadError m] [inst : Lean.MonadResolveName m] [inst : Lean.MonadTrace m] [inst : Lean.MonadOptions m] [inst : Lean.AddMessageContext m] (x : Lean.Macro) (stx : Lean.Syntax) :
Equations
Equations
  • One or more equations did not get rendered due to their size.
partial def Lean.Elab.mkUnusedBaseName.loop (baseName : Lean.Name) (currNamespace : Lean.Name) (idx : Nat) :
def Lean.Elab.logException {m : TypeType} [inst : Monad m] [inst : Lean.MonadLog m] [inst : Lean.AddMessageContext m] [inst : MonadLiftT IO m] (ex : Lean.Exception) :
Equations
  • One or more equations did not get rendered due to their size.
@[inline]
def Lean.Elab.trace {m : TypeType} [inst : Monad m] [inst : Lean.MonadLog m] [inst : Lean.AddMessageContext m] [inst : Lean.MonadOptions m] (cls : Lean.Name) (msg : UnitLean.MessageData) :
Equations
def Lean.Elab.logDbgTrace {m : TypeType} [inst : Monad m] [inst : Lean.MonadLog m] [inst : Lean.AddMessageContext m] [inst : Lean.MonadOptions m] (msg : Lean.MessageData) :
Equations
def Lean.Elab.nestedExceptionToMessageData {m : TypeType} [inst : Monad m] [inst : Lean.MonadLog m] (ex : Lean.Exception) :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.throwErrorWithNestedErrors {m : TypeType} {α : Type} [inst : Lean.MonadError m] [inst : Monad m] [inst : Lean.MonadLog m] (msg : Lean.MessageData) (exs : Array Lean.Exception) :
m α
Equations
  • One or more equations did not get rendered due to their size.