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

Theorem ltoddhalfle 15998
Description: An integer is less than half of an odd number iff it is less than or equal to the half of the predecessor of the odd number (which is an even number). (Contributed by AV, 29-Jun-2021.)
Assertion
Ref Expression
ltoddhalfle ((𝑁 ∈ ℤ ∧ ¬ 2 ∥ 𝑁𝑀 ∈ ℤ) → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))

Proof of Theorem ltoddhalfle
Dummy variable 𝑛 is distinct from all other variables.
StepHypRef Expression
1 odd2np1 15978 . . 3 (𝑁 ∈ ℤ → (¬ 2 ∥ 𝑁 ↔ ∃𝑛 ∈ ℤ ((2 · 𝑛) + 1) = 𝑁))
2 halfre 12117 . . . . . . . . . . . . . . . 16 (1 / 2) ∈ ℝ
32a1i 11 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (1 / 2) ∈ ℝ)
4 1red 10907 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → 1 ∈ ℝ)
5 zre 12253 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → 𝑛 ∈ ℝ)
63, 4, 53jca 1126 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → ((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ))
76adantr 480 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ))
8 halflt1 12121 . . . . . . . . . . . . 13 (1 / 2) < 1
9 axltadd 10979 . . . . . . . . . . . . 13 (((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ) → ((1 / 2) < 1 → (𝑛 + (1 / 2)) < (𝑛 + 1)))
107, 8, 9mpisyl 21 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + (1 / 2)) < (𝑛 + 1))
11 zre 12253 . . . . . . . . . . . . . 14 (𝑀 ∈ ℤ → 𝑀 ∈ ℝ)
1211adantl 481 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑀 ∈ ℝ)
135, 3readdcld 10935 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (𝑛 + (1 / 2)) ∈ ℝ)
1413adantr 480 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + (1 / 2)) ∈ ℝ)
15 peano2z 12291 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (𝑛 + 1) ∈ ℤ)
1615zred 12355 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (𝑛 + 1) ∈ ℝ)
1716adantr 480 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + 1) ∈ ℝ)
18 lttr 10982 . . . . . . . . . . . . 13 ((𝑀 ∈ ℝ ∧ (𝑛 + (1 / 2)) ∈ ℝ ∧ (𝑛 + 1) ∈ ℝ) → ((𝑀 < (𝑛 + (1 / 2)) ∧ (𝑛 + (1 / 2)) < (𝑛 + 1)) → 𝑀 < (𝑛 + 1)))
1912, 14, 17, 18syl3anc 1369 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((𝑀 < (𝑛 + (1 / 2)) ∧ (𝑛 + (1 / 2)) < (𝑛 + 1)) → 𝑀 < (𝑛 + 1)))
2010, 19mpan2d 690 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) → 𝑀 < (𝑛 + 1)))
21 zleltp1 12301 . . . . . . . . . . . 12 ((𝑀 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + 1)))
2221ancoms 458 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + 1)))
2320, 22sylibrd 258 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) → 𝑀𝑛))
24 halfgt0 12119 . . . . . . . . . . . 12 0 < (1 / 2)
253, 5jca 511 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → ((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ))
2625adantr 480 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ))
27 ltaddpos 11395 . . . . . . . . . . . . 13 (((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ) → (0 < (1 / 2) ↔ 𝑛 < (𝑛 + (1 / 2))))
2826, 27syl 17 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (0 < (1 / 2) ↔ 𝑛 < (𝑛 + (1 / 2))))
2924, 28mpbii 232 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑛 < (𝑛 + (1 / 2)))
305adantr 480 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑛 ∈ ℝ)
31 lelttr 10996 . . . . . . . . . . . 12 ((𝑀 ∈ ℝ ∧ 𝑛 ∈ ℝ ∧ (𝑛 + (1 / 2)) ∈ ℝ) → ((𝑀𝑛𝑛 < (𝑛 + (1 / 2))) → 𝑀 < (𝑛 + (1 / 2))))
3212, 30, 14, 31syl3anc 1369 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((𝑀𝑛𝑛 < (𝑛 + (1 / 2))) → 𝑀 < (𝑛 + (1 / 2))))
3329, 32mpan2d 690 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + (1 / 2))))
3423, 33impbid 211 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) ↔ 𝑀𝑛))
35 zcn 12254 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → 𝑛 ∈ ℂ)
36 1cnd 10901 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → 1 ∈ ℂ)
37 2cnne0 12113 . . . . . . . . . . . . 13 (2 ∈ ℂ ∧ 2 ≠ 0)
3837a1i 11 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → (2 ∈ ℂ ∧ 2 ≠ 0))
39 muldivdir 11598 . . . . . . . . . . . 12 ((𝑛 ∈ ℂ ∧ 1 ∈ ℂ ∧ (2 ∈ ℂ ∧ 2 ≠ 0)) → (((2 · 𝑛) + 1) / 2) = (𝑛 + (1 / 2)))
4035, 36, 38, 39syl3anc 1369 . . . . . . . . . . 11 (𝑛 ∈ ℤ → (((2 · 𝑛) + 1) / 2) = (𝑛 + (1 / 2)))
4140breq2d 5082 . . . . . . . . . 10 (𝑛 ∈ ℤ → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑛 + (1 / 2))))
4241adantr 480 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑛 + (1 / 2))))
43 2z 12282 . . . . . . . . . . . . . . . . 17 2 ∈ ℤ
4443a1i 11 . . . . . . . . . . . . . . . 16 (𝑛 ∈ ℤ → 2 ∈ ℤ)
45 id 22 . . . . . . . . . . . . . . . 16 (𝑛 ∈ ℤ → 𝑛 ∈ ℤ)
4644, 45zmulcld 12361 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (2 · 𝑛) ∈ ℤ)
4746zcnd 12356 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (2 · 𝑛) ∈ ℂ)
4847adantr 480 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (2 · 𝑛) ∈ ℂ)
49 pncan1 11329 . . . . . . . . . . . . 13 ((2 · 𝑛) ∈ ℂ → (((2 · 𝑛) + 1) − 1) = (2 · 𝑛))
5048, 49syl 17 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (((2 · 𝑛) + 1) − 1) = (2 · 𝑛))
5150oveq1d 7270 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((((2 · 𝑛) + 1) − 1) / 2) = ((2 · 𝑛) / 2))
52 2cnd 11981 . . . . . . . . . . . . 13 (𝑛 ∈ ℤ → 2 ∈ ℂ)
53 2ne0 12007 . . . . . . . . . . . . . 14 2 ≠ 0
5453a1i 11 . . . . . . . . . . . . 13 (𝑛 ∈ ℤ → 2 ≠ 0)
5535, 52, 54divcan3d 11686 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → ((2 · 𝑛) / 2) = 𝑛)
5655adantr 480 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((2 · 𝑛) / 2) = 𝑛)
5751, 56eqtrd 2778 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((((2 · 𝑛) + 1) − 1) / 2) = 𝑛)
5857breq2d 5082 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2) ↔ 𝑀𝑛))
5934, 42, 583bitr4d 310 . . . . . . . 8 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2)))
60 oveq1 7262 . . . . . . . . . 10 (((2 · 𝑛) + 1) = 𝑁 → (((2 · 𝑛) + 1) / 2) = (𝑁 / 2))
6160breq2d 5082 . . . . . . . . 9 (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑁 / 2)))
62 oveq1 7262 . . . . . . . . . . 11 (((2 · 𝑛) + 1) = 𝑁 → (((2 · 𝑛) + 1) − 1) = (𝑁 − 1))
6362oveq1d 7270 . . . . . . . . . 10 (((2 · 𝑛) + 1) = 𝑁 → ((((2 · 𝑛) + 1) − 1) / 2) = ((𝑁 − 1) / 2))
6463breq2d 5082 . . . . . . . . 9 (((2 · 𝑛) + 1) = 𝑁 → (𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))
6561, 64bibi12d 345 . . . . . . . 8 (((2 · 𝑛) + 1) = 𝑁 → ((𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2)) ↔ (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2))))
6659, 65syl5ibcom 244 . . . . . . 7 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2))))
6766ex 412 . . . . . 6 (𝑛 ∈ ℤ → (𝑀 ∈ ℤ → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
6867adantl 481 . . . . 5 ((𝑁 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (𝑀 ∈ ℤ → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
6968com23 86 . . . 4 ((𝑁 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
7069rexlimdva 3212 . . 3 (𝑁 ∈ ℤ → (∃𝑛 ∈ ℤ ((2 · 𝑛) + 1) = 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
711, 70sylbid 239 . 2 (𝑁 ∈ ℤ → (¬ 2 ∥ 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
72713imp 1109 1 ((𝑁 ∈ ℤ ∧ ¬ 2 ∥ 𝑁𝑀 ∈ ℤ) → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))
Colors of variables: wff setvar class
Syntax hints:  ¬ wn 3  wi 4  wb 205  wa 395  w3a 1085   = wceq 1539  wcel 2108  wne 2942  wrex 3064   class class class wbr 5070  (class class class)co 7255  cc 10800  cr 10801  0cc0 10802  1c1 10803   + caddc 10805   · cmul 10807   < clt 10940  cle 10941  cmin 11135   / cdiv 11562  2c2 11958  cz 12249  cdvds 15891
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1799  ax-4 1813  ax-5 1914  ax-6 1972  ax-7 2012  ax-8 2110  ax-9 2118  ax-10 2139  ax-11 2156  ax-12 2173  ax-ext 2709  ax-sep 5218  ax-nul 5225  ax-pow 5283  ax-pr 5347  ax-un 7566  ax-resscn 10859  ax-1cn 10860  ax-icn 10861  ax-addcl 10862  ax-addrcl 10863  ax-mulcl 10864  ax-mulrcl 10865  ax-mulcom 10866  ax-addass 10867  ax-mulass 10868  ax-distr 10869  ax-i2m1 10870  ax-1ne0 10871  ax-1rid 10872  ax-rnegex 10873  ax-rrecex 10874  ax-cnre 10875  ax-pre-lttri 10876  ax-pre-lttrn 10877  ax-pre-ltadd 10878  ax-pre-mulgt0 10879
This theorem depends on definitions:  df-bi 206  df-an 396  df-or 844  df-3or 1086  df-3an 1087  df-tru 1542  df-fal 1552  df-ex 1784  df-nf 1788  df-sb 2069  df-mo 2540  df-eu 2569  df-clab 2716  df-cleq 2730  df-clel 2817  df-nfc 2888  df-ne 2943  df-nel 3049  df-ral 3068  df-rex 3069  df-reu 3070  df-rmo 3071  df-rab 3072  df-v 3424  df-sbc 3712  df-csb 3829  df-dif 3886  df-un 3888  df-in 3890  df-ss 3900  df-pss 3902  df-nul 4254  df-if 4457  df-pw 4532  df-sn 4559  df-pr 4561  df-tp 4563  df-op 4565  df-uni 4837  df-iun 4923  df-br 5071  df-opab 5133  df-mpt 5154  df-tr 5188  df-id 5480  df-eprel 5486  df-po 5494  df-so 5495  df-fr 5535  df-we 5537  df-xp 5586  df-rel 5587  df-cnv 5588  df-co 5589  df-dm 5590  df-rn 5591  df-res 5592  df-ima 5593  df-pred 6191  df-ord 6254  df-on 6255  df-lim 6256  df-suc 6257  df-iota 6376  df-fun 6420  df-fn 6421  df-f 6422  df-f1 6423  df-fo 6424  df-f1o 6425  df-fv 6426  df-riota 7212  df-ov 7258  df-oprab 7259  df-mpo 7260  df-om 7688  df-2nd 7805  df-frecs 8068  df-wrecs 8099  df-recs 8173  df-rdg 8212  df-er 8456  df-en 8692  df-dom 8693  df-sdom 8694  df-pnf 10942  df-mnf 10943  df-xr 10944  df-ltxr 10945  df-le 10946  df-sub 11137  df-neg 11138  df-div 11563  df-nn 11904  df-2 11966  df-n0 12164  df-z 12250  df-dvds 15892
This theorem is referenced by:  gausslemma2dlem1a  26418
  Copyright terms: Public domain W3C validator