TheHoTTGame/1FundamentalGroup/Quest3Solutions.agda
2021-10-30 20:58:27 +01:00

10 lines
322 B
Agda

module 1FundamentalGroup.Quest3Solutions where
open import Cubical.Foundations.Prelude
open import Cubical.HITs.S1
open import 1FundamentalGroup.Quest1Solutions
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