| Metamath Proof Explorer |
< Previous
Next >
Nearby theorems |
||
| Mirrors > Home > MPE Home > Th. List > ruclem10 | Structured version Visualization version GIF version | ||
| Description: Lemma for ruc 16261. Every first component of the 𝐺 sequence is less than every second component. That is, the sequences form a chain a1 < a2 <... < b2 < b1, where ai are the first components and bi are the second components. (Contributed by Mario Carneiro, 28-May-2014.) |
| Ref | Expression |
|---|---|
| ruc.1 | ⊢ (𝜑 → 𝐹:ℕ⟶ℝ) |
| ruc.2 | ⊢ (𝜑 → 𝐷 = (𝑥 ∈ (ℝ × ℝ), 𝑦 ∈ ℝ ↦ ⦋(((1st ‘𝑥) + (2nd ‘𝑥)) / 2) / 𝑚⦌if(𝑚 < 𝑦, 〈(1st ‘𝑥), 𝑚〉, 〈((𝑚 + (2nd ‘𝑥)) / 2), (2nd ‘𝑥)〉))) |
| ruc.4 | ⊢ 𝐶 = ({〈0, 〈0, 1〉〉} ∪ 𝐹) |
| ruc.5 | ⊢ 𝐺 = seq0(𝐷, 𝐶) |
| ruclem10.6 | ⊢ (𝜑 → 𝑀 ∈ ℕ0) |
| ruclem10.7 | ⊢ (𝜑 → 𝑁 ∈ ℕ0) |
| Ref | Expression |
|---|---|
| ruclem10 | ⊢ (𝜑 → (1st ‘(𝐺‘𝑀)) < (2nd ‘(𝐺‘𝑁))) |
| Step | Hyp | Ref | Expression |
|---|---|---|---|
| 1 | ruc.1 | . . . . 5 ⊢ (𝜑 → 𝐹:ℕ⟶ℝ) | |
| 2 | ruc.2 | . . . . 5 ⊢ (𝜑 → 𝐷 = (𝑥 ∈ (ℝ × ℝ), 𝑦 ∈ ℝ ↦ ⦋(((1st ‘𝑥) + (2nd ‘𝑥)) / 2) / 𝑚⦌if(𝑚 < 𝑦, 〈(1st ‘𝑥), 𝑚〉, 〈((𝑚 + (2nd ‘𝑥)) / 2), (2nd ‘𝑥)〉))) | |
| 3 | ruc.4 | . . . . 5 ⊢ 𝐶 = ({〈0, 〈0, 1〉〉} ∪ 𝐹) | |
| 4 | ruc.5 | . . . . 5 ⊢ 𝐺 = seq0(𝐷, 𝐶) | |
| 5 | 1, 2, 3, 4 | ruclem6 16253 | . . . 4 ⊢ (𝜑 → 𝐺:ℕ0⟶(ℝ × ℝ)) |
| 6 | ruclem10.6 | . . . 4 ⊢ (𝜑 → 𝑀 ∈ ℕ0) | |
| 7 | 5, 6 | ffvelcdmd 7085 | . . 3 ⊢ (𝜑 → (𝐺‘𝑀) ∈ (ℝ × ℝ)) |
| 8 | xp1st 8028 | . . 3 ⊢ ((𝐺‘𝑀) ∈ (ℝ × ℝ) → (1st ‘(𝐺‘𝑀)) ∈ ℝ) | |
| 9 | 7, 8 | syl 17 | . 2 ⊢ (𝜑 → (1st ‘(𝐺‘𝑀)) ∈ ℝ) |
| 10 | ruclem10.7 | . . . . 5 ⊢ (𝜑 → 𝑁 ∈ ℕ0) | |
| 11 | 10, 6 | ifcld 4552 | . . . 4 ⊢ (𝜑 → if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ ℕ0) |
| 12 | 5, 11 | ffvelcdmd 7085 | . . 3 ⊢ (𝜑 → (𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀)) ∈ (ℝ × ℝ)) |
| 13 | xp1st 8028 | . . 3 ⊢ ((𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀)) ∈ (ℝ × ℝ) → (1st ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ∈ ℝ) | |
| 14 | 12, 13 | syl 17 | . 2 ⊢ (𝜑 → (1st ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ∈ ℝ) |
| 15 | 5, 10 | ffvelcdmd 7085 | . . 3 ⊢ (𝜑 → (𝐺‘𝑁) ∈ (ℝ × ℝ)) |
| 16 | xp2nd 8029 | . . 3 ⊢ ((𝐺‘𝑁) ∈ (ℝ × ℝ) → (2nd ‘(𝐺‘𝑁)) ∈ ℝ) | |
| 17 | 15, 16 | syl 17 | . 2 ⊢ (𝜑 → (2nd ‘(𝐺‘𝑁)) ∈ ℝ) |
| 18 | 6 | nn0red 12571 | . . . . . 6 ⊢ (𝜑 → 𝑀 ∈ ℝ) |
| 19 | 10 | nn0red 12571 | . . . . . 6 ⊢ (𝜑 → 𝑁 ∈ ℝ) |
| 20 | max1 13209 | . . . . . 6 ⊢ ((𝑀 ∈ ℝ ∧ 𝑁 ∈ ℝ) → 𝑀 ≤ if(𝑀 ≤ 𝑁, 𝑁, 𝑀)) | |
| 21 | 18, 19, 20 | syl2anc 584 | . . . . 5 ⊢ (𝜑 → 𝑀 ≤ if(𝑀 ≤ 𝑁, 𝑁, 𝑀)) |
| 22 | 6 | nn0zd 12622 | . . . . . 6 ⊢ (𝜑 → 𝑀 ∈ ℤ) |
| 23 | 11 | nn0zd 12622 | . . . . . 6 ⊢ (𝜑 → if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ ℤ) |
| 24 | eluz 12874 | . . . . . 6 ⊢ ((𝑀 ∈ ℤ ∧ if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ ℤ) → (if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ (ℤ≥‘𝑀) ↔ 𝑀 ≤ if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) | |
| 25 | 22, 23, 24 | syl2anc 584 | . . . . 5 ⊢ (𝜑 → (if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ (ℤ≥‘𝑀) ↔ 𝑀 ≤ if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) |
| 26 | 21, 25 | mpbird 257 | . . . 4 ⊢ (𝜑 → if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ (ℤ≥‘𝑀)) |
| 27 | 1, 2, 3, 4, 6, 26 | ruclem9 16256 | . . 3 ⊢ (𝜑 → ((1st ‘(𝐺‘𝑀)) ≤ (1st ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ∧ (2nd ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ≤ (2nd ‘(𝐺‘𝑀)))) |
| 28 | 27 | simpld 494 | . 2 ⊢ (𝜑 → (1st ‘(𝐺‘𝑀)) ≤ (1st ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀)))) |
| 29 | xp2nd 8029 | . . . 4 ⊢ ((𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀)) ∈ (ℝ × ℝ) → (2nd ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ∈ ℝ) | |
| 30 | 12, 29 | syl 17 | . . 3 ⊢ (𝜑 → (2nd ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ∈ ℝ) |
| 31 | 1, 2, 3, 4 | ruclem8 16255 | . . . 4 ⊢ ((𝜑 ∧ if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ ℕ0) → (1st ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) < (2nd ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀)))) |
| 32 | 11, 31 | mpdan 687 | . . 3 ⊢ (𝜑 → (1st ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) < (2nd ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀)))) |
| 33 | max2 13211 | . . . . . . 7 ⊢ ((𝑀 ∈ ℝ ∧ 𝑁 ∈ ℝ) → 𝑁 ≤ if(𝑀 ≤ 𝑁, 𝑁, 𝑀)) | |
| 34 | 18, 19, 33 | syl2anc 584 | . . . . . 6 ⊢ (𝜑 → 𝑁 ≤ if(𝑀 ≤ 𝑁, 𝑁, 𝑀)) |
| 35 | 10 | nn0zd 12622 | . . . . . . 7 ⊢ (𝜑 → 𝑁 ∈ ℤ) |
| 36 | eluz 12874 | . . . . . . 7 ⊢ ((𝑁 ∈ ℤ ∧ if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ ℤ) → (if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ (ℤ≥‘𝑁) ↔ 𝑁 ≤ if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) | |
| 37 | 35, 23, 36 | syl2anc 584 | . . . . . 6 ⊢ (𝜑 → (if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ (ℤ≥‘𝑁) ↔ 𝑁 ≤ if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) |
| 38 | 34, 37 | mpbird 257 | . . . . 5 ⊢ (𝜑 → if(𝑀 ≤ 𝑁, 𝑁, 𝑀) ∈ (ℤ≥‘𝑁)) |
| 39 | 1, 2, 3, 4, 10, 38 | ruclem9 16256 | . . . 4 ⊢ (𝜑 → ((1st ‘(𝐺‘𝑁)) ≤ (1st ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ∧ (2nd ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ≤ (2nd ‘(𝐺‘𝑁)))) |
| 40 | 39 | simprd 495 | . . 3 ⊢ (𝜑 → (2nd ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) ≤ (2nd ‘(𝐺‘𝑁))) |
| 41 | 14, 30, 17, 32, 40 | ltletrd 11403 | . 2 ⊢ (𝜑 → (1st ‘(𝐺‘if(𝑀 ≤ 𝑁, 𝑁, 𝑀))) < (2nd ‘(𝐺‘𝑁))) |
| 42 | 9, 14, 17, 28, 41 | lelttrd 11401 | 1 ⊢ (𝜑 → (1st ‘(𝐺‘𝑀)) < (2nd ‘(𝐺‘𝑁))) |
| Colors of variables: wff setvar class |
| Syntax hints: → wi 4 ↔ wb 206 = wceq 1539 ∈ wcel 2107 ⦋csb 3879 ∪ cun 3929 ifcif 4505 {csn 4606 〈cop 4612 class class class wbr 5123 × cxp 5663 ⟶wf 6537 ‘cfv 6541 (class class class)co 7413 ∈ cmpo 7415 1st c1st 7994 2nd c2nd 7995 ℝcr 11136 0cc0 11137 1c1 11138 + caddc 11140 < clt 11277 ≤ cle 11278 / cdiv 11902 ℕcn 12248 2c2 12303 ℕ0cn0 12509 ℤcz 12596 ℤ≥cuz 12860 seqcseq 14024 |
| This theorem was proved from axioms: ax-mp 5 ax-1 6 ax-2 7 ax-3 8 ax-gen 1794 ax-4 1808 ax-5 1909 ax-6 1966 ax-7 2006 ax-8 2109 ax-9 2117 ax-10 2140 ax-11 2156 ax-12 2176 ax-ext 2706 ax-sep 5276 ax-nul 5286 ax-pow 5345 ax-pr 5412 ax-un 7737 ax-cnex 11193 ax-resscn 11194 ax-1cn 11195 ax-icn 11196 ax-addcl 11197 ax-addrcl 11198 ax-mulcl 11199 ax-mulrcl 11200 ax-mulcom 11201 ax-addass 11202 ax-mulass 11203 ax-distr 11204 ax-i2m1 11205 ax-1ne0 11206 ax-1rid 11207 ax-rnegex 11208 ax-rrecex 11209 ax-cnre 11210 ax-pre-lttri 11211 ax-pre-lttrn 11212 ax-pre-ltadd 11213 ax-pre-mulgt0 11214 |
| This theorem depends on definitions: df-bi 207 df-an 396 df-or 848 df-3or 1087 df-3an 1088 df-tru 1542 df-fal 1552 df-ex 1779 df-nf 1783 df-sb 2064 df-mo 2538 df-eu 2567 df-clab 2713 df-cleq 2726 df-clel 2808 df-nfc 2884 df-ne 2932 df-nel 3036 df-ral 3051 df-rex 3060 df-rmo 3363 df-reu 3364 df-rab 3420 df-v 3465 df-sbc 3771 df-csb 3880 df-dif 3934 df-un 3936 df-in 3938 df-ss 3948 df-pss 3951 df-nul 4314 df-if 4506 df-pw 4582 df-sn 4607 df-pr 4609 df-op 4613 df-uni 4888 df-iun 4973 df-br 5124 df-opab 5186 df-mpt 5206 df-tr 5240 df-id 5558 df-eprel 5564 df-po 5572 df-so 5573 df-fr 5617 df-we 5619 df-xp 5671 df-rel 5672 df-cnv 5673 df-co 5674 df-dm 5675 df-rn 5676 df-res 5677 df-ima 5678 df-pred 6301 df-ord 6366 df-on 6367 df-lim 6368 df-suc 6369 df-iota 6494 df-fun 6543 df-fn 6544 df-f 6545 df-f1 6546 df-fo 6547 df-f1o 6548 df-fv 6549 df-riota 7370 df-ov 7416 df-oprab 7417 df-mpo 7418 df-om 7870 df-1st 7996 df-2nd 7997 df-frecs 8288 df-wrecs 8319 df-recs 8393 df-rdg 8432 df-er 8727 df-en 8968 df-dom 8969 df-sdom 8970 df-pnf 11279 df-mnf 11280 df-xr 11281 df-ltxr 11282 df-le 11283 df-sub 11476 df-neg 11477 df-div 11903 df-nn 12249 df-2 12311 df-n0 12510 df-z 12597 df-uz 12861 df-fz 13530 df-seq 14025 |
| This theorem is referenced by: ruclem11 16258 ruclem12 16259 |
| Copyright terms: Public domain | W3C validator |