Documentation

Mathlib.AlgebraicTopology.SimplicialSet.Op

The covariant involution of the category of simplicial sets #

In this file, we define the covariant involution opFunctor : SSetSSet of the category of simplicial sets that is induced by the covariant involution SimplexCategory.op : SimplexCategorySimplexCategory. We use an abbreviation X.op for opFunctor.obj X.

TODO #

The covariant involution of the category of simplicial sets that is induced by SimplexCategory.rev : SimplexCategorySimplexCategory.

Equations
Instances For
    @[reducible, inline]
    abbrev SSet.op (X : SSet) :

    The image of a simplicial set by the involution opFunctor : SSetSSet.

    Equations
    Instances For

      The type of n-simplices of X.op identify to type of n-simplices of X.

      Equations
      Instances For
        theorem SSet.opFunctor_map {X Y : SSet} (f : X Y) {n : SimplexCategoryᵒᵖ} (x : X.op.obj n) :
        theorem SSet.op_map (X : SSet) {n m : SimplexCategoryᵒᵖ} (f : n m) (x : X.op.obj n) :

        The functor opFunctor : SSetSSet is an involution.

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

          The covariant involution opFunctor : SSetSSet, as an equivalence of categories.

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