type-theory/src/CircleThing2.agda
2023-04-10 13:39:17 -05:00

34 lines
973 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.

{-# OPTIONS --without-K #-}
module CircleThing2 where
open import Agda.Primitive renaming (Set to Type)
open import elementary-number-theory.integers
open import elementary-number-theory.natural-numbers
open import foundation-core.identity-types
open import foundation.univalence
open import synthetic-homotopy-theory.circle
infix 10 _≡_
_≡_ = __
loops-to- : base-𝕊¹ base-𝕊¹
loops-to- p = ?
-to-loops : base-𝕊¹ base-𝕊¹
-to-loops = ind-
(λ _ base-𝕊¹ base-𝕊¹)
(inv loop-𝕊¹)
neg-ver
refl
(loop-𝕊¹)
pos-ver
where
pos-ver : base-𝕊¹ base-𝕊¹ base-𝕊¹ base-𝕊¹
pos-ver zero- p = refl
pos-ver (succ- n) p = loop-𝕊¹ pos-ver n p
neg-ver : base-𝕊¹ base-𝕊¹ base-𝕊¹ base-𝕊¹
neg-ver zero- p = refl
neg-ver (succ- n) p = (inv loop-𝕊¹) neg-ver n p