MPE Home Metamath Proof Explorer < Previous   Next >
Nearby theorems
Mirrors  >  Home  >  MPE Home  >  Th. List  >  ruclem8 Structured version   Visualization version   GIF version

Theorem ruclem8 16285
Description: Lemma for ruc 16291. The intervals of the 𝐺 sequence are all nonempty. (Contributed by Mario Carneiro, 28-May-2014.)
Hypotheses
Ref Expression
ruc.1 (𝜑𝐹:ℕ⟶ℝ)
ruc.2 (𝜑𝐷 = (𝑥 ∈ (ℝ × ℝ), 𝑦 ∈ ℝ ↦ (((1st𝑥) + (2nd𝑥)) / 2) / 𝑚if(𝑚 < 𝑦, ⟨(1st𝑥), 𝑚⟩, ⟨((𝑚 + (2nd𝑥)) / 2), (2nd𝑥)⟩)))
ruc.4 𝐶 = ({⟨0, ⟨0, 1⟩⟩} ∪ 𝐹)
ruc.5 𝐺 = seq0(𝐷, 𝐶)
Assertion
Ref Expression
ruclem8 ((𝜑𝑁 ∈ ℕ0) → (1st ‘(𝐺𝑁)) < (2nd ‘(𝐺𝑁)))
Distinct variable groups:   𝑥,𝑚,𝑦,𝐹   𝑚,𝐺,𝑥,𝑦   𝑚,𝑁,𝑥,𝑦
Allowed substitution hints:   𝜑(𝑥,𝑦,𝑚)   𝐶(𝑥,𝑦,𝑚)   𝐷(𝑥,𝑦,𝑚)

