def
Lean.Elab.checkNotAlreadyDeclared
{m : Type → Type}
[inst : Monad m]
[inst : Lean.MonadEnv m]
[inst : Lean.MonadError m]
(declName : Lean.Name)
:
m Unit
Equations
- One or more equations did not get rendered due to their size.
- regular: Lean.Elab.Visibility
- protected: Lean.Elab.Visibility
- private: Lean.Elab.Visibility
Declaration visibility modifier. That is, whether a declaration is regular, protected or private.
Equations
- Lean.Elab.instInhabitedVisibility = { default := Lean.Elab.Visibility.regular }
Equations
- One or more equations did not get rendered due to their size.
- partial: Lean.Elab.RecKind
- nonrec: Lean.Elab.RecKind
- default: Lean.Elab.RecKind
Whether a declaration is default, partial or nonrec.
Equations
- Lean.Elab.instInhabitedRecKind = { default := Lean.Elab.RecKind.partial }
- visibility : Lean.Elab.Visibility
- isNoncomputable : Bool
- recKind : Lean.Elab.RecKind
- isUnsafe : Bool
- attrs : Array Lean.Elab.Attribute
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.
def
Lean.Elab.Modifiers.addAttribute
(modifiers : Lean.Elab.Modifiers)
(attr : Lean.Elab.Attribute)
:
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
- Lean.Elab.instToStringModifiers = { toString := toString ∘ Lean.format }
def
Lean.Elab.expandOptDocComment?
{m : Type → Type}
[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 : Type → Type}
[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 : Type → Type}
[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 : Type → Type}
[inst : Monad m]
[inst : Lean.MonadEnv m]
[inst : Lean.MonadError m]
(declName : Lean.Name)
:
m Unit
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.mkDeclName
{m : Type → Type}
[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 : Type → Type}
[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.