Skip to content

Commit

Permalink
feat(category_theory/adjunction): additional simp lemmas (#1143)
Browse files Browse the repository at this point in the history
* feat(category_theory/adjunction): additional simp lemmas

* spaces

Co-Authored-By: Johan Commelin <johan@commelin.net>
  • Loading branch information
2 people authored and mergify[bot] committed Jul 3, 2019
1 parent f1b5473 commit e4ee18b
Showing 1 changed file with 26 additions and 2 deletions.
28 changes: 26 additions & 2 deletions src/category_theory/adjunction/basic.lean
Expand Up @@ -72,13 +72,37 @@ begin
end

@[simp] lemma left_triangle_components :
F.map (adj.unit.app X) ≫ adj.counit.app (F.obj X) = 𝟙 _ :=
F.map (adj.unit.app X) ≫ adj.counit.app (F.obj X) = 𝟙 (F.obj X) :=
congr_arg (λ (t : nat_trans _ (functor.id C ⋙ F)), t.app X) adj.left_triangle

@[simp] lemma right_triangle_components {Y : D} :
adj.unit.app (G.obj Y) ≫ G.map (adj.counit.app Y) = 𝟙 _ :=
adj.unit.app (G.obj Y) ≫ G.map (adj.counit.app Y) = 𝟙 (G.obj Y) :=
congr_arg (λ (t : nat_trans _ (G ⋙ functor.id C)), t.app Y) adj.right_triangle

@[simp] lemma left_triangle_components_assoc {Z : D} (f : F.obj X ⟶ Z) :
F.map (adj.unit.app X) ≫ adj.counit.app (F.obj X) ≫ f = f :=
by { rw [←assoc], dsimp, simp }

@[simp] lemma right_triangle_components_assoc {Y : D} {Z : C} (f : G.obj Y ⟶ Z) :
adj.unit.app (G.obj Y) ≫ G.map (adj.counit.app Y) ≫ f = f :=
by { rw [←assoc], dsimp, simp }

@[simp] lemma counit_naturality {X Y : D} (f : X ⟶ Y) :
F.map (G.map f) ≫ (adj.counit).app Y = (adj.counit).app X ≫ f :=
adj.counit.naturality f

@[simp] lemma unit_naturality {X Y : C} (f : X ⟶ Y) :
(adj.unit).app X ≫ G.map (F.map f) = f ≫ (adj.unit).app Y :=
(adj.unit.naturality f).symm

@[simp] lemma counit_naturality_assoc {X Y Z : D} (f : X ⟶ Y) (g : Y ⟶ Z) :
F.map (G.map f) ≫ (adj.counit).app Y ≫ g = (adj.counit).app X ≫ f ≫ g :=
by { rw [←assoc], dsimp, simp }

@[simp] lemma unit_naturality_assoc {X Y Z : C} (f : X ⟶ Y) (g : G.obj (F.obj Y) ⟶ Z) :
(adj.unit).app X ≫ G.map (F.map f) ≫ g = f ≫ (adj.unit).app Y ≫ g :=
by { rw [←assoc], dsimp, simp }

end

structure core_hom_equiv (F : C ⥤ D) (G : D ⥤ C) :=
Expand Down

0 comments on commit e4ee18b

Please sign in to comment.