mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-18 09:48:38 +00:00
13 lines
427 B
Agda
13 lines
427 B
Agda
{-# OPTIONS --safe --warning=error --without-K #-}
|
|
|
|
open import Functions.Definition
|
|
open import Sets.CantorBijection.Proofs
|
|
|
|
module Sets.CantorBijection.CantorBijection where
|
|
|
|
open Sets.CantorBijection.Proofs using (cantorInverse ; cantorInverseLemma) public
|
|
|
|
cantorBijection : Bijection cantorInverse
|
|
Bijection.inj cantorBijection {x} {y} = cantorInverseInjective x y
|
|
Bijection.surj cantorBijection = cantorInverseSurjective
|