Nonempty finite linear orders #
This defines NonemptyFinLinOrd
, the category of nonempty finite linear
orders with monotone maps. This is the index category for simplicial objects.
Note: NonemptyFinLinOrd
is not a subcategory of FinBddDistLat
because its morphisms do not
preserve ⊥
and ⊤
.
Equations
- NonemptyFinLinOrd.instCoeSortType = { coe := fun (X : NonemptyFinLinOrd) => ↑X.toLinOrd }
instance
NonemptyFinLinOrd.instConcreteCategoryOrderHomCarrier :
CategoryTheory.ConcreteCategory NonemptyFinLinOrd fun (x1 x2 : NonemptyFinLinOrd) => ↑x1.toLinOrd →o ↑x2.toLinOrd
Equations
@[reducible, inline]
Construct a bundled NonemptyFinLinOrd
from the underlying type and typeclass.
Equations
Instances For
@[reducible, inline]
abbrev
NonemptyFinLinOrd.ofHom
{X Y : Type u}
[Nonempty X]
[LinearOrder X]
[Fintype X]
[Nonempty Y]
[LinearOrder Y]
[Fintype Y]
(f : X →o Y)
:
Typecheck a OrderHom
as a morphism in NonemptyFinLinOrd
.
Instances For
@[simp]
@[simp]
theorem
NonemptyFinLinOrd.comp_apply
{X Y Z : NonemptyFinLinOrd}
(f : X ⟶ Y)
(g : Y ⟶ Z)
(x : ↑X.toLinOrd)
:
theorem
NonemptyFinLinOrd.hom_ext
{X Y : NonemptyFinLinOrd}
{f g : X ⟶ Y}
(hf : LinOrd.Hom.hom f = LinOrd.Hom.hom g)
:
@[simp]
theorem
NonemptyFinLinOrd.hom_ofHom
{X Y : Type u}
[Nonempty X]
[LinearOrder X]
[Fintype X]
[Nonempty Y]
[LinearOrder Y]
[Fintype Y]
(f : X →o Y)
:
@[simp]
Equations
- NonemptyFinLinOrd.instInhabited = { default := NonemptyFinLinOrd.of PUnit.{?u.3 + 1} }
Equations
- One or more equations did not get rendered due to their size.
Constructs an equivalence between nonempty finite linear orders from an order isomorphism between them.
Equations
- NonemptyFinLinOrd.Iso.mk e = { hom := NonemptyFinLinOrd.ofHom ↑e, inv := NonemptyFinLinOrd.ofHom ↑e.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
@[simp]
OrderDual
as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
The equivalence between NonemptyFinLinOrd
and itself induced by OrderDual
both ways.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The forgetful functor NonemptyFinLinOrd ⥤ FinPartOrd
and OrderDual
commute.
Equations
- One or more equations did not get rendered due to their size.