Documentation

Mathlib.Algebra.Tropical.Lattice

Order on tropical algebraic structure #

This file defines the orders induced on tropical algebraic structures by the underlying type.

Main declarations #

Implementation notes #

The order induced is the definitionally equal underlying order, which makes the proofs and constructions quicker to implement.

instance instSupTropical {R : Type u_1} [Sup R] :
Equations
instance instInfTropical {R : Type u_1} [Inf R] :
Equations
Equations
  • instSemilatticeInfTropical = let __src := instInfTropical; let __src_1 := Tropical.instPartialOrderTropical; SemilatticeInf.mk
Equations
  • instSemilatticeSupTropical = let __src := instSupTropical; let __src_1 := Tropical.instPartialOrderTropical; SemilatticeSup.mk
instance instLatticeTropical {R : Type u_1} [Lattice R] :
Equations
  • instLatticeTropical = let __src := instSemilatticeInfTropical; let __src_1 := instSemilatticeSupTropical; Lattice.mk
instance instSupSetTropical {R : Type u_1} [SupSet R] :
Equations
instance instInfSetTropical {R : Type u_1} [InfSet R] :
Equations
Equations
  • instConditionallyCompleteLatticeTropical = let __src := instInfTropical; let __src_1 := instSupTropical; let __src_2 := instLatticeTropical; ConditionallyCompleteLattice.mk
Equations
  • One or more equations did not get rendered due to their size.