- impl : AttributeImpl
Instances For
Equations
- Lean.ParserCompiler.instInhabitedCombinatorAttribute = { default := { impl := default, ext := default } }
def
Lean.ParserCompiler.registerCombinatorAttribute
(name : Name)
(descr : String)
(ref : Name := by exact decl_name%)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.ParserCompiler.CombinatorAttribute.getDeclFor?
(attr : CombinatorAttribute)
(env : Environment)
(parserDecl : Name)
:
Equations
- attr.getDeclFor? env parserDecl = (attr.ext.getState env).find? parserDecl
Instances For
def
Lean.ParserCompiler.CombinatorAttribute.setDeclFor
(attr : CombinatorAttribute)
(env : Environment)
(parserDecl decl : Name)
:
Equations
- attr.setDeclFor env parserDecl decl = Lean.PersistentEnvExtension.addEntry attr.ext env (parserDecl, decl)
Instances For
unsafe def
Lean.ParserCompiler.CombinatorAttribute.runDeclFor
{α : Type}
(attr : CombinatorAttribute)
(parserDecl : Name)
:
CoreM α
Equations
- One or more equations did not get rendered due to their size.