@[export lean_mk_antiquot_parenthesizer]
def
Lean.PrettyPrinter.Parenthesizer.mkAntiquot.parenthesizer
(name : String)
(kind : Lean.SyntaxNodeKind)
(anonymous isPseudoKind : Bool := true)
:
Equations
- Lean.PrettyPrinter.Parenthesizer.mkAntiquot.parenthesizer name kind anonymous isPseudoKind = Lean.Parser.mkAntiquot.parenthesizer name kind anonymous isPseudoKind
Instances For
@[export lean_pretty_printer_parenthesizer_interpret_parser_descr]
Equations
- One or more equations did not get rendered due to their size.
- Lean.PrettyPrinter.Parenthesizer.interpretParserDescr (Lean.ParserDescr.const n) = liftM (Lean.Parser.getConstAlias Lean.PrettyPrinter.Parenthesizer.parenthesizerAliasesRef n)
- Lean.PrettyPrinter.Parenthesizer.interpretParserDescr (Lean.ParserDescr.symbol tk) = pure (Lean.Parser.symbol.parenthesizer tk)
- Lean.PrettyPrinter.Parenthesizer.interpretParserDescr (Lean.ParserDescr.nonReservedSymbol tk includeIdent) = pure (Lean.Parser.nonReservedSymbol.parenthesizer tk includeIdent)
- Lean.PrettyPrinter.Parenthesizer.interpretParserDescr (Lean.ParserDescr.parser constName) = Lean.PrettyPrinter.combinatorParenthesizerAttribute.runDeclFor constName
- Lean.PrettyPrinter.Parenthesizer.interpretParserDescr (Lean.ParserDescr.cat catName prec) = pure (Lean.PrettyPrinter.Parenthesizer.categoryParser.parenthesizer catName prec)
Instances For
@[export lean_mk_antiquot_formatter]
def
Lean.PrettyPrinter.Formatter.mkAntiquot.formatter
(name : String)
(kind : Lean.SyntaxNodeKind)
(anonymous isPseudoKind : Bool := true)
:
Equations
- Lean.PrettyPrinter.Formatter.mkAntiquot.formatter name kind anonymous isPseudoKind = Lean.Parser.mkAntiquot.formatter name kind anonymous isPseudoKind
Instances For
@[export lean_pretty_printer_formatter_interpret_parser_descr]
Equations
- One or more equations did not get rendered due to their size.
- Lean.PrettyPrinter.Formatter.interpretParserDescr (Lean.ParserDescr.const n) = liftM (Lean.Parser.getConstAlias Lean.PrettyPrinter.Formatter.formatterAliasesRef n)
- Lean.PrettyPrinter.Formatter.interpretParserDescr (Lean.ParserDescr.symbol tk) = pure (Lean.Parser.symbol.formatter tk)
- Lean.PrettyPrinter.Formatter.interpretParserDescr (Lean.ParserDescr.nonReservedSymbol tk includeIdent) = pure (Lean.Parser.nonReservedSymbol.formatter tk)
- Lean.PrettyPrinter.Formatter.interpretParserDescr (Lean.ParserDescr.parser constName) = Lean.PrettyPrinter.combinatorFormatterAttribute.runDeclFor constName
- Lean.PrettyPrinter.Formatter.interpretParserDescr (Lean.ParserDescr.cat catName prec) = pure (Lean.PrettyPrinter.Formatter.categoryParser.formatter catName)