Skip to content

Commit c992d17

Browse files
committed
feat(CategoryTheory/EssentialImage): show that surjective functors are essentially surjective (#11239)
Show that if `F.obj` is surjective, `F` is essentially surjective.
1 parent 158514f commit c992d17

File tree

1 file changed

+5
-0
lines changed

1 file changed

+5
-0
lines changed

Mathlib/CategoryTheory/EssentialImage.lean

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -167,6 +167,11 @@ instance Full.toEssImage (F : C ⥤ D) [Full F] : Full F.toEssImage :=
167167
instance instEssSurjId : EssSurj (𝟭 C) where
168168
mem_essImage Y := ⟨Y, ⟨Iso.refl _⟩⟩
169169

170+
theorem Functor.essSurj_of_surj (h : Function.Surjective F.obj) : EssSurj F where
171+
mem_essImage Y := by
172+
obtain ⟨X, rfl⟩ := h Y
173+
apply obj_mem_essImage
174+
170175
theorem Iso.map_essSurj {F G : C ⥤ D} [EssSurj F] (α : F ≅ G) : EssSurj G where
171176
mem_essImage Y := Functor.essImage.ofNatIso α (EssSurj.mem_essImage Y)
172177

0 commit comments

Comments
 (0)