mathlib3 documentation

category_theory.functor.const

The constant functor #

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

const J : C ⥤ (J ⥤ C) is the functor that sends an object X : C to the functor J ⥤ C sending every object in J to X, and every morphism to 𝟙 X.

When J is nonempty, const is faithful.

We have (const J).obj X ⋙ F ≅ (const J).obj (F.obj X) for any F : C ⥤ D.

The functor sending X : C to the constant functor J ⥤ C sending everything to X.

Equations
Instances for category_theory.functor.const
@[simp]
theorem category_theory.functor.const_obj_map (J : Type u₁) [category_theory.category J] {C : Type u₂} [category_theory.category C] (X : C) (j j' : J) (f : j j') :
@[simp]
theorem category_theory.functor.const_map_app (J : Type u₁) [category_theory.category J] {C : Type u₂} [category_theory.category C] (X Y : C) (f : X Y) (j : J) :

The contant functor Jᵒᵖ ⥤ Cᵒᵖ sending everything to op X is (naturally isomorphic to) the opposite of the constant functor J ⥤ C sending everything to X.

Equations

The contant functor Jᵒᵖ ⥤ C sending everything to unop X is (naturally isomorphic to) the opposite of the constant functor J ⥤ Cᵒᵖ sending everything to X.

Equations

These are actually equal, of course, but not definitionally equal (the equality requires F.map (𝟙 _) = 𝟙 _). A natural isomorphism is more convenient than an equality between functors (compare id_to_iso).

Equations
@[protected, instance]

If J is nonempty, then the constant functor over J is faithful.