Idris2/libs/contrib/Language/JSON.idr
2020-05-18 14:00:08 +01:00

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)