Idris2/tests/idris2/basic003/Ambig1.idr
Edwin Brady a972778eab Add test script
They don't all pass yet, for minor reasons. Coming shortly...
Unfortunately the startup overhead for chez is really noticeable here!
2020-05-19 18:25:18 +01:00

23 lines
346 B
Idris

data Things : Type where
MkThings : a -> a -> Things
namespace X
public export
data Test = A | B
namespace Y
public export
data TestType = Test | Baz
test1 : Things
test1 = MkThings Baz Test
test2 : Things
test2 = MkThings Int Test
test3 : Integer -> Things
test3 x = MkThings Test Baz
test4 : Things
test4 = MkThings Test Int