type-theory/src/HIT.agda
2022-10-31 16:05:18 -05:00

13 lines
281 B
Agda

{-# OPTIONS --cubical #-}
module HIT where
open import Cubical.Core.Everything
data : Set where
base :
loop : base base
apd : {A : Set} {B : A Set} (f : (x : A) B x) {x y : A} (p : x y)
PathP (λ i B (p i)) (f x) (f y)
apd f p i = f (p i)