Problem 1 of Project Euler (#85)

This commit is contained in:
Patrick Stevens
2019-12-04 19:53:34 +00:00
committed by GitHub
parent 2ed7bd8044
commit cfd9787bb8
10 changed files with 526 additions and 447 deletions

10
Decidable/Sets.agda Normal file
View 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))