unimath2024/Exercises1.agda
2024-08-01 10:32:27 -05:00

30 lines
No EOL
698 B
Agda
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

module Exercises1 where
open import Agda.Primitive
open import foundation-core.empty-types
open import foundation-core.equivalences
open import foundation-core.negation
open import foundation.natural-numbers
open import foundation.dependent-pair-types
open import foundation.identity-types
open import foundation.univalence
open import foundation.sections
open import foundation.retractions
_≡_ = __
= empty
equal-to-zero : {A : Set} (f : ¬ A) A
equal-to-zero {A} f = eq-equiv A eqv
where
s : section f
s = (λ ()) , λ x ex-falso x
r : retraction f
r = (λ ()) , λ x ex-falso (f x)
eqv : A
eqv = f , s , r
asdf : 0 1