Idris2/tests/idris2/interactive033/UninhIndent.idr
2021-06-08 17:03:06 +01:00

10 lines
281 B
Idris

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