Idris2/tests/idris2/reg015/anyfail.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

22 lines
697 B
Idris

data SimpleData = PtrAndSize AnyPtr Int
record Complicated where
constructor MkComplicated
simple : SimpleData
record MoreComplicated where
constructor MkMoreComplicated
something : Complicated
record EvenMoreComplicated where
constructor MkEvenMoreComplicated
somethingEven : MoreComplicated
data TooComplicatedToBeTrue : (something : EvenMoreComplicated) -> Type where
SomethingVeryComplicatedIs :
TooComplicatedToBeTrue
(MkEvenMoreComplicated (MkMoreComplicated (MkComplicated (PtrAndSize addr len))))
showing : (something : EvenMoreComplicated) -> (TooComplicatedToBeTrue something) -> Void
showing _ SomethingVeryComplicatedIs impossible