mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-01 09:49:24 +03:00
15 lines
279 B
Idris
15 lines
279 B
Idris
||| The JSON language, as described at https://json.org/
|
|
module Language.JSON
|
|
|
|
import Language.JSON.Lexer
|
|
import Language.JSON.Parser
|
|
|
|
import public Language.JSON.Data
|
|
|
|
%default total
|
|
|
|
||| Parse a JSON string.
|
|
export
|
|
parse : String -> Maybe JSON
|
|
parse x = parseJSON !(lexJSON x)
|