Skip to content

Commit

Permalink
Commit before major refactor
Browse files Browse the repository at this point in the history
  • Loading branch information
rahulc29 committed Dec 2, 2023
1 parent 34e2747 commit 2edec16
Show file tree
Hide file tree
Showing 2 changed files with 22 additions and 6 deletions.
27 changes: 21 additions & 6 deletions src/Realizability/Assembly.agda
Original file line number Diff line number Diff line change
Expand Up @@ -701,16 +701,31 @@ module Realizability.Assembly {ℓ} {A : Type ℓ} (ca : CombinatoryAlgebra A) w

∃t→Σt : ∃[ t ∈ AssemblyMorphism ys ws ] (e ⊚ t ≡ q) Σ[ t ∈ AssemblyMorphism ys ws ] (e ⊚ t ≡ q)
∃t→Σt ∃t = equivFun (propTruncIdempotent≃ e⊚t≡qIsProp) ∃t


-- I have cooked one ugly proof ngl 😀🔫
open IsCoequalizer
eIsCoequalizer : IsCoequalizer {C = ASM} k₁ k₂ e
eIsCoequalizer .glues = AssemblyMorphism≡ _ _ (funExt λ (x , x' , ex≡ex') ex≡ex')
eIsCoequalizer .univProp {W , ws} q k₁q≡k₂q =
uniqueExists {!!} {!!} {!!} {!!} where
_⊩W_ = ws ._⊩_
∃t : ∃[ t ∈ AssemblyMorphism ys ws ] (e ⊚ t ≡ q)
∃t = do
∃t = (do
(e⁻¹ , e⁻¹IsSection) choice X Y (e .map) surjection
return (record { map = λ y q .map (e⁻¹ y)
; tracker = do
(r , rIsSurjective) surjectionIsTracked
return (r , λ y b b⊩y {!rIsSurjective y b b⊩y!}) } , {!!})
return (h e⁻¹ e⁻¹IsSection , {!!})) where
module _
(e⁻¹ : Y X)
(e⁻¹IsSection : section (e .map) e⁻¹) where
h : AssemblyMorphism ys ws
h .map y = q .map (e⁻¹ y)
h .tracker =
do
(q~ , q~tracks) q .tracker
(r , rWitness) surjectionIsTracked
return (s ⨾ (k ⨾ q~) ⨾ (s ⨾ (k ⨾ r) ⨾ Id) , (λ y b b⊩y {!!}))

e⊚h≡q : e ⊚ h ≡ q
e⊚h≡q = AssemblyMorphism≡ _ _ (funExt λ x {!e⁻¹IsSection (e .map x)!})

hy≡qx : x y e .map x ≡ y h .map y ≡ q .map x
hy≡qx x y ex≡y = {!e⁻¹IsSection y!}
1 change: 1 addition & 0 deletions src/index.agda
Original file line number Diff line number Diff line change
Expand Up @@ -7,3 +7,4 @@ open import Realizability.PartialCombinatoryAlgebra
open import Realizability.CombinatoryAlgebra
open import Realizability.ApplicativeStructure
open import Realizability.Assembly
open import Realizability.Choice

0 comments on commit 2edec16

Please sign in to comment.