module Decidable where

open import Equality
open import Level
open import Proposition

----------------------------------------------------------------------
-- Decidable properties
----------------------------------------------------------------------
data Dec { : Level} (A : Set ) : Set  where
  yes : (x : A)     Dec A
  no  : (¬x : ¬ A)  Dec A

----------------------------------------------------------------------
-- Decidable equality
----------------------------------------------------------------------
record hasDecEq { : Level}(A : Set ) : Set  where
  infix 4 _≐_
  field _≐_ : (x y : A)  Dec (x  y)

open hasDecEq {{...}} public

{-# DISPLAY hasDecEq._≐_ x y = x  y #-}