Equations
- One or more equations did not get rendered due to their size.
Instances For
@[inline]
Instances For
@[inline]
Equations
- Lean.Json.Parser.natNonZero = do Lean.Json.Parser.lookahead (fun (c : Char) => (decide ('1' ≤ c) && decide (c ≤ '9')) = true) "1-9" Lean.Json.Parser.natCore 0
Instances For
@[inline]
Equations
- Lean.Json.Parser.natNumDigits = do Lean.Json.Parser.lookahead (fun (c : Char) => (decide ('0' ≤ c) && decide (c ≤ '9')) = true) "digit" Lean.Json.Parser.natCoreNumDigits 0 0
Instances For
@[inline]
Instances For
@[inline]
Equations
Instances For
@[inline]
Instances For
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
partial def
Lean.Json.Parser.objectCore
(kvs : Lean.RBNode String fun (x : String) => Lean.Json)
:
Std.Internal.Parsec.String.Parser (Lean.RBNode String fun (x : String) => Lean.Json)
Equations
- Lean.Json.Parser.any = do Std.Internal.Parsec.String.ws let res ← Lean.Json.Parser.anyCore Std.Internal.Parsec.eof pure res
Instances For
Equations
- Lean.Json.parse s = Lean.Json.Parser.any.run s