Injective objects and categories with enough injectives #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
An object J
is injective iff every morphism into J
can be obtained by extending a monomorphism.
- factors : ∀ {X Y : C} (g : X ⟶ J) (f : X ⟶ Y) [_inst_2 : category_theory.mono f], ∃ (h : Y ⟶ J), f ≫ h = g
An object J
is injective iff every morphism into J
can be obtained by extending a monomorphism.
Instances of this typeclass
- category_theory.injective_presentation.injective
- category_theory.injective.zero_injective
- category_theory.injective.injective
- category_theory.injective.category_theory.limits.prod.injective
- category_theory.injective.category_theory.limits.pi_obj.injective
- category_theory.injective.category_theory.limits.biprod.injective
- category_theory.injective.category_theory.limits.biproduct.injective
- category_theory.injective.opposite.unop.injective
- category_theory.injective.opposite.op.injective
- category_theory.injective.injective_under
- category_theory.injective.syzygies.injective
- category_theory.InjectiveResolution.injective
- AddCommGroup.injective_of_divisible
- J : C
- injective : category_theory.injective self.J . "apply_instance"
- f : X ⟶ self.J
- mono : category_theory.mono self.f . "apply_instance"
An injective presentation of an object X
consists of a monomorphism f : X ⟶ J
to some injective object J
.
Instances for category_theory.injective_presentation
- category_theory.injective_presentation.has_sizeof_inst
- presentation : ∀ (X : C), nonempty (category_theory.injective_presentation X)
A category "has enough injectives" if every object has an injective presentation,
i.e. if for every object X
there is an injective object J
and a monomorphism X ↪ J
.
Instances of this typeclass
Let J
be injective and g
a morphism into J
, then g
can be factored through any monomorphism.
Equations
The axiom of choice says that every nonempty type is an injective object in Type
.
injective.under X
provides an arbitrarily chosen injective object equipped with
an monomorphism injective.ι : X ⟶ injective.under X
.
Equations
Instances for category_theory.injective.under
The monomorphism injective.ι : X ⟶ injective.under X
from the arbitrarily chosen injective object under X
.
Equations
Instances for category_theory.injective.ι
When C
has enough injectives, the object injective.syzygies f
is
an arbitrarily chosen injective object under cokernel f
.
Equations
Instances for category_theory.injective.syzygies
When C
has enough injective,
injective.d f : Y ⟶ syzygies f
is the composition
cokernel.π f ≫ ι (cokernel f)
.
(When C
is abelian, we have exact f (injective.d f)
.)
Given a pair of exact morphism f : Q ⟶ R
and g : R ⟶ S
and a map h : R ⟶ J
to an injective
object J
such that f ≫ h = 0
, then g
descents to a map S ⟶ J
. See below:
Q --- f --> R --- g --> S
|
| h
v
J
Equations
- category_theory.injective.exact.desc h f g hgf w = (category_theory.exact.lift h.op g.op f.op hgf _).unop
Given an adjunction F ⊣ G
such that F
preserves monos, G
maps an injective presentation
of X
to an injective presentation of G(X)
.
Given an equivalence of categories F
, an injective presentation of F(X)
induces an
injective presentation of X.