type-theory/src/loopspace.agda

21 lines
381 B
Agda
Raw Normal View History

2022-10-31 21:05:18 +00:00
-- TODO: Define arbitrary high loop spaces
-- Prelude stuff
{-# OPTIONS --cubical #-}
open import Agda.Primitive public renaming ( Set to Type )
open import Agda.Builtin.Cubical.Path public
variable
: Level
Path : {} (A : Type ) A A Type
Path A a b = PathP (λ _ A) a b
-- Circle
data : Type where
base :
loop : base base