- attr : Lean.AttributeImpl
Instances For
Equations
- Lake.instInhabitedOrderedTagAttribute = { default := { attr := default, ext := default } }
def
Lake.registerOrderedTagAttribute
(name : Lean.Name)
(descr : String)
(validate : Lean.Name → Lean.AttrM Unit := fun (x : Lean.Name) => pure ())
(ref : Lean.Name := by exact decl_name%)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lake.OrderedTagAttribute.hasTag
(attr : Lake.OrderedTagAttribute)
(env : Lean.Environment)
(decl : Lean.Name)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lake.OrderedTagAttribute.getAllEntries
(attr : Lake.OrderedTagAttribute)
(env : Lean.Environment)
:
Get all tagged declaration names, both those imported and those in the current module.
Equations
- attr.getAllEntries env = Array.flatMap id (attr.ext.toEnvExtension.getState env).importedEntries ++ (attr.ext.toEnvExtension.getState env).state