mathlib3 documentation

algebra.tropical.big_operators

Tropicalization of finitary operations #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file provides the "big-op" or notation-based finitary operations on tropicalized types. This allows easy conversion between sums to Infs and prods to sums. Results here are important for expressing that evaluation of tropical polynomials are the minimum over a finite piecewise collection of linear functions.

Main declarations #

Implementation notes #

No concrete (semi)ring is used here, only ones with inferrable order/lattice structure, to support real, rat, ereal, and others (erat is not yet defined).

Minima over list α are defined as producing a value in with_top α so proofs about lists do not directly transfer to minima over multisets or finsets.

theorem trop_sum {R : Type u_1} {S : Type u_2} [add_comm_monoid R] (s : finset S) (f : S R) :
tropical.trop (s.sum (λ (i : S), f i)) = s.prod (λ (i : S), tropical.trop (f i))
theorem untrop_prod {R : Type u_1} {S : Type u_2} [add_comm_monoid R] (s : finset S) (f : S tropical R) :
tropical.untrop (s.prod (λ (i : S), f i)) = s.sum (λ (i : S), tropical.untrop (f i))
theorem finset.trop_inf {R : Type u_1} {S : Type u_2} [linear_order R] [order_top R] (s : finset S) (f : S R) :
tropical.trop (s.inf f) = s.sum (λ (i : S), tropical.trop (f i))
theorem trop_Inf_image {R : Type u_1} {S : Type u_2} [conditionally_complete_linear_order R] (s : finset S) (f : S with_top R) :
tropical.trop (has_Inf.Inf (f '' s)) = s.sum (λ (i : S), tropical.trop (f i))
theorem trop_infi {R : Type u_1} {S : Type u_2} [conditionally_complete_linear_order R] [fintype S] (f : S with_top R) :
tropical.trop ( (i : S), f i) = finset.univ.sum (λ (i : S), tropical.trop (f i))
theorem finset.untrop_sum' {R : Type u_1} {S : Type u_2} [linear_order R] [order_top R] (s : finset S) (f : S tropical R) :
tropical.untrop (s.sum (λ (i : S), f i)) = s.inf (tropical.untrop f)
theorem untrop_sum_eq_Inf_image {R : Type u_1} {S : Type u_2} [conditionally_complete_linear_order R] (s : finset S) (f : S tropical (with_top R)) :
theorem untrop_sum {R : Type u_1} {S : Type u_2} [conditionally_complete_linear_order R] [fintype S] (f : S tropical (with_top R)) :
tropical.untrop (finset.univ.sum (λ (i : S), f i)) = (i : S), tropical.untrop (f i)
theorem finset.untrop_sum {R : Type u_1} {S : Type u_2} [conditionally_complete_linear_order R] (s : finset S) (f : S tropical (with_top R)) :
tropical.untrop (s.sum (λ (i : S), f i)) = (i : s), tropical.untrop (f i)

Note we cannot use i ∈ s instead of i : s here as it is simply not true on conditionally complete lattices!