Documentation

Mathlib.Algebra.BigOperators.Module

Summation by parts #

theorem Finset.sum_Ico_by_parts {R : Type u_1} {M : Type u_2} [Ring R] [AddCommGroup M] [Module R M] (f : R) (g : M) {m n : } (hmn : m < n) :
iIco m n, f i g i = f (n - 1) irange n, g i - f m irange m, g i - iIco m (n - 1), (f (i + 1) - f i) irange (i + 1), g i

Summation by parts, also known as Abel's lemma or an Abel transformation

theorem Finset.sum_Ioc_by_parts {R : Type u_1} {M : Type u_2} [Ring R] [AddCommGroup M] [Module R M] (f : R) (g : M) {m n : } (hmn : m < n) :
iIoc m n, f i g i = f n irange (n + 1), g i - f (m + 1) irange (m + 1), g i - iIoc m (n - 1), (f (i + 1) - f i) irange (i + 1), g i
theorem Finset.sum_range_by_parts {R : Type u_1} {M : Type u_2} [Ring R] [AddCommGroup M] [Module R M] (f : R) (g : M) (n : ) :
irange n, f i g i = f (n - 1) irange n, g i - irange (n - 1), (f (i + 1) - f i) irange (i + 1), g i

Summation by parts for ranges