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

9 lines
217 B
Agda

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