Maps declaration names to α
.
Equations
Instances For
Look up a value in the given extension in the environment.
Equations
- ext.find? env = (Lean.SimplePersistentEnvExtension.getState ext env).find?
Instances For
def
Lean.NameMapExtension.add
{M : Type → Type}
{α : Type}
[Monad M]
[MonadEnv M]
[MonadError M]
(ext : NameMapExtension α)
(k : Name)
(v : α)
:
M Unit
Add the given k,v pair to the NameMapExtension.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.registerNameMapExtension
(α : Type)
(name : Name := by exact decl_name%)
:
IO (NameMapExtension α)
Registers a new extension with the given name and type.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The inputs to registerNameMapAttribute
.
- name : Name
The name of the attribute
- ref : Name
The declaration which creates the attribute
- descr : String
The description of the attribute
This function is called when the attribute is applied. It should produce a value of type
α
from the given attribute syntax.
Instances For
def
Lean.registerNameMapAttribute
{α : Type}
(impl : NameMapAttributeImpl α)
:
IO (NameMapExtension α)
Similar to registerParametricAttribute
except that attributes do not
have to be assigned in the same file as the declaration.
Equations
- One or more equations did not get rendered due to their size.