![]() |
Metamath Proof Explorer |
< Previous
Next >
Nearby theorems |
|
Mirrors > Home > MPE Home > Th. List > trirecip | Structured version Visualization version GIF version |
Description: The sum of the reciprocals of the triangle numbers converge to two. This is Metamath 100 proof #42. (Contributed by Scott Fenton, 23-Apr-2014.) (Revised by Mario Carneiro, 22-May-2014.) |
Ref | Expression |
---|---|
trirecip | ⊢ Σ𝑘 ∈ ℕ (2 / (𝑘 · (𝑘 + 1))) = 2 |
Step | Hyp | Ref | Expression |
---|---|---|---|
1 | 2cnd 12189 | . . . 4 ⊢ (𝑘 ∈ ℕ → 2 ∈ ℂ) | |
2 | peano2nn 12123 | . . . . . 6 ⊢ (𝑘 ∈ ℕ → (𝑘 + 1) ∈ ℕ) | |
3 | nnmulcl 12135 | . . . . . 6 ⊢ ((𝑘 ∈ ℕ ∧ (𝑘 + 1) ∈ ℕ) → (𝑘 · (𝑘 + 1)) ∈ ℕ) | |
4 | 2, 3 | mpdan 685 | . . . . 5 ⊢ (𝑘 ∈ ℕ → (𝑘 · (𝑘 + 1)) ∈ ℕ) |
5 | 4 | nncnd 12127 | . . . 4 ⊢ (𝑘 ∈ ℕ → (𝑘 · (𝑘 + 1)) ∈ ℂ) |
6 | 4 | nnne0d 12161 | . . . 4 ⊢ (𝑘 ∈ ℕ → (𝑘 · (𝑘 + 1)) ≠ 0) |
7 | 1, 5, 6 | divrecd 11892 | . . 3 ⊢ (𝑘 ∈ ℕ → (2 / (𝑘 · (𝑘 + 1))) = (2 · (1 / (𝑘 · (𝑘 + 1))))) |
8 | 7 | sumeq2i 15544 | . 2 ⊢ Σ𝑘 ∈ ℕ (2 / (𝑘 · (𝑘 + 1))) = Σ𝑘 ∈ ℕ (2 · (1 / (𝑘 · (𝑘 + 1)))) |
9 | nnuz 12760 | . . . . 5 ⊢ ℕ = (ℤ≥‘1) | |
10 | 1zzd 12492 | . . . . 5 ⊢ (⊤ → 1 ∈ ℤ) | |
11 | id 22 | . . . . . . . . 9 ⊢ (𝑛 = 𝑘 → 𝑛 = 𝑘) | |
12 | oveq1 7358 | . . . . . . . . 9 ⊢ (𝑛 = 𝑘 → (𝑛 + 1) = (𝑘 + 1)) | |
13 | 11, 12 | oveq12d 7369 | . . . . . . . 8 ⊢ (𝑛 = 𝑘 → (𝑛 · (𝑛 + 1)) = (𝑘 · (𝑘 + 1))) |
14 | 13 | oveq2d 7367 | . . . . . . 7 ⊢ (𝑛 = 𝑘 → (1 / (𝑛 · (𝑛 + 1))) = (1 / (𝑘 · (𝑘 + 1)))) |
15 | eqid 2737 | . . . . . . 7 ⊢ (𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1)))) = (𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1)))) | |
16 | ovex 7384 | . . . . . . 7 ⊢ (1 / (𝑘 · (𝑘 + 1))) ∈ V | |
17 | 14, 15, 16 | fvmpt 6945 | . . . . . 6 ⊢ (𝑘 ∈ ℕ → ((𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1))))‘𝑘) = (1 / (𝑘 · (𝑘 + 1)))) |
18 | 17 | adantl 482 | . . . . 5 ⊢ ((⊤ ∧ 𝑘 ∈ ℕ) → ((𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1))))‘𝑘) = (1 / (𝑘 · (𝑘 + 1)))) |
19 | 4 | nnrecred 12162 | . . . . . . 7 ⊢ (𝑘 ∈ ℕ → (1 / (𝑘 · (𝑘 + 1))) ∈ ℝ) |
20 | 19 | recnd 11141 | . . . . . 6 ⊢ (𝑘 ∈ ℕ → (1 / (𝑘 · (𝑘 + 1))) ∈ ℂ) |
21 | 20 | adantl 482 | . . . . 5 ⊢ ((⊤ ∧ 𝑘 ∈ ℕ) → (1 / (𝑘 · (𝑘 + 1))) ∈ ℂ) |
22 | 15 | trireciplem 15707 | . . . . . . 7 ⊢ seq1( + , (𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1))))) ⇝ 1 |
23 | 22 | a1i 11 | . . . . . 6 ⊢ (⊤ → seq1( + , (𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1))))) ⇝ 1) |
24 | climrel 15334 | . . . . . . 7 ⊢ Rel ⇝ | |
25 | 24 | releldmi 5901 | . . . . . 6 ⊢ (seq1( + , (𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1))))) ⇝ 1 → seq1( + , (𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1))))) ∈ dom ⇝ ) |
26 | 23, 25 | syl 17 | . . . . 5 ⊢ (⊤ → seq1( + , (𝑛 ∈ ℕ ↦ (1 / (𝑛 · (𝑛 + 1))))) ∈ dom ⇝ ) |
27 | 2cnd 12189 | . . . . 5 ⊢ (⊤ → 2 ∈ ℂ) | |
28 | 9, 10, 18, 21, 26, 27 | isummulc2 15607 | . . . 4 ⊢ (⊤ → (2 · Σ𝑘 ∈ ℕ (1 / (𝑘 · (𝑘 + 1)))) = Σ𝑘 ∈ ℕ (2 · (1 / (𝑘 · (𝑘 + 1))))) |
29 | 9, 10, 18, 21, 23 | isumclim 15602 | . . . . 5 ⊢ (⊤ → Σ𝑘 ∈ ℕ (1 / (𝑘 · (𝑘 + 1))) = 1) |
30 | 29 | oveq2d 7367 | . . . 4 ⊢ (⊤ → (2 · Σ𝑘 ∈ ℕ (1 / (𝑘 · (𝑘 + 1)))) = (2 · 1)) |
31 | 28, 30 | eqtr3d 2779 | . . 3 ⊢ (⊤ → Σ𝑘 ∈ ℕ (2 · (1 / (𝑘 · (𝑘 + 1)))) = (2 · 1)) |
32 | 31 | mptru 1548 | . 2 ⊢ Σ𝑘 ∈ ℕ (2 · (1 / (𝑘 · (𝑘 + 1)))) = (2 · 1) |
33 | 2t1e2 12274 | . 2 ⊢ (2 · 1) = 2 | |
34 | 8, 32, 33 | 3eqtri 2769 | 1 ⊢ Σ𝑘 ∈ ℕ (2 / (𝑘 · (𝑘 + 1))) = 2 |
Colors of variables: wff setvar class |
Syntax hints: = wceq 1541 ⊤wtru 1542 ∈ wcel 2106 class class class wbr 5103 ↦ cmpt 5186 dom cdm 5631 ‘cfv 6493 (class class class)co 7351 ℂcc 11007 1c1 11010 + caddc 11012 · cmul 11014 / cdiv 11770 ℕcn 12111 2c2 12166 seqcseq 13860 ⇝ cli 15326 Σcsu 15530 |
This theorem was proved from axioms: ax-mp 5 ax-1 6 ax-2 7 ax-3 8 ax-gen 1797 ax-4 1811 ax-5 1913 ax-6 1971 ax-7 2011 ax-8 2108 ax-9 2116 ax-10 2137 ax-11 2154 ax-12 2171 ax-ext 2708 ax-rep 5240 ax-sep 5254 ax-nul 5261 ax-pow 5318 ax-pr 5382 ax-un 7664 ax-inf2 9535 ax-cnex 11065 ax-resscn 11066 ax-1cn 11067 ax-icn 11068 ax-addcl 11069 ax-addrcl 11070 ax-mulcl 11071 ax-mulrcl 11072 ax-mulcom 11073 ax-addass 11074 ax-mulass 11075 ax-distr 11076 ax-i2m1 11077 ax-1ne0 11078 ax-1rid 11079 ax-rnegex 11080 ax-rrecex 11081 ax-cnre 11082 ax-pre-lttri 11083 ax-pre-lttrn 11084 ax-pre-ltadd 11085 ax-pre-mulgt0 11086 ax-pre-sup 11087 |
This theorem depends on definitions: df-bi 206 df-an 397 df-or 846 df-3or 1088 df-3an 1089 df-tru 1544 df-fal 1554 df-ex 1782 df-nf 1786 df-sb 2068 df-mo 2539 df-eu 2568 df-clab 2715 df-cleq 2729 df-clel 2815 df-nfc 2887 df-ne 2942 df-nel 3048 df-ral 3063 df-rex 3072 df-rmo 3351 df-reu 3352 df-rab 3406 df-v 3445 df-sbc 3738 df-csb 3854 df-dif 3911 df-un 3913 df-in 3915 df-ss 3925 df-pss 3927 df-nul 4281 df-if 4485 df-pw 4560 df-sn 4585 df-pr 4587 df-op 4591 df-uni 4864 df-int 4906 df-iun 4954 df-br 5104 df-opab 5166 df-mpt 5187 df-tr 5221 df-id 5529 df-eprel 5535 df-po 5543 df-so 5544 df-fr 5586 df-se 5587 df-we 5588 df-xp 5637 df-rel 5638 df-cnv 5639 df-co 5640 df-dm 5641 df-rn 5642 df-res 5643 df-ima 5644 df-pred 6251 df-ord 6318 df-on 6319 df-lim 6320 df-suc 6321 df-iota 6445 df-fun 6495 df-fn 6496 df-f 6497 df-f1 6498 df-fo 6499 df-f1o 6500 df-fv 6501 df-isom 6502 df-riota 7307 df-ov 7354 df-oprab 7355 df-mpo 7356 df-om 7795 df-1st 7913 df-2nd 7914 df-frecs 8204 df-wrecs 8235 df-recs 8309 df-rdg 8348 df-1o 8404 df-er 8606 df-pm 8726 df-en 8842 df-dom 8843 df-sdom 8844 df-fin 8845 df-sup 9336 df-inf 9337 df-oi 9404 df-card 9833 df-pnf 11149 df-mnf 11150 df-xr 11151 df-ltxr 11152 df-le 11153 df-sub 11345 df-neg 11346 df-div 11771 df-nn 12112 df-2 12174 df-3 12175 df-n0 12372 df-z 12458 df-uz 12722 df-rp 12870 df-fz 13379 df-fzo 13522 df-fl 13651 df-seq 13861 df-exp 13922 df-hash 14185 df-shft 14912 df-cj 14944 df-re 14945 df-im 14946 df-sqrt 15080 df-abs 15081 df-clim 15330 df-rlim 15331 df-sum 15531 |
This theorem is referenced by: (None) |
Copyright terms: Public domain | W3C validator |