mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-27 13:43:28 +03:00
22 lines
697 B
Idris
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
|