Documentation

Mathlib.CategoryTheory.ObjectProperty.Opposite

The opposite of a property of objects #

The property of objects of Cᵒᵖ corresponding to P : ObjectProperty C.

Equations
Instances For

    The property of objects of C corresponding to P : ObjectProperty Cᵒᵖ.

    Equations
    Instances For

      The bijection Subtype P.opSubtype P for P : ObjectProperty C.

      Equations
      Instances For
        @[simp]
        theorem CategoryTheory.ObjectProperty.op_ofObj {C : Type u} [Category.{v, u} C] {ι : Type u_1} (X : ιC) :
        (ofObj X).op = ofObj fun (i : ι) => Opposite.op (X i)
        @[simp]
        theorem CategoryTheory.ObjectProperty.unop_ofObj {C : Type u} [Category.{v, u} C] {ι : Type u_1} (X : ιCᵒᵖ) :
        (ofObj X).unop = ofObj fun (i : ι) => Opposite.unop (X i)