Skip to content

Commit

Permalink
feat(CategoryTheory/EqToHom): generalize Functor.congr_map to Prefunc…
Browse files Browse the repository at this point in the history
…tor.congr_map (#12384)
  • Loading branch information
callesonne committed Apr 24, 2024
1 parent d0ecb3c commit cba2f37
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 4 deletions.
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Category/Cat/Limit.lean
Original file line number Diff line number Diff line change
Expand Up @@ -106,7 +106,7 @@ def limitConeLift (F : J ⥤ Cat.{v, v}) (s : Cone F) : s.pt ⟶ limitConeX F wh
{ pt := s.pt
π :=
{ app := fun j => (s.π.app j).obj
naturality := fun _ _ f => Functor.congr_map objects (s.π.naturality f) } }
naturality := fun _ _ f => objects.congr_map (s.π.naturality f) } }
map f := by
fapply Types.Limit.mk.{v, v}
· intro j
Expand Down
3 changes: 0 additions & 3 deletions Mathlib/CategoryTheory/EqToHom.lean
Original file line number Diff line number Diff line change
Expand Up @@ -250,9 +250,6 @@ theorem congr_inv_of_congr_hom (F G : C ⥤ D) {X Y : C} (e : X ≅ Y) (hX : F.o
Category.assoc]
#align category_theory.functor.congr_inv_of_congr_hom CategoryTheory.Functor.congr_inv_of_congr_hom

theorem congr_map (F : C ⥤ D) {X Y : C} {f g : X ⟶ Y} (h : f = g) : F.map f = F.map g := by rw [h]
#align category_theory.functor.congr_map CategoryTheory.Functor.congr_map

section HEq

-- Composition of functors and maps w.r.t. heq
Expand Down
4 changes: 4 additions & 0 deletions Mathlib/Combinatorics/Quiver/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -135,6 +135,10 @@ infixl:60 " ⋙q " => Prefunctor.comp
/-- Notation for the identity prefunctor on a quiver. -/
notation "𝟭q" => id

theorem congr_map {U V : Type*} [Quiver U] [Quiver V] (F : U ⥤q V) {X Y : U} {f g : X ⟶ Y}
(h : f = g) : F.map f = F.map g := by
rw [h]

end Prefunctor

namespace Quiver
Expand Down

0 comments on commit cba2f37

Please sign in to comment.