Add Everything (#34)

This commit is contained in:
Patrick Stevens
2019-08-18 10:35:15 +01:00
committed by GitHub
parent a31ae0d1ea
commit e7c54fa48a
45 changed files with 415 additions and 378 deletions

View File

@@ -1,13 +1,13 @@
{-# OPTIONS --safe --warning=error #-}
{-# OPTIONS --safe --warning=error --without-K #-}
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import LogicalFormulae
open import Functions
open import Naturals
open import FinSet
open import Numbers.Naturals
open import Sets.FinSet
module Cardinality where
module Sets.Cardinality where
record CountablyInfiniteSet {a : _} (A : Set a) : Set a where
field
counting : A
@@ -227,5 +227,5 @@ module Cardinality where
-}
injectionToNMeansCountable : {a : _} {A : Set a} {f : A } Injection f InfiniteSet A Countable A
injectionToNMeansCountable {f = f} inj record { isInfinite = isInfinite } = {!!}
-- injectionToNMeansCountable : {a : _} {A : Set a} {f : A → } → Injection f → InfiniteSet A → Countable A
-- injectionToNMeansCountable {f = f} inj record { isInfinite = isInfinite } = {!!}