Metamath Proof Explorer |
< Previous
Next >
Nearby theorems |
||
Mirrors > Home > MPE Home > Th. List > seqcl | Structured version Visualization version GIF version |
Description: Closure properties of the recursive sequence builder. (Contributed by Mario Carneiro, 2-Jul-2013.) (Revised by Mario Carneiro, 27-May-2014.) |
Ref | Expression |
---|---|
seqcl.1 | ⊢ (𝜑 → 𝑁 ∈ (ℤ≥‘𝑀)) |
seqcl.2 | ⊢ ((𝜑 ∧ 𝑥 ∈ (𝑀...𝑁)) → (𝐹‘𝑥) ∈ 𝑆) |
seqcl.3 | ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 + 𝑦) ∈ 𝑆) |
Ref | Expression |
---|---|
seqcl | ⊢ (𝜑 → (seq𝑀( + , 𝐹)‘𝑁) ∈ 𝑆) |
Step | Hyp | Ref | Expression |
---|---|---|---|
1 | fveq2 6819 | . . . 4 ⊢ (𝑥 = 𝑀 → (𝐹‘𝑥) = (𝐹‘𝑀)) | |
2 | 1 | eleq1d 2821 | . . 3 ⊢ (𝑥 = 𝑀 → ((𝐹‘𝑥) ∈ 𝑆 ↔ (𝐹‘𝑀) ∈ 𝑆)) |
3 | seqcl.2 | . . . 4 ⊢ ((𝜑 ∧ 𝑥 ∈ (𝑀...𝑁)) → (𝐹‘𝑥) ∈ 𝑆) | |
4 | 3 | ralrimiva 3139 | . . 3 ⊢ (𝜑 → ∀𝑥 ∈ (𝑀...𝑁)(𝐹‘𝑥) ∈ 𝑆) |
5 | seqcl.1 | . . . 4 ⊢ (𝜑 → 𝑁 ∈ (ℤ≥‘𝑀)) | |
6 | eluzfz1 13356 | . . . 4 ⊢ (𝑁 ∈ (ℤ≥‘𝑀) → 𝑀 ∈ (𝑀...𝑁)) | |
7 | 5, 6 | syl 17 | . . 3 ⊢ (𝜑 → 𝑀 ∈ (𝑀...𝑁)) |
8 | 2, 4, 7 | rspcdva 3571 | . 2 ⊢ (𝜑 → (𝐹‘𝑀) ∈ 𝑆) |
9 | seqcl.3 | . 2 ⊢ ((𝜑 ∧ (𝑥 ∈ 𝑆 ∧ 𝑦 ∈ 𝑆)) → (𝑥 + 𝑦) ∈ 𝑆) | |
10 | eluzel2 12680 | . . . . . 6 ⊢ (𝑁 ∈ (ℤ≥‘𝑀) → 𝑀 ∈ ℤ) | |
11 | 5, 10 | syl 17 | . . . . 5 ⊢ (𝜑 → 𝑀 ∈ ℤ) |
12 | fzp1ss 13400 | . . . . 5 ⊢ (𝑀 ∈ ℤ → ((𝑀 + 1)...𝑁) ⊆ (𝑀...𝑁)) | |
13 | 11, 12 | syl 17 | . . . 4 ⊢ (𝜑 → ((𝑀 + 1)...𝑁) ⊆ (𝑀...𝑁)) |
14 | 13 | sselda 3931 | . . 3 ⊢ ((𝜑 ∧ 𝑥 ∈ ((𝑀 + 1)...𝑁)) → 𝑥 ∈ (𝑀...𝑁)) |
15 | 14, 3 | syldan 591 | . 2 ⊢ ((𝜑 ∧ 𝑥 ∈ ((𝑀 + 1)...𝑁)) → (𝐹‘𝑥) ∈ 𝑆) |
16 | 8, 9, 5, 15 | seqcl2 13834 | 1 ⊢ (𝜑 → (seq𝑀( + , 𝐹)‘𝑁) ∈ 𝑆) |
Colors of variables: wff setvar class |
Syntax hints: → wi 4 ∧ wa 396 = wceq 1540 ∈ wcel 2105 ⊆ wss 3897 ‘cfv 6473 (class class class)co 7329 1c1 10965 + caddc 10967 ℤcz 12412 ℤ≥cuz 12675 ...cfz 13332 seqcseq 13814 |
This theorem was proved from axioms: ax-mp 5 ax-1 6 ax-2 7 ax-3 8 ax-gen 1796 ax-4 1810 ax-5 1912 ax-6 1970 ax-7 2010 ax-8 2107 ax-9 2115 ax-10 2136 ax-11 2153 ax-12 2170 ax-ext 2707 ax-sep 5240 ax-nul 5247 ax-pow 5305 ax-pr 5369 ax-un 7642 ax-cnex 11020 ax-resscn 11021 ax-1cn 11022 ax-icn 11023 ax-addcl 11024 ax-addrcl 11025 ax-mulcl 11026 ax-mulrcl 11027 ax-mulcom 11028 ax-addass 11029 ax-mulass 11030 ax-distr 11031 ax-i2m1 11032 ax-1ne0 11033 ax-1rid 11034 ax-rnegex 11035 ax-rrecex 11036 ax-cnre 11037 ax-pre-lttri 11038 ax-pre-lttrn 11039 ax-pre-ltadd 11040 ax-pre-mulgt0 11041 |
This theorem depends on definitions: df-bi 206 df-an 397 df-or 845 df-3or 1087 df-3an 1088 df-tru 1543 df-fal 1553 df-ex 1781 df-nf 1785 df-sb 2067 df-mo 2538 df-eu 2567 df-clab 2714 df-cleq 2728 df-clel 2814 df-nfc 2886 df-ne 2941 df-nel 3047 df-ral 3062 df-rex 3071 df-reu 3350 df-rab 3404 df-v 3443 df-sbc 3727 df-csb 3843 df-dif 3900 df-un 3902 df-in 3904 df-ss 3914 df-pss 3916 df-nul 4269 df-if 4473 df-pw 4548 df-sn 4573 df-pr 4575 df-op 4579 df-uni 4852 df-iun 4940 df-br 5090 df-opab 5152 df-mpt 5173 df-tr 5207 df-id 5512 df-eprel 5518 df-po 5526 df-so 5527 df-fr 5569 df-we 5571 df-xp 5620 df-rel 5621 df-cnv 5622 df-co 5623 df-dm 5624 df-rn 5625 df-res 5626 df-ima 5627 df-pred 6232 df-ord 6299 df-on 6300 df-lim 6301 df-suc 6302 df-iota 6425 df-fun 6475 df-fn 6476 df-f 6477 df-f1 6478 df-fo 6479 df-f1o 6480 df-fv 6481 df-riota 7286 df-ov 7332 df-oprab 7333 df-mpo 7334 df-om 7773 df-1st 7891 df-2nd 7892 df-frecs 8159 df-wrecs 8190 df-recs 8264 df-rdg 8303 df-er 8561 df-en 8797 df-dom 8798 df-sdom 8799 df-pnf 11104 df-mnf 11105 df-xr 11106 df-ltxr 11107 df-le 11108 df-sub 11300 df-neg 11301 df-nn 12067 df-n0 12327 df-z 12413 df-uz 12676 df-fz 13333 df-seq 13815 |
This theorem is referenced by: sermono 13848 seqsplit 13849 seqcaopr2 13852 seqf1olem2a 13854 seqf1olem2 13856 seqid3 13860 seqhomo 13863 seqz 13864 seqdistr 13867 serge0 13870 serle 13871 seqof 13873 seqcoll 14270 seqcoll2 14271 fsumcl2lem 15534 prodfn0 15697 prodfrec 15698 prodfdiv 15699 fprodcl2lem 15751 eulerthlem2 16572 gsumwsubmcl 18564 mulgnnsubcl 18804 gsumzcl2 19598 gsumzaddlem 19609 gsummptfzcl 19657 lgscllem 26550 lgsval4a 26565 lgsneg 26567 lgsdir 26578 lgsdilem2 26579 lgsdi 26580 lgsne0 26581 gsumncl 32760 faclim 33946 knoppcnlem8 34771 mblfinlem2 35913 fmul01 43446 fmulcl 43447 fmuldfeq 43449 fmul01lt1lem1 43450 fmul01lt1lem2 43451 stoweidlem3 43869 stoweidlem42 43908 stoweidlem48 43914 wallispilem4 43934 wallispi 43936 wallispi2lem1 43937 wallispi2 43939 stirlinglem5 43944 stirlinglem7 43946 stirlinglem10 43949 sge0isum 44291 |
Copyright terms: Public domain | W3C validator |