mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-13 23:58:38 +00:00
12 lines
312 B
Agda
12 lines
312 B
Agda
{-# OPTIONS --safe --warning=error --without-K #-}
|
|
|
|
open import LogicalFormulae
|
|
open import Decidable.Sets
|
|
|
|
module Decidable.Lemmas {a : _} {A : Set a} (dec : DecidableSet A) where
|
|
|
|
squash : {x y : A} → .(x ≡ y) → x ≡ y
|
|
squash {x} {y} x=y with dec x y
|
|
... | inl pr = pr
|
|
... | inr bad = exFalso (bad x=y)
|