mathlib documentation

category_theory.​single_obj

category_theory.​single_obj

Single-object category

Single object category with a given monoid of endomorphisms. It is defined to facilitate transfering some definitions and lemmas (e.g., conjugacy etc.) from category theory to monoids and groups.

Main definitions

Given a type α with a monoid structure, single_obj α is unit type with category structure such that End (single_obj α).star is the monoid α. This can be extended to a functor Mon ⥤ Cat.

If α is a group, then single_obj α is a groupoid.

An element x : α can be reinterpreted as an element of End (single_obj.star α) using single_obj.to_End.

Implementation notes

@[nolint]
def category_theory.​single_obj  :
Type u → Type

Type tag on unit used to define single-object categories and groupoids.

Equations
@[instance]

One and flip (*) become id and comp for morphisms of the single object category.

Equations
@[instance]

Monoid laws become category laws for the single object category.

Equations

The single object in single_obj α.

Equations

The endomorphisms monoid of the only object in single_obj α is equivalent to the original monoid α.

Equations

There is a 1-1 correspondence between monoid homomorphisms α → β and functors between the corresponding single-object categories. It means that single_obj is a fully faithful functor.

Equations
theorem category_theory.​single_obj.​map_hom_comp {α : Type u} {β : Type v} [monoid α] [monoid β] (f : α →* β) {γ : Type w} [monoid γ] (g : β →* γ) :

def monoid_hom.​to_functor {α : Type u} {β : Type v} [monoid α] [monoid β] :

Reinterpret a monoid homomorphism f : α → β as a functor (single_obj α) ⥤ (single_obj β). See also category_theory.single_obj.map_hom for an equivalence between these types.

Equations
@[simp]
theorem monoid_hom.​comp_to_functor {α : Type u} {β : Type v} [monoid α] [monoid β] (f : α →* β) {γ : Type w} [monoid γ] (g : β →* γ) :

The units in a monoid are (multiplicatively) equivalent to the automorphisms of star when we think of the monoid as a single-object category.

Equations
@[simp]
theorem units.​to_Aut_hom (α : Type u) [monoid α] (x : units α) :

@[simp]
theorem units.​to_Aut_inv (α : Type u) [monoid α] (x : units α) :

The fully faithful functor from Mon to Cat.

Equations
@[instance]

Equations