Documentation

Mathlib.CategoryTheory.ObjectProperty.Orthogonal

Orthogonal of a property of objects #

Let P be a property of objects in a category with zero morphisms. We define P.rightOrthogonal as the property of objects Y such that any map f : X ⟶ Y vanishes when P X holds. Similarly, we define P.leftOrthogonal as the property of objects X such that any map f : X ⟶ Y vanishes when P Y holds.

In a category with zero morphisms, the right orthogonal of a property of objects P is the property of objects Y such that any map X ⟶ Y vanishes when P X holds.

Equations
Instances For
    theorem CategoryTheory.ObjectProperty.rightOrthogonal_iff {C : Type u} [Category.{v, u} C] [Limits.HasZeroMorphisms C] (P : ObjectProperty C) (Y : C) :
    P.rightOrthogonal Y ∀ ⦃X : C⦄ (f : X Y), P Xf = 0

    In a category with zero morphisms, the left orthogonal of a property of objects P is the property of objects X such that any map X ⟶ Y vanishes when P Y holds.

    Equations
    Instances For
      theorem CategoryTheory.ObjectProperty.leftOrthogonal_iff {C : Type u} [Category.{v, u} C] [Limits.HasZeroMorphisms C] (P : ObjectProperty C) (X : C) :
      P.leftOrthogonal X ∀ ⦃Y : C⦄ (f : X Y), P Yf = 0