mathlib3 documentation

category_theory.endofunctor.algebra

Algebras of endofunctors #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines (co)algebras of an endofunctor, and provides the category instance for them. It also defines the forgetful functor from the category of (co)algebras. It is shown that the structure map of the initial algebra of an endofunctor is an isomorphism. Furthermore, it is shown that for an adjunction F ⊣ G the category of algebras over F is equivalent to the category of coalgebras over G.

TODO #

structure category_theory.endofunctor.algebra {C : Type u} [category_theory.category C] (F : C C) :
Type (max u v)

An algebra of an endofunctor; str stands for "structure morphism"

Instances for category_theory.endofunctor.algebra
@[ext]

A morphism between algebras of endofunctor F

Instances for category_theory.endofunctor.algebra.hom
theorem category_theory.endofunctor.algebra.hom.ext {C : Type u} {_inst_1 : category_theory.category C} {F : C C} {A₀ A₁ : category_theory.endofunctor.algebra F} (x y : A₀.hom A₁) (h : x.f = y.f) :
x = y
theorem category_theory.endofunctor.algebra.hom.ext_iff {C : Type u} {_inst_1 : category_theory.category C} {F : C C} {A₀ A₁ : category_theory.endofunctor.algebra F} (x y : A₀.hom A₁) :
x = y x.f = y.f
@[simp]
theorem category_theory.endofunctor.algebra.hom.h {C : Type u} [category_theory.category C] {F : C C} {A₀ A₁ : category_theory.endofunctor.algebra F} (self : A₀.hom A₁) :
F.map self.f A₁.str = A₀.str self.f
@[simp]
theorem category_theory.endofunctor.algebra.hom.h_assoc {C : Type u} [category_theory.category C] {F : C C} {A₀ A₁ : category_theory.endofunctor.algebra F} (self : A₀.hom A₁) {X' : C} (f' : A₁.A X') :
F.map self.f A₁.str f' = A₀.str self.f f'

The identity morphism of an algebra of endofunctor F

Equations
def category_theory.endofunctor.algebra.hom.comp {C : Type u} [category_theory.category C] {F : C C} {A₀ A₁ A₂ : category_theory.endofunctor.algebra F} (f : A₀.hom A₁) (g : A₁.hom A₂) :
A₀.hom A₂

The composition of morphisms between algebras of endofunctor F

Equations
@[simp]
theorem category_theory.endofunctor.algebra.comp_f {C : Type u} [category_theory.category C] {F : C C} {A₀ A₁ A₂ : category_theory.endofunctor.algebra F} (f : A₀ A₁) (g : A₁ A₂) :
(f g).f = f.f g.f
def category_theory.endofunctor.algebra.iso_mk {C : Type u} [category_theory.category C] {F : C C} {A₀ A₁ : category_theory.endofunctor.algebra F} (h : A₀.A A₁.A) (w : F.map h.hom A₁.str = A₀.str h.hom) :
A₀ A₁

To construct an isomorphism of algebras, it suffices to give an isomorphism of the As which commutes with the structure morphisms.

Equations

The forgetful functor from the category of algebras, forgetting the algebraic structure.

Equations
Instances for category_theory.endofunctor.algebra.forget

An algebra morphism with an underlying isomorphism hom in C is an algebra isomorphism.

An algebra morphism with an underlying epimorphism hom in C is an algebra epimorphism.

An algebra morphism with an underlying monomorphism hom in C is an algebra monomorphism.

From a natural transformation α : G → F we get a functor from algebras of F to algebras of G.

Equations

If α and β are two equal natural transformations, then the functors of algebras induced by them are isomorphic. We define it like this as opposed to using eq_to_iso so that the components are nicer to prove lemmas about.

Equations
@[simp]

The inverse of the structure map of an initial algebra

Equations

The structure map of the inital algebra is an isomorphism, hence endofunctors preserve their initial algebras

structure category_theory.endofunctor.coalgebra {C : Type u} [category_theory.category C] (F : C C) :
Type (max u v)

A coalgebra of an endofunctor; str stands for "structure morphism"

Instances for category_theory.endofunctor.coalgebra
theorem category_theory.endofunctor.coalgebra.hom.ext {C : Type u} {_inst_1 : category_theory.category C} {F : C C} {V₀ V₁ : category_theory.endofunctor.coalgebra F} (x y : V₀.hom V₁) (h : x.f = y.f) :
x = y
theorem category_theory.endofunctor.coalgebra.hom.ext_iff {C : Type u} {_inst_1 : category_theory.category C} {F : C C} {V₀ V₁ : category_theory.endofunctor.coalgebra F} (x y : V₀.hom V₁) :
x = y x.f = y.f
@[ext]

A morphism between coalgebras of an endofunctor F

Instances for category_theory.endofunctor.coalgebra.hom
@[simp]
theorem category_theory.endofunctor.coalgebra.hom.h {C : Type u} [category_theory.category C] {F : C C} {V₀ V₁ : category_theory.endofunctor.coalgebra F} (self : V₀.hom V₁) :
V₀.str F.map self.f = self.f V₁.str
@[simp]
theorem category_theory.endofunctor.coalgebra.hom.h_assoc {C : Type u} [category_theory.category C] {F : C C} {V₀ V₁ : category_theory.endofunctor.coalgebra F} (self : V₀.hom V₁) {X' : C} (f' : F.obj V₁.V X') :
V₀.str F.map self.f f' = self.f V₁.str f'

The identity morphism of an algebra of endofunctor F

Equations
def category_theory.endofunctor.coalgebra.hom.comp {C : Type u} [category_theory.category C] {F : C C} {V₀ V₁ V₂ : category_theory.endofunctor.coalgebra F} (f : V₀.hom V₁) (g : V₁.hom V₂) :
V₀.hom V₂

The composition of morphisms between algebras of endofunctor F

Equations
@[simp]
theorem category_theory.endofunctor.coalgebra.comp_f {C : Type u} [category_theory.category C] {F : C C} {V₀ V₁ V₂ : category_theory.endofunctor.coalgebra F} (f : V₀ V₁) (g : V₁ V₂) :
(f g).f = f.f g.f
def category_theory.endofunctor.coalgebra.iso_mk {C : Type u} [category_theory.category C] {F : C C} {V₀ V₁ : category_theory.endofunctor.coalgebra F} (h : V₀.V V₁.V) (w : V₀.str F.map h.hom = h.hom V₁.str) :
V₀ V₁

To construct an isomorphism of coalgebras, it suffices to give an isomorphism of the Vs which commutes with the structure morphisms.

Equations

A coalgebra morphism with an underlying isomorphism hom in C is a coalgebra isomorphism.

An algebra morphism with an underlying epimorphism hom in C is an algebra epimorphism.

An algebra morphism with an underlying monomorphism hom in C is an algebra monomorphism.

From a natural transformation α : F → G we get a functor from coalgebras of F to coalgebras of G.

Equations

If α and β are two equal natural transformations, then the functors of coalgebras induced by them are isomorphic. We define it like this as opposed to using eq_to_iso so that the components are nicer to prove lemmas about.

Equations
theorem category_theory.endofunctor.adjunction.algebra.hom_equiv_naturality_str {C : Type u} [category_theory.category C] {F G : C C} (adj : F G) (A₁ A₂ : category_theory.endofunctor.algebra F) (f : A₁ A₂) :
(adj.hom_equiv A₁.A A₁.A) A₁.str G.map f.f = f.f (adj.hom_equiv A₂.A A₂.A) A₂.str
theorem category_theory.endofunctor.adjunction.coalgebra.hom_equiv_naturality_str_symm {C : Type u} [category_theory.category C] {F G : C C} (adj : F G) (V₁ V₂ : category_theory.endofunctor.coalgebra G) (f : V₁ V₂) :
F.map f.f ((adj.hom_equiv V₂.V V₂.V).symm) V₂.str = ((adj.hom_equiv V₁.V V₁.V).symm) V₁.str f.f

Given an adjunction F ⊣ G, the functor that associates to an algebra over F a coalgebra over G defined via adjunction applied to the structure map.

Equations

Given an adjunction F ⊣ G, the functor that associates to a coalgebra over G an algebra over F defined via adjunction applied to the structure map.

Equations

Given an adjunction, assigning to an algebra over the left adjoint a coalgebra over its right adjoint and going back is isomorphic to the identity functor.

Equations

Given an adjunction, assigning to a coalgebra over the right adjoint an algebra over the left adjoint and going back is isomorphic to the identity functor.

Equations