Skip to content

Commit

Permalink
fix(topology/algebra/infinite_sum): tsum_neg doesn't need summable (
Browse files Browse the repository at this point in the history
#13950)

Both sides are 0 in the not-summable case.
  • Loading branch information
kbuzzard committed May 5, 2022
1 parent ec44f45 commit 54af9e9
Showing 1 changed file with 6 additions and 2 deletions.
8 changes: 6 additions & 2 deletions src/topology/algebra/infinite_sum.lean
Expand Up @@ -676,8 +676,12 @@ end
section tsum
variables [t2_space α]

lemma tsum_neg (hf : summable f) : ∑'b, - f b = - ∑'b, f b :=
hf.has_sum.neg.tsum_eq
lemma tsum_neg : ∑'b, - f b = - ∑'b, f b :=
begin
by_cases hf : summable f,
{ exact hf.has_sum.neg.tsum_eq, },
{ simp [tsum_eq_zero_of_not_summable hf, tsum_eq_zero_of_not_summable (mt summable.of_neg hf)] },
end

lemma tsum_sub (hf : summable f) (hg : summable g) : ∑'b, (f b - g b) = ∑'b, f b - ∑'b, g b :=
(hf.has_sum.sub hg.has_sum).tsum_eq
Expand Down

0 comments on commit 54af9e9

Please sign in to comment.