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