Order instances on Shrink #
If α : Type v
is u
-small, we transport various order related
instances on α
to Shrink.{u} α
.
Equations
- instPreorderShrink α = Preorder.mk ⋯ ⋯ ⋯
The order isomorphism α ≃o Shrink.{u} α
.
Equations
- orderIsoShrink α = { toEquiv := equivShrink α, map_rel_iff' := ⋯ }
Instances For
@[simp]
@[simp]
theorem
orderIsoShrink_symm_apply
{α : Type v}
[Small.{u, v} α]
[Preorder α]
(a : Shrink.{u, v} α)
:
Equations
Equations
- One or more equations did not get rendered due to their size.
Equations
- instBotShrink = { bot := (equivShrink α) ⊥ }
@[simp]
Equations
- instTopShrink = { top := (equivShrink α) ⊤ }
@[simp]
Equations
Equations
noncomputable instance
instSuccOrderShrink
{α : Type v}
[Small.{u, v} α]
[Preorder α]
[SuccOrder α]
:
Equations
noncomputable instance
instPredOrderShrink
{α : Type v}
[Small.{u, v} α]
[Preorder α]
[PredOrder α]
: