Documentation

Mathlib.CategoryTheory.ConcreteCategory.EpiMono

Epi and mono in concrete categories #

In this file, we relate epimorphisms and monomorphisms in a concrete category C to surjective and injective morphisms, and we show that if C has strong epi mono factorizations and is such that forget C preserves both epi and mono, then any morphism in C can be factored in a functorial manner as a composition of a surjective morphism followed by an injective morphism.

In any concrete category, injective morphisms are monomorphisms.

instance CategoryTheory.ConcreteCategory.forget₂_preservesMonomorphisms (C : Type u) (D : Type u') [Category.{v, u} C] [HasForget C] [Category.{v', u'} D] [HasForget D] [HasForget₂ C D] [(forget C).PreservesMonomorphisms] :
(forget₂ C D).PreservesMonomorphisms
instance CategoryTheory.ConcreteCategory.forget₂_preservesEpimorphisms (C : Type u) (D : Type u') [Category.{v, u} C] [HasForget C] [Category.{v', u'} D] [HasForget D] [HasForget₂ C D] [(forget C).PreservesEpimorphisms] :
(forget₂ C D).PreservesEpimorphisms

A concrete category with strong epi mono factorizations and such that the forget functor preserves mono and epi admits functorial surjective/injective factorizations.

Equations
Instances For

    In any concrete category, surjective morphisms are epimorphisms.

    theorem CategoryTheory.ConcreteCategory.isIso_iff_bijective {C : Type u} [Category.{v, u} C] [HasForget C] [(forget C).ReflectsIsomorphisms] {X Y : C} (f : X Y) :

    If the forgetful functor of a concrete category reflects isomorphisms, being an isomorphism is equivalent to being bijective.