Files
agdaproofs/Decidable/Sets.agda
2020-01-05 15:06:35 +00:00

10 lines
232 B
Agda

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