Skip to content

Commit

Permalink
feat(category_theory/limits): any functor preserves split coequalizers (
Browse files Browse the repository at this point in the history
#5246)

Once #5230 merges, the only diff in this PR should be in `src/category_theory/limits/preserves/shapes/equalizers.lean`
  • Loading branch information
b-mehta committed Dec 10, 2020
1 parent 12d097e commit cdb1398
Showing 1 changed file with 11 additions and 1 deletion.
12 changes: 11 additions & 1 deletion src/category_theory/limits/preserves/shapes/equalizers.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Bhavik Mehta. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Bhavik Mehta
-/
import category_theory.limits.shapes.equalizers
import category_theory.limits.shapes.split_coequalizer
import category_theory.limits.preserves.basic

/-!
Expand Down Expand Up @@ -179,6 +179,16 @@ begin
apply_instance
end

/-- Any functor preserves coequalizers of split pairs. -/
@[priority 1]
instance preserves_split_coequalizers (f g : X ⟶ Y) [has_split_coequalizer f g] :
preserves_colimit (parallel_pair f g) G :=
begin
apply preserves_colimit_of_preserves_colimit_cocone
((has_split_coequalizer.is_split_coequalizer f g).is_coequalizer),
apply (is_colimit_map_cocone_cofork_equiv G _).symm
((has_split_coequalizer.is_split_coequalizer f g).map G).is_coequalizer,
end
end coequalizers

end category_theory.limits

0 comments on commit cdb1398

Please sign in to comment.