Functors from the category of the ordered set ℕ
#
In this file, we provide a constructor Functor.ofSequence
for functors ℕ ⥤ C
which takes as an input a sequence
of morphisms f : X n ⟶ X (n + 1)
for all n : ℕ
.
We also provide a constructor NatTrans.ofSequence
for natural
transformations between functors ℕ ⥤ C
which allows to check
the naturality condition only for morphisms n ⟶ n + 1
.
The duals of the above for functors ℕᵒᵖ ⥤ C
are given by Functor.ofOpSequence
and
NatTrans.ofOpSequence
.
The morphism X i ⟶ X j
obtained by composing morphisms of
the form X n ⟶ X (n + 1)
when i ≤ j
.
Equations
- CategoryTheory.Functor.OfSequence.map x 0 0 = fun (x : 0 ≤ 0) => CategoryTheory.CategoryStruct.id (x✝ 0)
- CategoryTheory.Functor.OfSequence.map x 0 1 = fun (x_1 : 0 ≤ 1) => x 0
- CategoryTheory.Functor.OfSequence.map x 0 l.succ = fun (x_1 : 0 ≤ l + 1) => CategoryTheory.CategoryStruct.comp (x 0) (CategoryTheory.Functor.OfSequence.map (fun (n : ℕ) => x (n + 1)) 0 l ⋯)
- CategoryTheory.Functor.OfSequence.map x n.succ 0 = fun (a : n + 1 ≤ 0) => nomatch a
- CategoryTheory.Functor.OfSequence.map x k.succ l.succ = fun (x_1 : k + 1 ≤ l + 1) => CategoryTheory.Functor.OfSequence.map (fun (n : ℕ) => x (n + 1)) k l ⋯
Instances For
The functor ℕ ⥤ C
constructed from a sequence of
morphisms f : X n ⟶ X (n + 1)
for all n : ℕ
.
Equations
- CategoryTheory.Functor.ofSequence f = { obj := X, map := fun {i j : ℕ} (φ : i ⟶ j) => CategoryTheory.Functor.OfSequence.map f i j ⋯, map_id := ⋯, map_comp := ⋯ }
Instances For
Constructor for natural transformations F ⟶ G
in ℕ ⥤ C
which takes as inputs
the morphisms F.obj n ⟶ G.obj n
for all n : ℕ
and the naturality condition only
for morphisms of the form n ⟶ n + 1
.
Equations
- CategoryTheory.NatTrans.ofSequence app naturality = { app := app, naturality := ⋯ }
Instances For
The functor ℕᵒᵖ ⥤ C
constructed from a sequence of
morphisms f : X (n + 1) ⟶ X n
for all n : ℕ
.
Equations
- CategoryTheory.Functor.ofOpSequence f = (CategoryTheory.Functor.ofSequence fun (n : ℕ) => (f n).op).leftOp
Instances For
Constructor for natural transformations F ⟶ G
in ℕᵒᵖ ⥤ C
which takes as inputs
the morphisms F.obj ⟨n⟩ ⟶ G.obj ⟨n⟩
for all n : ℕ
and the naturality condition only
for morphisms of the form n ⟶ n + 1
.
Equations
- CategoryTheory.NatTrans.ofOpSequence app naturality = { app := fun (n : ℕᵒᵖ) => app (Opposite.unop n), naturality := ⋯ }