Equations
- Lean.Parser.optional p = Lean.Parser.optionalNoAntiquot (Lean.Parser.withAntiquotSpliceAndSuffix `optional p (Lean.Parser.symbol "?"))
Equations
- Lean.Parser.many p = Lean.Parser.manyNoAntiquot (Lean.Parser.withAntiquotSpliceAndSuffix `many p (Lean.Parser.symbol "*"))
Equations
- Lean.Parser.many1 p = Lean.Parser.many1NoAntiquot (Lean.Parser.withAntiquotSpliceAndSuffix `many p (Lean.Parser.symbol "*"))
Equations
Equations
Equations
- Lean.Parser.many1Indent p = Lean.Parser.withPosition (Lean.Parser.many1 (HAndThen.hAndThen (Lean.Parser.checkColGe "irrelevant") fun x => p))
Equations
- Lean.Parser.manyIndent p = Lean.Parser.withPosition (Lean.Parser.many (HAndThen.hAndThen (Lean.Parser.checkColGe "irrelevant") fun x => p))
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
No-op parser that advises the pretty printer to emit a non-breaking space.
Equations
No-op parser that advises the pretty printer to emit a space/soft line break.
Equations
No-op parser that advises the pretty printer to emit a hard line break.
Equations
No-op parser combinator that advises the pretty printer to emit a Format.fill
node.
Equations
No-op parser combinator that advises the pretty printer to emit a Format.group
node.
Equations
No-op parser combinator that advises the pretty printer to indent the given syntax without grouping it.
Equations
No-op parser combinator that advises the pretty printer to group and indent the given syntax. By default, only syntax categories are grouped.
Equations
No-op parser combinator that advises the pretty printer to dedent the given syntax. Dedenting can in particular be used to counteract automatic indentation.
Equations
No-op parser combinator that allows the pretty printer to omit the group and indent operation in the enclosing category parser.
syntax ppAllowUngrouped "by " tacticSeq : term
-- allows a `by` after `:=` without linebreak in between:
theorem foo : True := by
trivial
No-op parser combinator that advises the pretty printer to dedent the given syntax, if it was grouped by the category parser. Dedenting can in particular be used to counteract automatic indentation.
Equations
No-op parser combinator that prints a line break. The line break is soft if the combinator is followed by an ungrouped parser (see ppAllowUngrouped), otherwise hard.
Equations
- Lean.ppDedent.formatter p = do let opts ← Lean.getOptions Lean.PrettyPrinter.Formatter.indent p (some (0 - Int.ofNat (Std.Format.getIndent opts)))
Equations
- Lean.ppAllowUngrouped.formatter = modify fun a => { stxTrav := a.stxTrav, leadWord := a.leadWord, isUngrouped := a.isUngrouped, mustBeGrouped := false, stack := a.stack }
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.ppHardLineUnlessUngrouped.formatter = do let a ← get if a.isUngrouped = true then Lean.PrettyPrinter.Formatter.pushLine else Lean.ppLine.formatter
Equations
- One or more equations did not get rendered due to their size.