Equations
Equations
- One or more equations did not get rendered due to their size.
partial def
Lean.Parser.interpolatedStrFn.parse
(p : Lean.Parser.ParserFn)
(input : String)
(stackSize : Nat)
(startPos : String.Pos)
(c : Lean.Parser.ParserContext)
(s : Lean.Parser.ParserState)
:
@[inline]
Equations
- Lean.Parser.interpolatedStrNoAntiquot p = { info := Lean.Parser.mkAtomicInfo "interpolatedStr", fn := Lean.Parser.interpolatedStrFn p.fn }
Equations
- Lean.Parser.interpolatedStr p = Lean.Parser.withAntiquot (Lean.Parser.mkAntiquot "interpolatedStr" Lean.interpolatedStrKind true) (Lean.Parser.interpolatedStrNoAntiquot p)