Documentation

Mathlib.CategoryTheory.Closed.Ideal

Exponential ideals #

An exponential ideal of a cartesian closed category C is a subcategory D ⊆ C such that for any B : D and A : C, the exponential A ⟹ B is in D: resembling ring theoretic ideals. We define the notion here for inclusion functors i : D ⥤ C rather than explicit subcategories to preserve the principle of equivalence.

We additionally show that if C is cartesian closed and i : D ⥤ C is a reflective functor, the following are equivalent.

The subcategory D of C expressed as an inclusion functor is an exponential ideal if B ∈ D implies A ⟹ B ∈ D for all A.

  • exp_closed {B : C} : B i.essImage∀ (A : C), (AB) i.essImage
Instances
    theorem CategoryTheory.ExponentialIdeal.mk' {C : Type u₁} {D : Type u₂} [Category.{v₁, u₁} C] [Category.{v₁, u₂} D] (i : Functor D C) [ChosenFiniteProducts C] [CartesianClosed C] (h : ∀ (B : D) (A : C), (Ai.obj B) i.essImage) :

    To show i is an exponential ideal it suffices to show that A ⟹ iB is "in" D for any A in C and B in D.

    The entire category viewed as a subcategory is an exponential ideal.

    def CategoryTheory.exponentialIdealReflective {C : Type u₁} {D : Type u₂} [Category.{v₁, u₁} C] [Category.{v₁, u₂} D] (i : Functor D C) [ChosenFiniteProducts C] [CartesianClosed C] (A : C) [Reflective i] [ExponentialIdeal i] :
    i.comp ((exp A).comp ((reflector i).comp i)) i.comp (exp A)

    If D is a reflective subcategory, the property of being an exponential ideal is equivalent to the presence of a natural isomorphism i ⋙ exp A ⋙ leftAdjoint i ⋙ i ≅ i ⋙ exp A, that is: (A ⟹ iB) ≅ i L (A ⟹ iB), naturally in B. The converse is given in ExponentialIdeal.mk_of_iso.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem CategoryTheory.ExponentialIdeal.mk_of_iso {C : Type u₁} {D : Type u₂} [Category.{v₁, u₁} C] [Category.{v₁, u₂} D] (i : Functor D C) [ChosenFiniteProducts C] [CartesianClosed C] [Reflective i] (h : (A : C) → i.comp ((exp A).comp ((reflector i).comp i)) i.comp (exp A)) :

      Given a natural isomorphism i ⋙ exp A ⋙ leftAdjoint i ⋙ i ≅ i ⋙ exp A, we can show i is an exponential ideal.

      Given a reflective subcategory D of a category with chosen finite products C, D admits finite chosen products.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[instance 10]

        If the reflector preserves binary products, the subcategory is an exponential ideal. This is the converse of preservesBinaryProductsOfExponentialIdeal.

        If i witnesses that D is a reflective subcategory and an exponential ideal, then D is itself cartesian closed.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          We construct a bijection between morphisms L(A ⊗ B) ⟶ X and morphisms LA ⊗ LB ⟶ X. This bijection has two key properties:

          Together these help show that L preserves binary products. This should be considered internal implementation towards preservesBinaryProductsOfExponentialIdeal.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For

            The bijection allows us to show that prodComparison L A B is an isomorphism, where the inverse is the forward map of the identity morphism.

            If a reflective subcategory is an exponential ideal, then the reflector preserves binary products. This is the converse of exponentialIdeal_of_preserves_binary_products.

            If a reflective subcategory is an exponential ideal, then the reflector preserves finite products.