TheHoTTGame/1FundamentalGroup/Quest3Solutions.agda
2021-11-01 00:07:28 +00:00

22 lines
615 B
Agda

module 1FundamentalGroup.Quest3Solutions where
open import Cubical.Foundations.Prelude
open import Cubical.HITs.S1 using ( ; base ; loop )
open import 1FundamentalGroup.Quest1Solutions
open import Cubical.Foundations.Path
outOfS¹ : (B : Type) (b : B base) PathP (λ i B (loop i)) b b (x : ) B x
outOfS¹ B b p base = b
outOfS¹ B b p (loop i) = p i
rewind : (x : ) helix x base x
rewind base = loop_times
rewind (loop i) = path i where
path : PathP (λ i helix (loop i) base loop i) loop_times loop_times
path = {!!}
thing = PathPIsoPath