Documentation

Mathlib.CategoryTheory.Equivalence.Symmetry

Functoriality of the symmetry of equivalences #

Using the calculus of mates in CategoryTheory.Adjunction.Mates, we prove that passing to the symmetric equivalence defines an equivalence between C ≌ D and (D ≌ C)ᵒᵖ, and provides the definition of the functor that takes an equivalence to its inverse.

Main definitions #

The forward functor of the equivalence (C ≌ D) ≌ (D ≌ C)ᵒᵖ.

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

    The inverse functor of the equivalence (C ≌ D) ≌ (D ≌ C)ᵒᵖ.

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

      Taking the symmetric of an equivalence induces an equivalence of categories (C ≌ D) ≌ (D ≌ C)ᵒᵖ.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem CategoryTheory.Equivalence.inverseFunctor_map (C : Type u_1) [Category.{u_3, u_1} C] (D : Type u_2) [Category.{u_4, u_2} D] {X✝ Y✝ : C D} (f : X✝ Y✝) :

        The inverse functor sends an equivalence to its inverse.

        Equations
        Instances For

          We can compare the way we obtain a natural isomorphism e.inverse ≅ f.inverse from an isomorphism e ≌ f via inverseFunctor with the way we get one through Iso.isoInverseOfIsoFunctor.

          An "unopped" version of the equivalence `inverseFunctorObj'.

          Equations
          Instances For

            Promoting Equivalence.congrLeft to a functor.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              @[simp]
              theorem CategoryTheory.Equivalence.congrLeftFunctor_map (C : Type u_1) [Category.{u_4, u_1} C] (D : Type u_2) [Category.{u_5, u_2} D] (E : Type u_3) [Category.{u_6, u_3} E] {X✝ Y✝ : C D} (f : X✝ Y✝) :