Equations
- Lean.Elab.instInhabitedAttribute = { default := { kind := default, name := default, stx := default } }
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.mkAttrKindGlobal = (Lean.mkNode `Lean.Parser.Term.attrKind #[Lean.mkNullNode]).raw
def
Lean.Elab.elabAttr
{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]
(attrInstance : Lean.Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.elabAttrs
{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]
(attrInstances : Array Lean.Syntax)
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Elab.elabDeclAttrs
{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)
: