quest2 -> quest1

This commit is contained in:
Jlh18 2021-10-02 14:59:07 +01:00
parent 87834c2ae0
commit 8c8c1618d1
6 changed files with 75 additions and 12 deletions

View File

@ -1,9 +1,9 @@
module 1FundamentalGroup.Preambles.P1 where
open import Cubical.HITs.S1 public
open import Cubical.HITs.S1 using ( ; base ; loop) public
open import Cubical.Data.Nat using ( ; suc ; zero) public
open import Cubical.Data.Int using ( ; pos ; negsuc) public
open import Cubical.Data.Int using ( ; pos ; negsuc ; -_) public
open import Cubical.Data.Empty public
open import Cubical.Foundations.Prelude public
open import Cubical.Foundations.HLevels public
open import Cubical.Foundations.Prelude renaming (subst to endPt) public
open import Cubical.Foundations.Isomorphism renaming (Iso to _≅_) public
open import 1FundamentalGroup.Quest0Solutions using ( Refl ; Refl≢loop ) public

View File

@ -9,8 +9,27 @@ open import 1FundamentalGroup.Preambles.P1
loop_times : Ω base
loop n times = {!!}
¬isSetS¹ : isSet
¬isSetS¹ = {!!}
{-
The definition of suc goes here.
-}
¬isPropS¹ : isProp
¬isPropS¹ = {!!}
{-
The definition of pred goes here.
-}
{-
The definition of sucIso goes here.
-}
{-
The definition of sucPath goes here.
-}
helix : Type
helix = {!!}
windingNumberBase : base base
windingNumberBase = {!!}
windingNumber : (x : ) base x helix x
windingNumber = {!!}

View File

@ -12,8 +12,40 @@ loop pos (suc n) times = loop pos n times ∙ loop
loop negsuc zero times = sym loop
loop negsuc (suc n) times = loop negsuc n times sym loop
¬isSetS¹ : isSet
¬isSetS¹ h = Refl≢loop (h base base Refl loop)
suc :
suc (pos n) = pos (suc n)
suc (negsuc zero) = pos zero
suc (negsuc (suc n)) = negsuc n
¬isPropS¹ : isProp
¬isPropS¹ h = ¬isSetS¹ (isProp→isSet h)
pred :
pred (pos zero) = negsuc zero
pred (pos (suc n)) = pos n
pred (negsuc n) = negsuc (suc n)
sucIso :
sucIso = iso suc pred s r where
s : section suc pred
s (pos zero) = refl
s (pos (suc n)) = refl
s (negsuc zero) = refl
s (negsuc (suc n)) = refl
r : retract suc pred
r (pos zero) = refl
r (pos (suc n)) = refl
r (negsuc zero) = refl
r (negsuc (suc n)) = refl
sucPath :
sucPath = isoToPath sucIso
helix : Type
helix base =
helix (loop i) = sucPath i
windingNumberBase : base base
windingNumberBase p = endPt helix p (pos zero)
windingNumber : (x : ) base x helix x
windingNumber x p = endPt helix p (pos zero)

View File

@ -0,0 +1,12 @@
¬isSetS¹ : isSet
¬isSetS¹ = {!!}
¬isPropS¹ : isProp
¬isPropS¹ = {!!}
-------------solutions------
¬isSetS¹ : isSet
¬isSetS¹ h = Refl≢loop (h base base Refl loop)
¬isPropS¹ : isProp
¬isPropS¹ h = ¬isSetS¹ (isProp→isSet h)