Elem.agda 153 B

123456789
  1. module Elem where
  2. open import Prelude
  3. open import Star
  4. Elem : {X : Set}(R : Rel X) -> Rel X
  5. Elem R x y = Star (LeqBool [×] R) (false , x) (true , y)