Idris2/tests/idris2/coverage019/Issue1632.idr

15 lines
249 B
Idris
Raw Normal View History

%default total
data Command : Type -> Type where
Empty : Command ()
Pure : t -> Command t
test : Command (List a) -> ()
test (Pure x) = ()
test2 : Command (a -> b) -> ()
test2 (Pure x) = ()
test3 : Command Type -> ()
test3 (Pure x) = ()