Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 218fe1f

Browse files
jcommelindigama0
authored andcommitted
feat(category_theory/opposites): opposites of full and faithful functors (#504)
1 parent 9506e6c commit 218fe1f

File tree

1 file changed

+9
-0
lines changed

1 file changed

+9
-0
lines changed

category_theory/opposites.lean

Lines changed: 9 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -77,6 +77,15 @@ definition op_inv : (Cᵒᵖ ⥤ Dᵒᵖ) ⥤ (C ⥤ D)ᵒᵖ :=
7777

7878
-- TODO show these form an equivalence
7979

80+
instance {F : C ⥤ D} [full F] : full F.op :=
81+
{ preimage := λ X Y f, F.preimage f }
82+
83+
instance {F : C ⥤ D} [faithful F] : faithful F.op :=
84+
{ injectivity' := λ X Y f g h, by simpa using injectivity F h }
85+
86+
@[simp] lemma preimage_id (F : C ⥤ D) [fully_faithful F] (X : C) : F.preimage (𝟙 (F.obj X)) = 𝟙 X :=
87+
injectivity F (by simp)
88+
8089
end
8190

8291
namespace category

0 commit comments

Comments
 (0)