Documentation

Mathlib.CategoryTheory.Monoidal.Subcategory

Full monoidal subcategories #

Given a monoidal category C and a monoidal predicate on C, that is a function P : C → Prop closed under 𝟙_ and , we can put a monoidal structure on {X : C // P X} (the category structure is defined in Mathlib.CategoryTheory.FullSubcategory).

When C is also braided/symmetric, the full monoidal subcategory also inherits the braided/symmetric structure.

TODO #

A property C → Prop is a monoidal predicate if it is closed under 𝟙_ and .

  • prop_id : P (𝟙_ C)
  • prop_tensor {X Y : C} : P XP YP (tensorObj X Y)
Instances
    Equations
    • One or more equations did not get rendered due to their size.
    @[simp]
    theorem CategoryTheory.MonoidalCategory.instMonoidalCategoryStructFullSubcategory_tensorHom {C : Type u} [Category.{v, u} C] [MonoidalCategory C] (P : CProp) [MonoidalPredicate P] {X₁✝ Y₁✝ X₂✝ Y₂✝ : FullSubcategory P} (f : X₁✝ Y₁✝) (g : X₂✝ Y₂✝) :

    When P is a monoidal predicate, the full subcategory for P inherits the monoidal structure of C.

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

    The forgetful monoidal functor from a full monoidal subcategory into the original category ("forgetting" the condition).

    Equations
    • One or more equations did not get rendered due to their size.
    instance CategoryTheory.MonoidalCategory.instMonoidalFullSubcategoryMap {C : Type u} [Category.{v, u} C] [MonoidalCategory C] {P : CProp} [MonoidalPredicate P] {P' : CProp} [MonoidalPredicate P'] (h : ∀ ⦃X : C⦄, P XP' X) :
    (FullSubcategory.map h).Monoidal

    An implication of predicates P → P' induces a monoidal functor between full monoidal subcategories.

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

    The braided structure on a full subcategory inherited by the braided structure on C.

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

    The forgetful braided functor from a full braided subcategory into the original category ("forgetting" the condition).

    Equations
    instance CategoryTheory.MonoidalCategory.instBraidedFullSubcategoryMap {C : Type u} [Category.{v, u} C] [MonoidalCategory C] {P : CProp} [MonoidalPredicate P] [BraidedCategory C] {P' : CProp} [MonoidalPredicate P'] (h : ∀ ⦃X : C⦄, P XP' X) :

    An implication of predicates P → P' induces a braided functor between full braided subcategories.

    Equations

    A property C → Prop is a closed predicate if it is closed under taking internal homs

    • prop_ihom {X Y : C} : P XP YP ((ihom X).obj Y)
    Instances
      Equations
      • One or more equations did not get rendered due to their size.