Idris2/tests/idris2/basic/basic064/Issue2072.idr
2023-09-07 14:57:22 +01:00

10 lines
249 B
Idris

data Elem : Type -> List Type -> Type where
Types : (0 a : Type) -> Eq a => List Type
export
body : (0 _ : Eq t1)
=> {auto 0 _ : Elem Bool (Types t1)}
-> (obj : t1)
-> (obj == obj) === maybe True (const False) (guard (obj == obj))