File tree Expand file tree Collapse file tree 1 file changed +8
-0
lines changed Expand file tree Collapse file tree 1 file changed +8
-0
lines changed Original file line number Diff line number Diff line change @@ -132,6 +132,14 @@ theorem four_pow_le_two_mul_add_one_mul_central_binom (n : ℕ) :
132
132
_ = (2 * n + 1 ) * choose (2 * n) n := by simp
133
133
#align nat.four_pow_le_two_mul_add_one_mul_central_binom Nat.four_pow_le_two_mul_add_one_mul_central_binom
134
134
135
+ /-- **Zhu Shijie's identity** aka hockey-stick identity. -/
136
+ theorem sum_Icc_choose (n k : ℕ) : ∑ m in Icc k n, m.choose k = (n + 1 ).choose (k + 1 ) := by
137
+ cases' le_or_gt k n with h h
138
+ · induction' n, h using le_induction with n _ ih; · simp
139
+ rw [← Ico_insert_right (by linarith), sum_insert (by simp),
140
+ show Ico k (n + 1 ) = Icc k n by rfl, ih, choose_succ_succ' (n + 1 )]
141
+ · rw [choose_eq_zero_of_lt (by linarith), Icc_eq_empty_of_lt h, sum_empty]
142
+
135
143
end Nat
136
144
137
145
theorem Int.alternating_sum_range_choose {n : ℕ} :
You can’t perform that action at this time.
0 commit comments