mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-16 15:52:43 +03:00
a972778eab
They don't all pass yet, for minor reasons. Coming shortly... Unfortunately the startup overhead for chez is really noticeable here!
18 lines
468 B
Idris
18 lines
468 B
Idris
data ErlList : List Type -> Type where
|
|
Nil : ErlList []
|
|
(::) : x -> ErlList xs -> ErlList (x :: xs)
|
|
|
|
data ErlType : Type -> Type where
|
|
ETInteger : ErlType Integer
|
|
ETString : ErlType String
|
|
|
|
data ErlTypes : List Type -> Type where
|
|
ETErlTypesNil : ErlTypes []
|
|
ETErlTypesCons : (ErlType x, ErlTypes xs) => ErlTypes (x :: xs)
|
|
|
|
erlCall : ErlList xs -> {auto prf : ErlTypes xs} -> ()
|
|
erlCall args = ()
|
|
|
|
foo : ()
|
|
foo = erlCall [1,2,3, "foo", "bar", "baz", 4,5,6]
|