Files
agdaproofs/Decidable/Sets.agda
2020-04-05 11:09:12 +01:00

9 lines
223 B
Agda

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