TheHoTTGame/1FundamentalGroup/Quest0.agda

25 lines
418 B
Agda

module 1FundamentalGroup.Quest0 where
open import 1FundamentalGroup.Preambles.P0
Refl : base base
Refl = {!!}
Flip : Bool Bool
Flip x = {!!}
flipIso : Bool Bool
flipIso = {!!}
flipPath : Bool Bool
flipPath = {!!}
doubleCover : Type
doubleCover x = {!!}
endPtOfTrue : (p : base base) doubleCover base
endPtOfTrue p = {!!}
Refl≢loop : Refl loop
Refl≢loop p = {!!}