Documentation

Mathlib.Algebra.BigOperators.RingEquiv

Results about mapping big operators across ring equivalences #

theorem RingEquiv.map_list_prod {R : Type u_2} {S : Type u_3} [Semiring R] [Semiring S] (f : R ≃+* S) (l : List R) :
f l.prod = (List.map (f) l).prod
theorem RingEquiv.map_list_sum {R : Type u_2} {S : Type u_3} [NonAssocSemiring R] [NonAssocSemiring S] (f : R ≃+* S) (l : List R) :
f l.sum = (List.map (f) l).sum
theorem RingEquiv.unop_map_list_prod {R : Type u_2} {S : Type u_3} [Semiring R] [Semiring S] (f : R ≃+* Sᵐᵒᵖ) (l : List R) :
(f l.prod).unop = (List.map (MulOpposite.unop f) l).reverse.prod

An isomorphism into the opposite ring acts on the product by acting on the reversed elements

theorem RingEquiv.map_multiset_prod {R : Type u_2} {S : Type u_3} [CommSemiring R] [CommSemiring S] (f : R ≃+* S) (s : Multiset R) :
f s.prod = (Multiset.map (f) s).prod
theorem RingEquiv.map_multiset_sum {R : Type u_2} {S : Type u_3} [NonAssocSemiring R] [NonAssocSemiring S] (f : R ≃+* S) (s : Multiset R) :
f s.sum = (Multiset.map (f) s).sum
theorem RingEquiv.map_prod {α : Type u_1} {R : Type u_2} {S : Type u_3} [CommSemiring R] [CommSemiring S] (g : R ≃+* S) (f : αR) (s : Finset α) :
g (s.prod fun (x : α) => f x) = s.prod fun (x : α) => g (f x)
theorem RingEquiv.map_sum {α : Type u_1} {R : Type u_2} {S : Type u_3} [NonAssocSemiring R] [NonAssocSemiring S] (g : R ≃+* S) (f : αR) (s : Finset α) :
g (s.sum fun (x : α) => f x) = s.sum fun (x : α) => g (f x)