Definitions and basic properties of normal monomorphisms and epimorphisms. #
A normal monomorphism is a morphism that is the kernel of some other morphism.
We give the construction NormalMono → RegularMono
(CategoryTheory.NormalMono.regularMono
)
as well as the dual construction for normal epimorphisms. We show equivalences reflect normal
monomorphisms (CategoryTheory.equivalenceReflectsNormalMono
), and that the pullback of a
normal monomorphism is normal (CategoryTheory.normalOfIsPullbackSndOfNormal
).
We also define classes IsNormalMonoCategory
and IsNormalEpiCategory
for categories in which
every monomorphism or epimorphism is normal, and deduce that these categories are
RegularMonoCategory
s resp. RegularEpiCategory
s.
A normal monomorphism is a morphism which is the kernel of some morphism.
- Z : C
A normal monomorphism is a morphism which is the kernel of some morphism.
A normal monomorphism is a morphism which is the kernel of some morphism.
- w : CategoryStruct.comp f g = 0
A normal monomorphism is a morphism which is the kernel of some morphism.
- isLimit : Limits.IsLimit (Limits.KernelFork.ofι f ⋯)
A normal monomorphism is a morphism which is the kernel of some morphism.
Instances
If F
is an equivalence and F.map f
is a normal mono, then f
is a normal mono.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Every normal monomorphism is a regular monomorphism.
Equations
- CategoryTheory.NormalMono.regularMono f = { Z := CategoryTheory.NormalMono.Z f, left := CategoryTheory.NormalMono.g, right := 0, w := ⋯, isLimit := CategoryTheory.NormalMono.isLimit }
If f
is a normal mono, then any map k : W ⟶ Y
such that k ≫ normal_mono.g = 0
induces
a morphism l : W ⟶ X
such that l ≫ f = k
.
Equations
Instances For
The second leg of a pullback cone is a normal monomorphism if the right component is too.
See also pullback.sndOfMono
for the basic monomorphism version, and
normalOfIsPullbackFstOfNormal
for the flipped version.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The first leg of a pullback cone is a normal monomorphism if the left component is too.
See also pullback.fstOfMono
for the basic monomorphism version, and
normalOfIsPullbackSndOfNormal
for the flipped version.
Equations
Instances For
A normal mono category is a category in which every monomorphism is normal.
A normal mono category is a category in which every monomorphism is normal.
Instances
Alias of CategoryTheory.IsNormalMonoCategory
.
A normal mono category is a category in which every monomorphism is normal.
Instances For
In a category in which every monomorphism is normal, we can express every monomorphism as a kernel. This is not an instance because it would create an instance loop.
Equations
- CategoryTheory.normalMonoOfMono f = ⋯.some
Instances For
A normal epimorphism is a morphism which is the cokernel of some morphism.
- W : C
A normal epimorphism is a morphism which is the cokernel of some morphism.
A normal epimorphism is a morphism which is the cokernel of some morphism.
- w : CategoryStruct.comp g f = 0
A normal epimorphism is a morphism which is the cokernel of some morphism.
- isColimit : Limits.IsColimit (Limits.CokernelCofork.ofπ f ⋯)
A normal epimorphism is a morphism which is the cokernel of some morphism.
Instances
If F
is an equivalence and F.map f
is a normal epi, then f
is a normal epi.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Every normal epimorphism is a regular epimorphism.
Equations
- CategoryTheory.NormalEpi.regularEpi f = { W := CategoryTheory.NormalEpi.W f, left := CategoryTheory.NormalEpi.g, right := 0, w := ⋯, isColimit := CategoryTheory.NormalEpi.isColimit }
If f
is a normal epi, then every morphism k : X ⟶ W
satisfying NormalEpi.g ≫ k = 0
induces l : Y ⟶ W
such that f ≫ l = k
.
Equations
Instances For
The second leg of a pushout cocone is a normal epimorphism if the right component is too.
See also pushout.sndOfEpi
for the basic epimorphism version, and
normalOfIsPushoutFstOfNormal
for the flipped version.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The first leg of a pushout cocone is a normal epimorphism if the left component is too.
See also pushout.fstOfEpi
for the basic epimorphism version, and
normalOfIsPushoutSndOfNormal
for the flipped version.
Equations
Instances For
A normal mono becomes a normal epi in the opposite category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A normal epi becomes a normal mono in the opposite category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A normal epi category is a category in which every epimorphism is normal.
A normal epi category is a category in which every epimorphism is normal.
Instances
Alias of CategoryTheory.IsNormalEpiCategory
.
A normal epi category is a category in which every epimorphism is normal.
Instances For
In a category in which every epimorphism is normal, we can express every epimorphism as a kernel. This is not an instance because it would create an instance loop.
Equations
- CategoryTheory.normalEpiOfEpi f = ⋯.some