File tree Expand file tree Collapse file tree 1 file changed +7
-1
lines changed
src/Categories/Diagram/Coend Expand file tree Collapse file tree 1 file changed +7
-1
lines changed Original file line number Diff line number Diff line change @@ -6,7 +6,7 @@ open import Categories.Category.Core using (Category)
66open import Categories.Category.Product
77import Categories.Category.Construction.Cowedges as Cowedges
88open import Categories.Category.Construction.Functors
9- open import Categories.Category.Equivalence
9+ open import Categories.Category.Equivalence as SE
1010open import Categories.Category.Equivalence.Preserves
1111open import Categories.Diagram.Coend
1212open import Categories.Diagram.Colimit
@@ -137,6 +137,12 @@ module _ {o ℓ e o′ ℓ′ e′} {C : Category o ℓ e} {D : Category o′
137137
138138 open StrongEquivalence Eq renaming (F to F⇒)
139139
140+ Coend-yields-colimit : Coend F → Colimit (Twist′ C D F)
141+ Coend-yields-colimit ef = record { initial = pres-Initial (SE.sym Eq) (Coend⇒Initial F ef) }
142+
143+ colimit-yields-Coend : Colimit (Twist′ C D F) → Coend F
144+ colimit-yields-Coend l = Initial⇒Coend F (pres-Initial Eq (Colimit.initial l))
145+
140146 -- Coends and Colimits are equivalent, in the category Cowedge F
141147 Coend-as-Colimit : (coend : Coend F) → (cl : Colimit (Twist′ C D F)) → Coend.cowedge coend ≅ F₀ F⇒ (Colimit.initial.⊥ cl)
142148 Coend-as-Colimit coend cl = Initial.up-to-iso (Cowedges.Cowedges F) (Coend⇒Initial F coend) (pres-Initial Eq initial)
You can’t perform that action at this time.
0 commit comments