Differential objects in a category. #
A differential object in a category with zero morphisms and a shift is
an object X
equipped with
a morphism d : obj ⟶ obj⟦1⟧
, such that d^2 = 0
.
We build the category of differential objects, and some basic constructions such as the forgetful functor, zero morphisms and zero objects, and the shift functor on differential objects.
A differential object in a category with zero morphisms and a shift is
an object obj
equipped with
a morphism d : obj ⟶ obj⟦1⟧
, such that d^2 = 0
.
- obj : C
The underlying object of a differential object.
The differential of a differential object.
The differential
d
satisfies thatd² = 0
.
Instances For
A morphism of differential objects is a morphism commuting with the differentials.
The morphism between underlying objects of the two differentiable objects.
- comm : CategoryStruct.comp X.d ((CategoryTheory.shiftFunctor C 1).map self.f) = CategoryStruct.comp self.f Y.d
Instances For
The identity morphism of a differential object.
Equations
- CategoryTheory.DifferentialObject.Hom.id X = { f := CategoryTheory.CategoryStruct.id X.obj, comm := ⋯ }
Instances For
The composition of morphisms of differential objects.
Equations
- f.comp g = { f := CategoryTheory.CategoryStruct.comp f.f g.f, comm := ⋯ }
Instances For
The forgetful functor taking a differential object to its underlying object.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- CategoryTheory.DifferentialObject.instZeroHom = { zero := { f := 0, comm := ⋯ } }
An isomorphism of differential objects gives an isomorphism of the underlying objects.
Equations
Instances For
An isomorphism of differential objects can be constructed from an isomorphism of the underlying objects that commutes with the differentials.
Equations
- CategoryTheory.DifferentialObject.mkIso f hf = { hom := { f := f.hom, comm := hf }, inv := { f := f.inv, comm := ⋯ }, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
A functor F : C ⥤ D
which commutes with shift functors on C
and D
and preserves zero
morphisms can be lifted to a functor DifferentialObject S C ⥤ DifferentialObject S D
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- CategoryTheory.DifferentialObject.instHasForget₂ S C = { forget₂ := CategoryTheory.DifferentialObject.forget S C, forget_comp := ⋯ }
The type of C
-morphisms that can be lifted back to morphisms in the category DifferentialObject
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- CategoryTheory.DifferentialObject.instFunLikeHomSubtypeObj S C X Y = { coe := fun (f : CategoryTheory.DifferentialObject.HomSubtype S C X Y) => ⇑↑f, coe_injective' := ⋯ }
Equations
- One or more equations did not get rendered due to their size.
The category of differential objects itself has a shift functor.
The shift functor on DifferentialObject S C
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The shift functor on DifferentialObject S C
is additive.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The shift by zero is naturally isomorphic to the identity.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.