mathlib3 documentation

category_theory.discrete_category

Discrete categories #

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

We define discrete α as a structure containing a term a : α for any type α, and use this type alias to provide a small_category instance whose only morphisms are the identities.

There is an annoying technical difficulty that it has turned out to be inconvenient to allow categories with morphisms living in Prop, so instead of defining X ⟶ Y in discrete α as X = Y, one might define it as plift (X = Y). In fact, to allow discrete α to be a small_category (i.e. with morphisms in the same universe as the objects), we actually define the hom type X ⟶ Y as ulift (plift (X = Y)).

discrete.functor promotes a function f : I → C (for any category C) to a functor discrete.functor f : discrete I ⥤ C.

Similarly, discrete.nat_trans and discrete.nat_iso promote I-indexed families of morphisms, or I-indexed families of isomorphisms to natural transformations or natural isomorphism.

We show equivalences of types are the same as (categorical) equivalences of the corresponding discrete categories.

theorem category_theory.discrete.ext_iff {α : Type u₁} (x y : category_theory.discrete α) :
x = y x.as = y.as
@[ext]
structure category_theory.discrete (α : Type u₁) :
Type u₁
  • as : α

A wrapper for promoting any type to a category, with the only morphisms being equalities.

Instances for category_theory.discrete
theorem category_theory.discrete.ext {α : Type u₁} (x y : category_theory.discrete α) (h : x.as = y.as) :
x = y
@[simp]
theorem category_theory.discrete.mk_as {α : Type u₁} (X : category_theory.discrete α) :
{as := X.as} = X

discrete α is equivalent to the original type α.

Equations
@[protected, instance]

The "discrete" category on a type, whose morphisms are equalities.

Because we do not allow morphisms in Prop (only in Type), somewhat annoyingly we have to define X ⟶ Y as ulift (plift (X = Y)).

See https://stacks.math.columbia.edu/tag/001A

Equations

A simple tactic to run cases on any discrete α hypotheses.

A simple tactic to run cases on any discrete α hypotheses.

theorem category_theory.discrete.eq_of_hom {α : Type u₁} {X Y : category_theory.discrete α} (i : X Y) :
X.as = Y.as

Extract the equation from a morphism in a discrete category.

@[reducible]
def category_theory.discrete.eq_to_hom {α : Type u₁} {X Y : category_theory.discrete α} (h : X.as = Y.as) :
X Y

Promote an equation between the wrapped terms in X Y : discrete α to a morphism X ⟶ Y in the discrete category.

@[reducible]
def category_theory.discrete.eq_to_iso {α : Type u₁} {X Y : category_theory.discrete α} (h : X.as = Y.as) :
X Y

Promote an equation between the wrapped terms in X Y : discrete α to an isomorphism X ≅ Y in the discrete category.

@[reducible]
def category_theory.discrete.eq_to_hom' {α : Type u₁} {a b : α} (h : a = b) :
{as := a} {as := b}

A variant of eq_to_hom that lifts terms to the discrete category.

@[reducible]
def category_theory.discrete.eq_to_iso' {α : Type u₁} {a b : α} (h : a = b) :
{as := a} {as := b}

A variant of eq_to_iso that lifts terms to the discrete category.

@[simp]
theorem category_theory.discrete.id_def {α : Type u₁} (X : category_theory.discrete α) :
{down := {down := _}} = 𝟙 X

Any function I → C gives a functor discrete I ⥤ C.

Equations
Instances for category_theory.discrete.functor
@[simp]
theorem category_theory.discrete.functor_obj {C : Type u₂} [category_theory.category C] {I : Type u₁} (F : I C) (i : I) :

The discrete functor induced by a composition of maps can be written as a composition of two discrete functors.

Equations

For functors out of a discrete category, a natural transformation is just a collection of maps, as the naturality squares are trivial.

Equations

For functors out of a discrete category, a natural isomorphism is just a collection of isomorphisms, as the naturality squares are trivial.

Equations
@[simp]

Every functor F from a discrete category is naturally isomorphic (actually, equal) to discrete.functor (F.obj).

Equations
@[simp]