The category of R-modules has all limits #
Further, these limits are preserved by the forgetful functor --- that is, the underlying types are just the limits in the category of types.
Equations
- Eq (ModuleCat.addCommGroupObj F j) (inferInstanceAs (AddCommGroup (F.obj j).carrier))
Instances For
Equations
- Eq (ModuleCat.moduleObj F j) (inferInstanceAs (Module R (F.obj j).carrier))
Instances For
The flat sections of a functor into ModuleCat R
form a submodule of all sections.
Equations
- Eq (ModuleCat.sectionsSubmodule F) { carrier := (F.comp (CategoryTheory.forget (ModuleCat R))).sections, add_mem' := ⋯, zero_mem' := ⋯, smul_mem' := ⋯ }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Eq (ModuleCat.instModuleElemForallObjCompForgetSections F) (inferInstanceAs (Module R (Subtype fun (x : (j : J) → (F.obj j).carrier) => Membership.mem (ModuleCat.sectionsSubmodule F) x)))
Instances For
Equations
- Eq (ModuleCat.limitAddCommMonoid F) (inferInstanceAs (AddCommMonoid (Shrink (Subtype fun (x : (j : J) → (F.obj j).carrier) => Membership.mem (ModuleCat.sectionsSubmodule F) x))))
Instances For
Equations
- Eq (ModuleCat.limitAddCommGroup F) (inferInstanceAs (AddCommGroup (Shrink (Subtype fun (x : (j : J) → (F.obj j).carrier) => Membership.mem (ModuleCat.sectionsSubmodule F) x))))
Instances For
Equations
- Eq (ModuleCat.limitModule F) (inferInstanceAs (Module R (Shrink (Subtype fun (x : (j : J) → (F.obj j).carrier) => Membership.mem (ModuleCat.sectionsSubmodule F) x))))
Instances For
limit.π (F ⋙ forget (ModuleCat.{w} R)) j
as an R
-linear map.
Equations
- Eq (ModuleCat.limitπLinearMap F j) { toFun := (CategoryTheory.Limits.Types.Small.limitCone (F.comp (CategoryTheory.forget (ModuleCat R)))).π.app j, map_add' := ⋯, map_smul' := ⋯ }
Instances For
Construction of a limit cone in ModuleCat R
.
(Internal use only; use the limits API.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
Witness that the limit cone in ModuleCat R
is a limit cone.
(Internal use only; use the limits API.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
If (F ⋙ forget (ModuleCat R)).sections
is u
-small, F
has a limit.
If J
is u
-small, the category of R
-modules has limits of shape J
.
The category of R-modules has all limits.
An auxiliary declaration to speed up typechecking.
Equations
Instances For
The forgetful functor from R-modules to abelian groups preserves all limits.
The forgetful functor from R-modules to abelian groups preserves all limits.
The forgetful functor from R-modules to types preserves all limits.
The diagram (in the sense of CategoryTheory
)
of an unbundled directLimit
of modules.
Equations
- Eq (ModuleCat.directLimitDiagram G f) { obj := fun (i : ι) => ModuleCat.of R (G i), map := fun {X Y : ι} (hij : Quiver.Hom X Y) => ModuleCat.ofHom (f X Y ⋯), map_id := ⋯, map_comp := ⋯ }
Instances For
The Cocone
on directLimitDiagram
corresponding to
the unbundled directLimit
of modules.
In directLimitIsColimit
we show that it is a colimit cocone.
Equations
- Eq (ModuleCat.directLimitCocone G f) { pt := ModuleCat.of R (Module.DirectLimit G f), ι := { app := fun (x : ι) => ModuleCat.ofHom (Module.DirectLimit.of R ι G f x), naturality := ⋯ } }
Instances For
The unbundled directLimit
of modules is a colimit
in the sense of CategoryTheory
.
Equations
- One or more equations did not get rendered due to their size.