Documentation

Lean.Elab.DeclModifiers

def Lean.Elab.checkNotAlreadyDeclared {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] [inst : Lean.MonadError m] (declName : Lean.Name) :
Equations
  • One or more equations did not get rendered due to their size.
inductive Lean.Elab.Visibility:
Type

Declaration visibility modifier. That is, whether a declaration is regular, protected or private.

Equations
  • One or more equations did not get rendered due to their size.
inductive Lean.Elab.RecKind:
Type

Whether a declaration is default, partial or nonrec.

structure Lean.Elab.Modifiers:
Type

Flags and data added to declarations (eg docstrings, attributes, private, unsafe, partial, ...).

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.
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.
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.expandOptDocComment? {m : TypeType} [inst : Monad m] [inst : Lean.MonadError m] (optDocComment : Lean.Syntax) :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.elabModifiers {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] [inst : Lean.MonadResolveName m] [inst : Lean.MonadError m] [inst : Lean.Elab.MonadMacroAdapter m] [inst : Lean.MonadRecDepth m] [inst : Lean.MonadTrace m] [inst : Lean.MonadOptions m] [inst : Lean.AddMessageContext m] (stx : Lean.Syntax) :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.applyVisibility {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] [inst : Lean.MonadError m] (visibility : Lean.Elab.Visibility) (declName : Lean.Name) :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.checkIfShadowingStructureField {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] [inst : Lean.MonadError m] (declName : Lean.Name) :
Equations
  • One or more equations did not get rendered due to their size.
def Lean.Elab.mkDeclName {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] [inst : Lean.MonadError m] (currNamespace : Lean.Name) (modifiers : Lean.Elab.Modifiers) (shortName : Lean.Name) :
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.expandDeclId {m : TypeType} [inst : Monad m] [inst : Lean.MonadEnv m] [inst : Lean.MonadError m] (currNamespace : Lean.Name) (currLevelNames : List Lean.Name) (declId : Lean.Syntax) (modifiers : Lean.Elab.Modifiers) :
Equations
  • One or more equations did not get rendered due to their size.