mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-06 12:28:39 +00:00
Problem 1 of Project Euler (#85)
This commit is contained in:
10
Decidable/Sets.agda
Normal file
10
Decidable/Sets.agda
Normal file
@@ -0,0 +1,10 @@
|
||||
{-# 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))
|
Reference in New Issue
Block a user