Proof of Theorem ruclem8
Dummy variables 𝑛 𝑘 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 2fveq3 6925 . . . . 5 (𝑘 = 0 → (1st ‘(𝐺𝑘)) = (1st ‘(𝐺‘0)))
2 2fveq3 6925 . . . . 5 (𝑘 = 0 → (2nd ‘(𝐺𝑘)) = (2nd ‘(𝐺‘0)))
31, 2breq12d 5179 . . . 4 (𝑘 = 0 → ((1st ‘(𝐺𝑘)) < (2nd ‘(𝐺𝑘)) ↔ (1st ‘(𝐺‘0)) < (2nd ‘(𝐺‘0))))
43imbi2d 340 . . 3 (𝑘 = 0 → ((𝜑 → (1st ‘(𝐺𝑘)) < (2nd ‘(𝐺𝑘))) ↔ (𝜑 → (1st ‘(𝐺‘0)) < (2nd ‘(𝐺‘0)))))
5 2fveq3 6925 . . . . 5 (𝑘 = 𝑛 → (1st ‘(𝐺𝑘)) = (1st ‘(𝐺𝑛)))
6 2fveq3 6925 . . . . 5 (𝑘 = 𝑛 → (2nd ‘(𝐺𝑘)) = (2nd ‘(𝐺𝑛)))
75, 6breq12d 5179 . . . 4 (𝑘 = 𝑛 → ((1st ‘(𝐺𝑘)) < (2nd ‘(𝐺𝑘)) ↔ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛))))
87imbi2d 340 . . 3 (𝑘 = 𝑛 → ((𝜑 → (1st ‘(𝐺𝑘)) < (2nd ‘(𝐺𝑘))) ↔ (𝜑 → (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))))
9 2fveq3 6925 . . . . 5 (𝑘 = (𝑛 + 1) → (1st ‘(𝐺𝑘)) = (1st ‘(𝐺‘(𝑛 + 1))))
10 2fveq3 6925 . . . . 5 (𝑘 = (𝑛 + 1) → (2nd ‘(𝐺𝑘)) = (2nd ‘(𝐺‘(𝑛 + 1))))
119, 10breq12d 5179 . . . 4 (𝑘 = (𝑛 + 1) → ((1st ‘(𝐺𝑘)) < (2nd ‘(𝐺𝑘)) ↔ (1st ‘(𝐺‘(𝑛 + 1))) < (2nd ‘(𝐺‘(𝑛 + 1)))))
1211imbi2d 340 . . 3 (𝑘 = (𝑛 + 1) → ((𝜑 → (1st ‘(𝐺𝑘)) < (2nd ‘(𝐺𝑘))) ↔ (𝜑 → (1st ‘(𝐺‘(𝑛 + 1))) < (2nd ‘(𝐺‘(𝑛 + 1))))))
13 2fveq3 6925 . . . . 5 (𝑘 = 𝑁 → (1st ‘(𝐺𝑘)) = (1st ‘(𝐺𝑁)))
14 2fveq3 6925 . . . . 5 (𝑘 = 𝑁 → (2nd ‘(𝐺𝑘)) = (2nd ‘(𝐺𝑁)))
1513, 14breq12d 5179 . . . 4 (𝑘 = 𝑁 → ((1st ‘(𝐺𝑘)) < (2nd ‘(𝐺𝑘)) ↔ (1st ‘(𝐺𝑁)) < (2nd ‘(𝐺𝑁))))
1615imbi2d 340 . . 3 (𝑘 = 𝑁 → ((𝜑 → (1st ‘(𝐺𝑘)) < (2nd ‘(𝐺𝑘))) ↔ (𝜑 → (1st ‘(𝐺𝑁)) < (2nd ‘(𝐺𝑁)))))
17 0lt1 11812 . . . . 5 0 < 1
1817a1i 11 . . . 4 (𝜑 → 0 < 1)
19 ruc.1 . . . . . . 7 (𝜑𝐹:ℕ⟶ℝ)
20 ruc.2 . . . . . . 7 (𝜑𝐷 = (𝑥 ∈ (ℝ × ℝ), 𝑦 ∈ ℝ ↦ (((1st𝑥) + (2nd𝑥)) / 2) / 𝑚if(𝑚 < 𝑦, ⟨(1st𝑥), 𝑚⟩, ⟨((𝑚 + (2nd𝑥)) / 2), (2nd𝑥)⟩)))
21 ruc.4 . . . . . . 7 𝐶 = ({⟨0, ⟨0, 1⟩⟩} ∪ 𝐹)
22 ruc.5 . . . . . . 7 𝐺 = seq0(𝐷, 𝐶)
2319, 20, 21, 22ruclem4 16282 . . . . . 6 (𝜑 → (𝐺‘0) = ⟨0, 1⟩)
2423fveq2d 6924 . . . . 5 (𝜑 → (1st ‘(𝐺‘0)) = (1st ‘⟨0, 1⟩))
25 c0ex 11284 . . . . . 6 0 ∈ V
26 1ex 11286 . . . . . 6 1 ∈ V
2725, 26op1st 8038 . . . . 5 (1st ‘⟨0, 1⟩) = 0
2824, 27eqtrdi 2796 . . . 4 (𝜑 → (1st ‘(𝐺‘0)) = 0)
2923fveq2d 6924 . . . . 5 (𝜑 → (2nd ‘(𝐺‘0)) = (2nd ‘⟨0, 1⟩))
3025, 26op2nd 8039 . . . . 5 (2nd ‘⟨0, 1⟩) = 1
3129, 30eqtrdi 2796 . . . 4 (𝜑 → (2nd ‘(𝐺‘0)) = 1)
3218, 28, 313brtr4d 5198 . . 3 (𝜑 → (1st ‘(𝐺‘0)) < (2nd ‘(𝐺‘0)))
3319adantr 480 . . . . . . . . 9 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → 𝐹:ℕ⟶ℝ)
3420adantr 480 . . . . . . . . 9 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → 𝐷 = (𝑥 ∈ (ℝ × ℝ), 𝑦 ∈ ℝ ↦ (((1st𝑥) + (2nd𝑥)) / 2) / 𝑚if(𝑚 < 𝑦, ⟨(1st𝑥), 𝑚⟩, ⟨((𝑚 + (2nd𝑥)) / 2), (2nd𝑥)⟩)))
3519, 20, 21, 22ruclem6 16283 . . . . . . . . . . . 12 (𝜑𝐺:ℕ0⟶(ℝ × ℝ))
3635ffvelcdmda 7118 . . . . . . . . . . 11 ((𝜑𝑛 ∈ ℕ0) → (𝐺𝑛) ∈ (ℝ × ℝ))
3736adantrr 716 . . . . . . . . . 10 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (𝐺𝑛) ∈ (ℝ × ℝ))
38 xp1st 8062 . . . . . . . . . 10 ((𝐺𝑛) ∈ (ℝ × ℝ) → (1st ‘(𝐺𝑛)) ∈ ℝ)
3937, 38syl 17 . . . . . . . . 9 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (1st ‘(𝐺𝑛)) ∈ ℝ)
40 xp2nd 8063 . . . . . . . . . 10 ((𝐺𝑛) ∈ (ℝ × ℝ) → (2nd ‘(𝐺𝑛)) ∈ ℝ)
4137, 40syl 17 . . . . . . . . 9 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (2nd ‘(𝐺𝑛)) ∈ ℝ)
42 nn0p1nn 12592 . . . . . . . . . . 11 (𝑛 ∈ ℕ0 → (𝑛 + 1) ∈ ℕ)
43 ffvelcdm 7115 . . . . . . . . . . 11 ((𝐹:ℕ⟶ℝ ∧ (𝑛 + 1) ∈ ℕ) → (𝐹‘(𝑛 + 1)) ∈ ℝ)
4419, 42, 43syl2an 595 . . . . . . . . . 10 ((𝜑𝑛 ∈ ℕ0) → (𝐹‘(𝑛 + 1)) ∈ ℝ)
4544adantrr 716 . . . . . . . . 9 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (𝐹‘(𝑛 + 1)) ∈ ℝ)
46 eqid 2740 . . . . . . . . 9 (1st ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))) = (1st ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1))))
47 eqid 2740 . . . . . . . . 9 (2nd ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))) = (2nd ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1))))
48 simprr 772 . . . . . . . . 9 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))
4933, 34, 39, 41, 45, 46, 47, 48ruclem2 16280 . . . . . . . 8 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → ((1st ‘(𝐺𝑛)) ≤ (1st ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))) ∧ (1st ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))) < (2nd ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))) ∧ (2nd ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))) ≤ (2nd ‘(𝐺𝑛))))
5049simp2d 1143 . . . . . . 7 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (1st ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))) < (2nd ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))))
5119, 20, 21, 22ruclem7 16284 . . . . . . . . . 10 ((𝜑𝑛 ∈ ℕ0) → (𝐺‘(𝑛 + 1)) = ((𝐺𝑛)𝐷(𝐹‘(𝑛 + 1))))
5251adantrr 716 . . . . . . . . 9 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (𝐺‘(𝑛 + 1)) = ((𝐺𝑛)𝐷(𝐹‘(𝑛 + 1))))
53 1st2nd2 8069 . . . . . . . . . . 11 ((𝐺𝑛) ∈ (ℝ × ℝ) → (𝐺𝑛) = ⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩)
5437, 53syl 17 . . . . . . . . . 10 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (𝐺𝑛) = ⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩)
5554oveq1d 7463 . . . . . . . . 9 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → ((𝐺𝑛)𝐷(𝐹‘(𝑛 + 1))) = (⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1))))
5652, 55eqtrd 2780 . . . . . . . 8 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (𝐺‘(𝑛 + 1)) = (⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1))))
5756fveq2d 6924 . . . . . . 7 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (1st ‘(𝐺‘(𝑛 + 1))) = (1st ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))))
5856fveq2d 6924 . . . . . . 7 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (2nd ‘(𝐺‘(𝑛 + 1))) = (2nd ‘(⟨(1st ‘(𝐺𝑛)), (2nd ‘(𝐺𝑛))⟩𝐷(𝐹‘(𝑛 + 1)))))
5950, 57, 583brtr4d 5198 . . . . . 6 ((𝜑 ∧ (𝑛 ∈ ℕ0 ∧ (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)))) → (1st ‘(𝐺‘(𝑛 + 1))) < (2nd ‘(𝐺‘(𝑛 + 1))))
6059expr 456 . . . . 5 ((𝜑𝑛 ∈ ℕ0) → ((1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)) → (1st ‘(𝐺‘(𝑛 + 1))) < (2nd ‘(𝐺‘(𝑛 + 1)))))
6160expcom 413 . . . 4 (𝑛 ∈ ℕ0 → (𝜑 → ((1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛)) → (1st ‘(𝐺‘(𝑛 + 1))) < (2nd ‘(𝐺‘(𝑛 + 1))))))
6261a2d 29 . . 3 (𝑛 ∈ ℕ0 → ((𝜑 → (1st ‘(𝐺𝑛)) < (2nd ‘(𝐺𝑛))) → (𝜑 → (1st ‘(𝐺‘(𝑛 + 1))) < (2nd ‘(𝐺‘(𝑛 + 1))))))
634, 8, 12, 16, 32, 62nn0ind 12738 . 2 (𝑁 ∈ ℕ0 → (𝜑 → (1st ‘(𝐺𝑁)) < (2nd ‘(𝐺𝑁))))
6463impcom 407 1 ((𝜑𝑁 ∈ ℕ0) → (1st ‘(𝐺𝑁)) < (2nd ‘(𝐺𝑁)))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 395   = wceq 1537  wcel 2108  csb 3921  cun 3974  ifcif 4548  {csn 4648  cop 4654   class class class wbr 5166   × cxp 5698  wf 6569  cfv 6573  (class class class)co 7448  cmpo 7450  1st c1st 8028  2nd c2nd 8029  cr 11183  0cc0 11184  1c1 11185   + caddc 11187   < clt 11324  cle 11325   / cdiv 11947  cn 12293  2c2 12348  0cn0 12553  seqcseq 14052
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1793  ax-4 1807  ax-5 1909  ax-6 1967  ax-7 2007  ax-8 2110  ax-9 2118  ax-10 2141  ax-11 2158  ax-12 2178  ax-ext 2711  ax-sep 5317  ax-nul 5324  ax-pow 5383  ax-pr 5447  ax-un 7770  ax-cnex 11240  ax-resscn 11241  ax-1cn 11242  ax-icn 11243  ax-addcl 11244  ax-addrcl 11245  ax-mulcl 11246  ax-mulrcl 11247  ax-mulcom 11248  ax-addass 11249  ax-mulass 11250  ax-distr 11251  ax-i2m1 11252  ax-1ne0 11253  ax-1rid 11254  ax-rnegex 11255  ax-rrecex 11256  ax-cnre 11257  ax-pre-lttri 11258  ax-pre-lttrn 11259  ax-pre-ltadd 11260  ax-pre-mulgt0 11261
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 847  df-3or 1088  df-3an 1089  df-tru 1540  df-fal 1550  df-ex 1778  df-nf 1782  df-sb 2065  df-mo 2543  df-eu 2572  df-clab 2718  df-cleq 2732  df-clel 2819  df-nfc 2895  df-ne 2947  df-nel 3053  df-ral 3068  df-rex 3077  df-rmo 3388  df-reu 3389  df-rab 3444  df-v 3490  df-sbc 3805  df-csb 3922  df-dif 3979  df-un 3981  df-in 3983  df-ss 3993  df-pss 3996  df-nul 4353  df-if 4549  df-pw 4624  df-sn 4649  df-pr 4651  df-op 4655  df-uni 4932  df-iun 5017  df-br 5167  df-opab 5229  df-mpt 5250  df-tr 5284  df-id 5593  df-eprel 5599  df-po 5607  df-so 5608  df-fr 5652  df-we 5654  df-xp 5706  df-rel 5707  df-cnv 5708  df-co 5709  df-dm 5710  df-rn 5711  df-res 5712  df-ima 5713  df-pred 6332  df-ord 6398  df-on 6399  df-lim 6400  df-suc 6401  df-iota 6525  df-fun 6575  df-fn 6576  df-f 6577  df-f1 6578  df-fo 6579  df-f1o 6580  df-fv 6581  df-riota 7404  df-ov 7451  df-oprab 7452  df-mpo 7453  df-om 7904  df-1st 8030  df-2nd 8031  df-frecs 8322  df-wrecs 8353  df-recs 8427  df-rdg 8466  df-er 8763  df-en 9004  df-dom 9005  df-sdom 9006  df-pnf 11326  df-mnf 11327  df-xr 11328  df-ltxr 11329  df-le 11330  df-sub 11522  df-neg 11523  df-div 11948  df-nn 12294  df-2 12356  df-n0 12554  df-z 12640  df-uz 12904  df-fz 13568  df-seq 14053
This theorem is referenced by:  ruclem9  16286  ruclem10  16287  ruclem12  16289
  Copyright terms: Public domain W3C validator