mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 17:21:59 +03:00
10 lines
249 B
Idris
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))
|