Order on tropical algebraic structure #
This file defines the orders induced on tropical algebraic structures by the underlying type.
Main declarations #
ConditionallyCompleteLattice (Tropical R)
ConditionallyCompleteLinearOrder (Tropical R)
Implementation notes #
The order induced is the definitionally equal underlying order, which makes the proofs and constructions quicker to implement.
Equations
- instSemilatticeInfTropical = SemilatticeInf.mk (fun (x y : Tropical R) => Tropical.trop (Tropical.untrop x ⊓ Tropical.untrop y)) ⋯ ⋯ ⋯
Equations
- instSemilatticeSupTropical = SemilatticeSup.mk (fun (x y : Tropical R) => Tropical.trop (Tropical.untrop x ⊔ Tropical.untrop y)) ⋯ ⋯ ⋯
Equations
- instLatticeTropical = Lattice.mk SemilatticeInf.inf ⋯ ⋯ ⋯
Equations
- instConditionallyCompleteLatticeTropical = ConditionallyCompleteLattice.mk ⋯ ⋯ ⋯ ⋯
instance
instConditionallyCompleteLinearOrderTropical
{R : Type u_1}
[ConditionallyCompleteLinearOrder R]
:
Equations
- instConditionallyCompleteLinearOrderTropical = ConditionallyCompleteLinearOrder.mk ⋯ LinearOrder.decidableLE LinearOrder.decidableEq LinearOrder.decidableLT ⋯ ⋯