Definitions and basic properties of regular monomorphisms and epimorphisms. #
A regular monomorphism is a morphism that is the equalizer of some parallel pair.
In this file, we give the following definitions.
RegularMono f, which is a structure carrying the data that exhibitsfas a regular monomorphism. That is, it carries a fork and data specifyingfa the equalizer of that fork.IsRegularMono f, which is aProp-valued class stating thatfis a regular monomorphism. In particular, this doesn't carry any data. and constructionsIsSplitMono f → RegularMono fandRegularMono f → Mono fas well as the dual definitions/constructions for regular epimorphisms.
Additionally, we give the constructions
RegularEpi f → EffectiveEpi f, from which it can be deduced that regular epimorphisms are strong.regularEpiOfEffectiveEpi: constructs aRegularEpi finstance fromEffectiveEpi fandHasPullback f f.
We also define classes IsRegularMonoCategory and IsRegularEpiCategory for categories in which
every monomorphism or epimorphism is regular, and deduce that these categories are
StrongMonoCategorys resp. StrongEpiCategorys.
A regular monomorphism is a morphism which is the equalizer of some parallel pair.
- Z : C
An object in
C A map from the codomain of
ftoZAnother map from the codomain of
ftoZfequalizes the two maps- isLimit : Limits.IsLimit (Limits.Fork.ofι f ⋯)
fis the equalizer of the two maps
Instances For
Every regular monomorphism is a monomorphism.
Every isomorphism is a regular monomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Regular monomorphisms are preserved by isomorphisms in the arrow category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
IsRegularMono f is the assertion that f is a regular monomorphism.
- regularMono : Nonempty (RegularMono f)
Instances
The MorphismProperty C satisfied by regular monomorphisms in C.
Instances For
Given IsRegularMono f, a choice of data for RegularMono f.
Equations
Instances For
Alias of CategoryTheory.IsRegularMono.getStruct.
Given IsRegularMono f, a choice of data for RegularMono f.
Instances For
Given a regular monomorphism f : X ⟶ Y (i.e. a morphism satisfying the predicate IsRegularMono),
this section gives an equalizer diagram
X
f|
v
Y
left| |right
v v
Z
The names Z, left, and right all being in the IsRegularMono namespace.
The target of the equalizer diagram for f.
Equations
Instances For
The "left" map Y ⟶ Z.
Instances For
The "right" map Y ⟶ Z.
Instances For
The equalizer condition.
The fork is in fact an equalizer.
Equations
Instances For
Lift a morphism k : W ⟶ Y, equalized by the two morphisms left and right, along f.
Equations
Instances For
The chosen equalizer of a parallel pair is a regular monomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Every split monomorphism is a regular monomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If f is a regular mono, then any map k : W ⟶ Y equalizing RegularMono.left and
RegularMono.right induces a morphism l : W ⟶ X such that l ≫ f = k.
Equations
- hf.lift' k h = CategoryTheory.Limits.Fork.IsLimit.lift' hf.isLimit k h
Instances For
The second leg of a pullback cone is a regular monomorphism if the right component is too.
See also Pullback.sndOfMono for the basic monomorphism version, and
regularOfIsPullbackFstOfRegular 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 regular monomorphism if the left component is too.
See also Pullback.fstOfMono for the basic monomorphism version, and
regularOfIsPullbackSndOfRegular for the flipped version.
Equations
Instances For
Any regular monomorphism is a strong monomorphism.
A regular monomorphism is an isomorphism if it is an epimorphism.
A regular mono category is a category in which every monomorphism is regular.
Every monomorphism is a regular monomorphism
Instances
In a category in which every monomorphism is regular, we can express every monomorphism as an equalizer. This is not an instance because it would create an instance loop.
Instances For
A regular epimorphism is a morphism which is the coequalizer of some parallel pair.
- W : C
An object from
C Two maps to the domain of
fTwo maps to the domain of
ffcoequalizes the two maps- isColimit : Limits.IsColimit (Limits.Cofork.ofπ f ⋯)
fis the coequalizer
Instances For
Every regular epimorphism is an epimorphism.
Every isomorphism is a regular epimorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Regular epimorphisms are preserved by isomorphisms in the arrow category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
IsRegularEpi f is the assertion that f is a regular epimorphism.
- regularEpi : Nonempty (RegularEpi f)
Instances
The MorphismProperty C satisfied by regular epimorphisms in C.
Instances For
Given IsRegularEpi f, a choice of data for RegularEpi f.
Equations
Instances For
Alias of CategoryTheory.IsRegularEpi.getStruct.
Given IsRegularEpi f, a choice of data for RegularEpi f.
Instances For
Given a regular epimorphism f : X ⟶ Y (i.e. a morphism satisfying the predicate IsRegularEpi),
this section gives a coequalizer diagram
W
left| |right
v v
X
f|
v
Y
The names W, left, and right all being in the IsRegularEpi namespace.
The source of the coequalizer diagram for f.
Equations
Instances For
The "left" map W ⟶ X.
Instances For
The "right" map W ⟶ X.
Instances For
The coequalizer condition.
The cofork is in fact a coequalizer.
Equations
Instances For
Descend a morphism k : X ⟶ Z, coequalized by the two morphisms left and right, along f.
Equations
Instances For
The chosen coequalizer of a parallel pair is a regular epimorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A morphism which is a coequalizer for its kernel pair is a regular epi.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The data of an EffectiveEpi structure on a RegularEpi.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A morphism which is a coequalizer for its kernel pair is an effective epi.
Alias of CategoryTheory.effectiveEpi_of_kernelPair.
A morphism which is a coequalizer for its kernel pair is an effective epi.
Given a kernel pair of an effective epimorphism f : X ⟶ B, the induced cofork is a coequalizer.
Equations
- One or more equations did not get rendered due to their size.
Instances For
An effective epi which has a kernel pair is a regular epi.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Every split epimorphism is a regular epimorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If f is a regular epi, then every morphism k : X ⟶ W coequalizing RegularEpi.left and
RegularEpi.right induces l : Y ⟶ W such that f ≫ l = k.
Equations
- hf.desc' k h = CategoryTheory.Limits.Cofork.IsColimit.desc' hf.isColimit k h
Instances For
The second leg of a pushout cocone is a regular epimorphism if the right component is too.
See also Pushout.sndOfEpi for the basic epimorphism version, and
regularOfIsPushoutFstOfRegular 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 regular epimorphism if the left component is too.
See also Pushout.fstOfEpi for the basic epimorphism version, and
regularOfIsPushoutSndOfRegular for the flipped version.
Equations
Instances For
A regular epimorphism is an isomorphism if it is a monomorphism.
A regular epi category is a category in which every epimorphism is regular.
Everyone epimorphism is a regular epimorphism
Instances
In a category in which every epimorphism is regular, we can express every epimorphism as a coequalizer. This is not an instance because it would create an instance loop.