unimath2024/Lol.agda

39 lines
1 KiB
Agda
Raw Normal View History

2024-07-29 22:45:35 +00:00
{-# OPTIONS --cubical #-}
open import Cubical.Foundations.Prelude
data : Set where
zero :
suc :
add :
add zero n = n
add (suc m) n = add m (suc n)
data ℤ₀ : Set where
pos : ℤ₀
negsuc : ℤ₀
data : Set where
z :
p : (m n : ) z m n z (suc m) (suc n)
ℤ→ℤ₀ : ℤ₀
ℤ→ℤ₀ (z zero zero) = pos zero
ℤ→ℤ₀ (z zero (suc x₁)) = negsuc x₁
ℤ→ℤ₀ (z (suc x) zero) = pos (suc x)
ℤ→ℤ₀ (z (suc x) (suc x₁)) = ℤ→ℤ₀ (z x x₁)
ℤ→ℤ₀ (p m n i) = ℤ→ℤ₀ {! !}
ℤ₀→ℤ : ℤ₀
ℤ₀→ℤ (pos x) = z x zero
ℤ₀→ℤ (negsuc x) = z zero (suc x)
ap : {A B x y} (f : A B) (x y) (f x f y)
ap f x i = f (x i)
add- :
add- (z x x₁) (z x₂ x₃) = z (add x x₂) (add x₁ x₃)
add- (z x x₁) (p m n i) = z (add x {! !}) {! !}
add- (p m n i) (z x x₁) = {! !}
add- (p m n i) (p m₁ n₁ i₁) = {! !}