Skip to content

Commit

Permalink
chore(category_theory/adjunction): reflective lemmas (#5968)
Browse files Browse the repository at this point in the history
Improves the docstring and changes the name to be more appropriate (the lemma has nothing to do with essential images).
  • Loading branch information
b-mehta committed Apr 2, 2021
1 parent cf90e2c commit e4ce09f
Showing 1 changed file with 3 additions and 2 deletions.
5 changes: 3 additions & 2 deletions src/category_theory/adjunction/reflective.lean
Original file line number Diff line number Diff line change
Expand Up @@ -47,11 +47,12 @@ begin
end

/--
When restricted to objects in `D` given by `i : D ⥤ C`, the unit is an isomorphism.
When restricted to objects in `D` given by `i : D ⥤ C`, the unit is an isomorphism. In other words,
`η_iX` is an isomorphism for any `X` in `D`.
More generally this applies to objects essentially in the reflective subcategory, see
`functor.ess_image.unit_iso`.
-/
instance functor.ess_image.unit_iso_restrict [reflective i] {B : D} :
instance is_iso_unit_obj [reflective i] {B : D} :
is_iso ((adjunction.of_right_adjoint i).unit.app (i.obj B)) :=
begin
have : (adjunction.of_right_adjoint i).unit.app (i.obj B) =
Expand Down

0 comments on commit e4ce09f

Please sign in to comment.