Documentation

Lake.Util.OrderedTagAttribute

def Lake.registerOrderedTagAttribute (name : Lean.Name) (descr : String) (validate : Lean.NameLean.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
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      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
      Instances For