Skip to content

Commit

Permalink
chore(CategoryTheory/Adjunction): simplify some proofs in `Adjunction…
Browse files Browse the repository at this point in the history
…/Reflective` (#12375)

Some results in this file can be extracted from results added in #12344
  • Loading branch information
dagurtomas committed Apr 23, 2024
1 parent c160989 commit 81d26b1
Showing 1 changed file with 3 additions and 14 deletions.
17 changes: 3 additions & 14 deletions Mathlib/CategoryTheory/Adjunction/Reflective.lean
Expand Up @@ -55,13 +55,8 @@ When restricted to objects in `D` given by `i : D ⥤ C`, the unit is an isomorp
More generally this applies to objects essentially in the reflective subcategory, see
`Functor.essImage.unit_isIso`.
-/
instance isIso_unit_obj [Reflective i] {B : D} : IsIso ((ofRightAdjoint i).unit.app (i.obj B)) := by
have : (ofRightAdjoint i).unit.app (i.obj B) = inv (i.map ((ofRightAdjoint i).counit.app B)) := by
rw [← comp_hom_eq_id]
apply (ofRightAdjoint i).right_triangle_components
rw [this]
exact IsIso.inv_isIso
#align category_theory.is_iso_unit_obj CategoryTheory.isIso_unit_obj
example [Reflective i] {B : D} : IsIso ((ofRightAdjoint i).unit.app (i.obj B)) :=
inferInstance

/-- If `A` is essentially in the image of a reflective functor `i`, then `η_A` is an isomorphism.
This gives that the "witness" for `A` being in the essential image can instead be given as the
Expand All @@ -71,13 +66,7 @@ reflection of `A`, with the isomorphism as `η_A`.
-/
theorem Functor.essImage.unit_isIso [Reflective i] {A : C} (h : A ∈ i.essImage) :
IsIso ((ofRightAdjoint i).unit.app A) := by
suffices (ofRightAdjoint i).unit.app A = h.getIso.inv ≫
(ofRightAdjoint i).unit.app (i.obj (Functor.essImage.witness h)) ≫
(leftAdjoint i ⋙ i).map h.getIso.hom by
rw [this]
infer_instance
rw [← NatTrans.naturality]
simp
rwa [isIso_unit_app_iff_mem_essImage]
#align category_theory.functor.ess_image.unit_is_iso CategoryTheory.Functor.essImage.unit_isIso

/-- If `η_A` is an isomorphism, then `A` is in the essential image of `i`. -/
Expand Down

0 comments on commit 81d26b1

Please sign in to comment.