Skip to content

Commit

Permalink
feat: functoriality of coimage-image comparison (#21044)
Browse files Browse the repository at this point in the history
Co-authored-by: Markus Himmel <[email protected]>
  • Loading branch information
TwoFX and TwoFX committed Jan 25, 2025
1 parent f7d835a commit a1c3eb5
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions Mathlib/CategoryTheory/Abelian/Images.lean
Original file line number Diff line number Diff line change
Expand Up @@ -106,4 +106,12 @@ theorem coimageImageComparison_eq_coimageImageComparison' :
theorem coimage_image_factorisation : coimage.π f ≫ coimageImageComparison f ≫ image.ι f = f := by
simp [coimageImageComparison]

/-- The coimage-image comparison morphism is functorial. -/
@[simps!]
def coimageImageComparisonFunctor : Arrow C ⥤ Arrow C where
obj f := Arrow.mk (coimageImageComparison f.hom)
map {f g} η := Arrow.homMk
(cokernel.map _ _ (kernel.map _ _ η.left η.right (by simp)) η.left (by simp))
(kernel.map _ _ η.right (cokernel.map _ _ η.left η.right (by simp)) (by simp)) (by aesop_cat)

end CategoryTheory.Abelian

0 comments on commit a1c3eb5

Please sign in to comment.