Documentation

Mathlib.Algebra.Star.BigOperators

Big-operators lemmas about star algebraic operations #

These results are kept separate from Algebra.Star.Basic to avoid it needing to import Finset.

@[simp]
theorem star_prod {R : Type u_1} [CommMonoid R] [StarMul R] {α : Type u_2} (s : Finset α) (f : αR) :
star (∏ xs, f x) = xs, star (f x)
@[simp]
theorem star_sum {R : Type u_1} [AddCommMonoid R] [StarAddMonoid R] {α : Type u_2} (s : Finset α) (f : αR) :
star (∑ xs, f x) = xs, star (f x)
theorem isSelfAdjoint_sum {R : Type u_1} {ι : Type u_2} [AddCommMonoid R] [StarAddMonoid R] (s : Finset ι) {x : ιR} (h : is, IsSelfAdjoint (x i)) :
IsSelfAdjoint (∑ is, x i)