Idris2/tests/idris2/interactive/interactive032/Uninh.idr
2023-09-07 14:57:22 +01:00

13 lines
270 B
Idris

module Uninh
data MyElem : a -> List a -> Type where
MyHere : MyElem x (x :: xs)
MyThere : (later : MyElem x xs) -> MyElem x (y :: xs)
noIndent : (MyElem a []) -> Void
noIndent c = ?noIndent_rhs
Uninhabited (MyElem a []) where
uninhabited c = ?uninhabited_rhs