Documentation

Mathlib.Algebra.Order.Interval.Multiset

Algebraic properties of multiset intervals #

This file provides results about the interaction of algebra with Multiset.Ixx.

theorem Multiset.map_add_left_Icc {α : Type u_1} [OrderedCancelAddCommMonoid α] [ExistsAddOfLE α] [LocallyFiniteOrder α] (a b c : α) :
map (fun (x : α) => c + x) (Icc a b) = Icc (c + a) (c + b)
theorem Multiset.map_add_left_Ico {α : Type u_1} [OrderedCancelAddCommMonoid α] [ExistsAddOfLE α] [LocallyFiniteOrder α] (a b c : α) :
map (fun (x : α) => c + x) (Ico a b) = Ico (c + a) (c + b)
theorem Multiset.map_add_left_Ioc {α : Type u_1} [OrderedCancelAddCommMonoid α] [ExistsAddOfLE α] [LocallyFiniteOrder α] (a b c : α) :
map (fun (x : α) => c + x) (Ioc a b) = Ioc (c + a) (c + b)
theorem Multiset.map_add_left_Ioo {α : Type u_1} [OrderedCancelAddCommMonoid α] [ExistsAddOfLE α] [LocallyFiniteOrder α] (a b c : α) :
map (fun (x : α) => c + x) (Ioo a b) = Ioo (c + a) (c + b)
theorem Multiset.map_add_right_Icc {α : Type u_1} [OrderedCancelAddCommMonoid α] [ExistsAddOfLE α] [LocallyFiniteOrder α] (a b c : α) :
map (fun (x : α) => x + c) (Icc a b) = Icc (a + c) (b + c)
theorem Multiset.map_add_right_Ico {α : Type u_1} [OrderedCancelAddCommMonoid α] [ExistsAddOfLE α] [LocallyFiniteOrder α] (a b c : α) :
map (fun (x : α) => x + c) (Ico a b) = Ico (a + c) (b + c)
theorem Multiset.map_add_right_Ioc {α : Type u_1} [OrderedCancelAddCommMonoid α] [ExistsAddOfLE α] [LocallyFiniteOrder α] (a b c : α) :
map (fun (x : α) => x + c) (Ioc a b) = Ioc (a + c) (b + c)
theorem Multiset.map_add_right_Ioo {α : Type u_1} [OrderedCancelAddCommMonoid α] [ExistsAddOfLE α] [LocallyFiniteOrder α] (a b c : α) :
map (fun (x : α) => x + c) (Ioo a b) = Ioo (a + c) (b + c)