mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-05 20:08:41 +00:00
10 lines
232 B
Agda
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))
|