def
Lean.Elab.Command.expandNotationItemIntoSyntaxItem:
Lean.TSyntax `Lean.Parser.Command.notationItem → Lean.MacroM (Lean.TSyntax `stx)
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
- 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.
def
Lean.Elab.Command.mkSimpleDelab
(attrKind : Lean.TSyntax `Lean.Parser.Term.attrKind)
(pat : Lean.Term)
(qrhs : Lean.Term)
:
Try to derive a SimpleDelab from a notation.
The notation must be of the form notation ... => c body
where c is a declaration in the current scope and body any syntax
that contains each variable from the LHS at most once.
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.