mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-08 13:28:39 +00:00
9 lines
217 B
Agda
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))
|