Bundled exact functors #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We say that a functor F
is left exact if it preserves finite limits, it is right exact if it
preserves finite colimits, and it is exact if it is both left exact and right exact.
In this file, we define the categories of bundled left exact, right exact and exact functors.
Bundled left-exact functors.
Equations
- (C ⥤ₗ D) = category_theory.full_subcategory (λ (F : C ⥤ D), nonempty (category_theory.limits.preserves_finite_limits F))
Instances for category_theory.LeftExactFunctor
A left exact functor is in particular a functor.
Equations
Instances for category_theory.LeftExactFunctor.forget
Bundled right-exact functors.
Equations
- (C ⥤ᵣ D) = category_theory.full_subcategory (λ (F : C ⥤ D), nonempty (category_theory.limits.preserves_finite_colimits F))
Instances for category_theory.RightExactFunctor
A right exact functor is in particular a functor.
Equations
Instances for category_theory.RightExactFunctor.forget
Bundled exact functors.
Equations
- (C ⥤ₑ D) = category_theory.full_subcategory (λ (F : C ⥤ D), nonempty (category_theory.limits.preserves_finite_limits F) ∧ nonempty (category_theory.limits.preserves_finite_colimits F))
Instances for category_theory.ExactFunctor
An exact functor is in particular a functor.
Equations
Instances for category_theory.ExactFunctor.forget
Turn an exact functor into a left exact functor.
Instances for category_theory.LeftExactFunctor.of_exact
Turn an exact functor into a left exact functor.
Instances for category_theory.RightExactFunctor.of_exact
Turn a left exact functor into an object of the category LeftExactFunctor C D
.
Equations
- category_theory.LeftExactFunctor.of F = {obj := F, property := _}
Turn a right exact functor into an object of the category RightExactFunctor C D
.
Equations
- category_theory.RightExactFunctor.of F = {obj := F, property := _}
Turn an exact functor into an object of the category ExactFunctor C D
.
Equations
- category_theory.ExactFunctor.of F = {obj := F, property := _}