mathlib documentation

category_theory.​graded_object

category_theory.​graded_object

The category of graded objects

For any type β, a β-graded object over some category C is just a function β → C into the objects of C. We put the "pointwise" category structure on these, as the non-dependent specialization of category_theory.pi.

We describe the comap functors obtained by precomposing with functions β → γ.

As a consequence a fixed element (e.g. 1) in an additive group β provides a shift functor on β-graded objects

When C has coproducts we construct the total functor graded_object β C ⥤ C, show that it is faithful, and deduce that when C is concrete so is graded_object β C.

def category_theory.​graded_object  :
Type wType uType (max w u)

A type synonym for β → C, used for β-graded objects in a category C.

Equations
@[nolint]
def category_theory.​graded_object_with_shift {β : Type w} [add_comm_group β] :
β → Type uType (max w u)

A type synonym for β → C, used for β-graded objects in a category C with a shift functor given by translation by s.

def category_theory.​graded_object.​comap_eq (C : Type u) [category_theory.category C] {β γ : Type w} {f g : β → γ} :
f = g(category_theory.pi.comap (λ (_x : γ), C) f category_theory.pi.comap (λ (_x : γ), C) g)

The natural isomorphism comparing between pulling back along two propositionally equal functions.

Equations
@[simp]
theorem category_theory.​graded_object.​comap_eq_hom_app (C : Type u) [category_theory.category C] {β γ : Type w} {f g : β → γ} (h : f = g) (X : γ → C) (b : β) :

@[simp]
theorem category_theory.​graded_object.​comap_eq_inv_app (C : Type u) [category_theory.category C] {β γ : Type w} {f g : β → γ} (h : f = g) (X : γ → C) (b : β) :

The equivalence between β-graded objects and γ-graded objects, given an equivalence between β and γ.

Equations
@[simp]

The total object of a graded object is the coproduct of the graded components.

Equations
@[instance]

The total functor taking a graded object to the coproduct of its graded components is faithful. To prove this, we need to know that the coprojections into the coproduct are monomorphisms, which follows from the fact we have zero morphisms and decidable equality for the grading.

Equations
  • _ = _