Files
agdaproofs/Decidable/Sets.agda
2019-12-04 19:53:34 +00:00

11 lines
293 B
Agda

{-# OPTIONS --safe --warning=error --without-K #-}
open import LogicalFormulae
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
module Decidable.Sets where
record DecidableSet {a : _} (A : Set a) : Set a where
field
eq : (a b : A) ((a b) || ((a b) False))