mirror of
https://github.com/luau-lang/luau.git
synced 2024-11-15 22:35:43 +08:00
041838a942
* First cut reading JSON into an Agda representation of Luau syntax
17 lines
449 B
Agda
17 lines
449 B
Agda
module FFI.Data.HaskellString where
|
|
|
|
open import Agda.Builtin.String using (String)
|
|
|
|
{-# FOREIGN GHC import qualified Data.String #-}
|
|
{-# FOREIGN GHC import qualified Data.Text #-}
|
|
|
|
postulate HaskellString : Set
|
|
{-# COMPILE GHC HaskellString = type Data.String.String #-}
|
|
|
|
postulate pack : HaskellString → String
|
|
{-# COMPILE GHC pack = Data.Text.pack #-}
|
|
|
|
postulate unpack : String → HaskellString
|
|
{-# COMPILE GHC unpack = Data.Text.unpack #-}
|
|
|