Strong generators #
If P : ObjectProperty C, we say that P is a strong generator if it is a
generator (in the sense that IsSeparating P holds) such that for any
proper subobject A ⊂ X, there exists a morphism G ⟶ X which does not factor
through A from an object satisfying P.
The main result is the lemma isStrongGenerator_iff_exists_extremalEpi which
says that if P is w-small, C is locally w-small and
has coproducts of size w, then P is a strong generator iff any
object of C is the target of an extremal epimorphism from a coproduct of
objects satisfying P.
We also show that if any object in C is a colimit of objects in S,
then S is a strong generator.
References #
A property P : ObjectProperty C is a strong generator
if it is separating and for any proper subobject A ⊂ X, there exists
a morphism G ⟶ X which does not factor through A from an object
such that P G holds.
Equations
- P.IsStrongGenerator = (P.IsSeparating ∧ ∀ ⦃X : C⦄ (A : CategoryTheory.Subobject X), (∀ (G : C), P G → ∀ (f : G ⟶ X), A.Factors f) → A = ⊤)