Skip to content

Commit

Permalink
feat(category_theory/adjunction/reflective): show compositions of ref…
Browse files Browse the repository at this point in the history
…lective are reflective (#6298)

Show compositions of reflective are reflective.
  • Loading branch information
callesonne committed Feb 18, 2021
1 parent 96f8933 commit 8696990
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/category_theory/adjunction/reflective.lean
Expand Up @@ -102,4 +102,11 @@ begin
exact mem_ess_image_of_unit_is_iso A,
end

universes v₃ u₃
variables {E : Type u₃} [category.{v₃} E]

/-- Composition of reflective functors. -/
instance reflective.comp (F : C ⥤ D) (G : D ⥤ E) [Fr : reflective F] [Gr : reflective G] :
reflective (F ⋙ G) := { to_faithful := faithful.comp F G, }

end category_theory

0 comments on commit 8696990

Please sign in to comment.