added quest 4 and preamble

This commit is contained in:
Jlh18 2021-10-30 19:02:51 +01:00
parent 6b97d4b790
commit 4a2e69d92d
6 changed files with 18 additions and 11 deletions

View File

@ -0,0 +1,5 @@
module 0Trinitarianism.Preambles.P4 where
open import Cubical.Foundations.Prelude using
( Level ; Type ; _≡_ ; J ; JRefl ; refl ; i1 ; i0 ; I ; cong) public
open import Cubical.Foundations.Isomorphism renaming (Iso to _≅_) public

View File

@ -0,0 +1,3 @@
module 0Trinitarianism.Quest4 where
open import 0Trinitarianism.Preambles.P4

View File

@ -1,11 +1,6 @@
module 0Trinitarianism.Quest4Solutions where module 0Trinitarianism.Quest4Solutions where
open import Cubical.Foundations.Prelude using ( Level ; Type ; _≡_ ; J ; JRefl ; refl ; i1 ; i0 ; I) open import 0Trinitarianism.Preambles.P4
open import Cubical.Foundations.Isomorphism renaming (Iso to _≅_)
infixr 30 _∙_
infix 3 _∎
infixr 2 _≡⟨_⟩_
private private
variable variable
@ -76,11 +71,11 @@ Id→Path rfl = refl
Cong : (f : A B) Id x y Id (f x) (f y) Cong : (f : A B) Id x y Id (f x) (f y)
Cong f rfl = rfl Cong f rfl = rfl
cong : (f : A B) (p : x y) f x f y
cong {x = x} f = J (λ y p f x f y) refl
cong' : (f : A B) (p : x y) f x f y cong' : (f : A B) (p : x y) f x f y
cong' f p = Id→Path (Cong f (Path→Id p)) cong' {x = x} f = J (λ y p f x f y) refl
cong'' : (f : A B) (p : x y) f x f y
cong'' f p = Id→Path (Cong f (Path→Id p))
------------Path vs Id--------------------- ------------Path vs Id---------------------
@ -115,6 +110,10 @@ _ ≡⟨ x≡y ⟩ y≡z = x≡y ∙ y≡z
_∎ : (x : A) x x _∎ : (x : A) x x
_ = refl _ = refl
infixr 30 _∙_
infix 3 _∎
infixr 2 _≡⟨_⟩_
TransRefl : {x y : A} Trans {A} {x} {x} {y} refl λ q q TransRefl : {x y : A} Trans {A} {x} {x} {y} refl λ q q
TransRefl {x = x} {y = y} = JRefl ((λ y1 p y1 y x y)) λ q q TransRefl {x = x} {y = y} = JRefl ((λ y1 p y1 y x y)) λ q q
@ -182,7 +181,7 @@ endPtRefl : (B : A → Type) → endPt B (refl {x = x}) ≡ id
endPtRefl {x = x} B = JRefl ((λ y p B x B y)) id endPtRefl {x = x} B = JRefl ((λ y p B x B y)) id
endPt' : (B : A Type) (p : x y) B x B y endPt' : (B : A Type) (p : x y) B x B y
endPt' B p = pathToFun (Cubical.Foundations.Prelude.cong B p ) endPt' B p = pathToFun (cong B p )
--------------funExt--------------------- --------------funExt---------------------

Binary file not shown.

Binary file not shown.