Strong epimorphisms
In this file, we define strong epimorphisms. A strong epimorphism is an epimorphism f
, such
that for every commutative square with f
at the top and a monomorphism at the bottom, there is
a diagonal morphism making the two triangles commute. This lift is necessarily unique (as shown in
comma.lean
).
Main results
Besides the definition, we show that
- the composition of two strong epimorphisms is a strong epimorphism,
- if
f ≫ g
is a strong epimorphism, then so isg
, - if
f
is both a strong epimorphism and a monomorphism, then it is an isomorphism
Future work
There is also the dual notion of strong monomorphism.
References
- [F. Borceux, Handbook of Categorical Algebra 1][borceux-vol1]
- epi : category_theory.epi f
- has_lift : ∀ {X Y : C} {u : P ⟶ X} {v : Q ⟶ Y} {z : X ⟶ Y} [_inst_2 : category_theory.mono z] (h : u ≫ z = f ≫ v), category_theory.arrow.has_lift (category_theory.arrow.hom_mk' h)
A strong epimorphism f
is an epimorphism such that every commutative square with f
at the
top and a monomorphism at the bottom has a lift.
The composition of two strong epimorphisms is a strong epimorphism.
If f ≫ g
is a strong epimorphism, then so is g.
An isomorphism is in particular a strong epimorphism.
A strong epimorphism that is a monomorphism is an isomorphism.