step 1
This commit is contained in:
parent
e0c0e56967
commit
196eeec6e2
1 changed files with 18 additions and 0 deletions
18
src/ThesisWork/Pi3S2/Step1.agda
Normal file
18
src/ThesisWork/Pi3S2/Step1.agda
Normal file
|
@ -0,0 +1,18 @@
|
|||
{-# OPTIONS --cubical #-}
|
||||
|
||||
module ThesisWork.Pi3S2.Step1 where
|
||||
|
||||
open import Agda.Primitive
|
||||
open import Cubical.Data.Sigma
|
||||
open import Cubical.Foundations.Equiv
|
||||
open import Cubical.Foundations.Equiv.Properties
|
||||
open import Cubical.Foundations.Isomorphism
|
||||
open import Cubical.Foundations.Pointed
|
||||
open import Cubical.Foundations.Prelude
|
||||
open import Cubical.Homotopy.Loopspace
|
||||
|
||||
arrow∙ : {l : Level} → Type (lsuc l)
|
||||
arrow∙ {l} = Σ (Pointed l) (λ X → Σ (Pointed l) (λ Y → X →∙ Y))
|
||||
|
||||
F : {l : Level} → arrow∙ {l} → arrow∙ {l}
|
||||
F x @ (X , Y , f) = {! fiber !} , X , {! fst !}
|
Loading…
Reference in a new issue