Zulip Chat Archive
Stream: new members
Topic: Sub of Finset.sum
Junjie Bai (Mar 27 2024 at 07:24):
Is there any function can prove that
variable {a : ℤ} (f : ℚ → ℚ)
example : (∑ x in Icc 0 (a + 1), f x) - (∑ x in Icc 0 a, f x) = f (a + 1) := by sorry
Kevin Buzzard (Mar 27 2024 at 08:35):
I don't think that's true. What if a=-37?
Junjie Bai (Mar 27 2024 at 09:02):
You're right. I think this is what I mean:
variable {a : ℤ} (f : ℚ → ℚ)
example (ha : a ≥ 0) : (∑ x in Icc 0 (a + 1), f x) - (∑ x in Icc 0 a, f x) = f (a + 1) := by sorry
Eric Wieser (Mar 27 2024 at 09:05):
We won't have this lemma, but it follows in not too many steps. Can you see how to break the problem down? Try doing so with have
statements, and using exact?
for each
Johan Commelin (Mar 27 2024 at 09:05):
Can you prove Icc 0 (a + 1) = Icc 0 a \cup {a+1}
?
Eric Wieser (Mar 27 2024 at 09:06):
(or possibly, Icc 0 (a + 1) = (Icc 0 a).cons a sorry
, which is a slightly stronger result)
Junjie Bai (Mar 28 2024 at 02:07):
I think I can solve this now, thanks a lot!
Last updated: May 02 2025 at 03:31 UTC