Idris2/tests/idris2/basic035/using.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

20 lines
386 B
Idris

import Data.Vect
using (Show a, Eq a)
foo : a -> String
foo x = show x ++ show x
bar : Int -> Int
bar x = x + x
using (xs : Vect n a, n : Nat) -- get reordered in dependency order by
-- the usual implicit rules
baz : xs = xs
data Test : Type -> Type -> Type where
using (Test a b)
needle : a -> b -> ()
nardle : a -> ()
noo : b -> ()