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

Theorem ltoddhalfle 15702
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 15682 . . 3 (𝑁 ∈ ℤ → (¬ 2 ∥ 𝑁 ↔ ∃𝑛 ∈ ℤ ((2 · 𝑛) + 1) = 𝑁))
2 halfre 11839 . . . . . . . . . . . . . . . 16 (1 / 2) ∈ ℝ
32a1i 11 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (1 / 2) ∈ ℝ)
4 1red 10631 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → 1 ∈ ℝ)
5 zre 11973 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → 𝑛 ∈ ℝ)
63, 4, 53jca 1125 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → ((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ))
76adantr 484 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ))
8 halflt1 11843 . . . . . . . . . . . . 13 (1 / 2) < 1
9 axltadd 10703 . . . . . . . . . . . . 13 (((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ) → ((1 / 2) < 1 → (𝑛 + (1 / 2)) < (𝑛 + 1)))
107, 8, 9mpisyl 21 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + (1 / 2)) < (𝑛 + 1))
11 zre 11973 . . . . . . . . . . . . . 14 (𝑀 ∈ ℤ → 𝑀 ∈ ℝ)
1211adantl 485 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑀 ∈ ℝ)
135, 3readdcld 10659 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (𝑛 + (1 / 2)) ∈ ℝ)
1413adantr 484 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + (1 / 2)) ∈ ℝ)
15 peano2z 12011 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (𝑛 + 1) ∈ ℤ)
1615zred 12075 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (𝑛 + 1) ∈ ℝ)
1716adantr 484 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + 1) ∈ ℝ)
18 lttr 10706 . . . . . . . . . . . . 13 ((𝑀 ∈ ℝ ∧ (𝑛 + (1 / 2)) ∈ ℝ ∧ (𝑛 + 1) ∈ ℝ) → ((𝑀 < (𝑛 + (1 / 2)) ∧ (𝑛 + (1 / 2)) < (𝑛 + 1)) → 𝑀 < (𝑛 + 1)))
1912, 14, 17, 18syl3anc 1368 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((𝑀 < (𝑛 + (1 / 2)) ∧ (𝑛 + (1 / 2)) < (𝑛 + 1)) → 𝑀 < (𝑛 + 1)))
2010, 19mpan2d 693 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) → 𝑀 < (𝑛 + 1)))
21 zleltp1 12021 . . . . . . . . . . . 12 ((𝑀 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + 1)))
2221ancoms 462 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + 1)))
2320, 22sylibrd 262 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) → 𝑀𝑛))
24 halfgt0 11841 . . . . . . . . . . . 12 0 < (1 / 2)
253, 5jca 515 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → ((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ))
2625adantr 484 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ))
27 ltaddpos 11119 . . . . . . . . . . . . 13 (((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ) → (0 < (1 / 2) ↔ 𝑛 < (𝑛 + (1 / 2))))
2826, 27syl 17 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (0 < (1 / 2) ↔ 𝑛 < (𝑛 + (1 / 2))))
2924, 28mpbii 236 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑛 < (𝑛 + (1 / 2)))
305adantr 484 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑛 ∈ ℝ)
31 lelttr 10720 . . . . . . . . . . . 12 ((𝑀 ∈ ℝ ∧ 𝑛 ∈ ℝ ∧ (𝑛 + (1 / 2)) ∈ ℝ) → ((𝑀𝑛𝑛 < (𝑛 + (1 / 2))) → 𝑀 < (𝑛 + (1 / 2))))
3212, 30, 14, 31syl3anc 1368 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((𝑀𝑛𝑛 < (𝑛 + (1 / 2))) → 𝑀 < (𝑛 + (1 / 2))))
3329, 32mpan2d 693 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + (1 / 2))))
3423, 33impbid 215 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) ↔ 𝑀𝑛))
35 zcn 11974 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → 𝑛 ∈ ℂ)
36 1cnd 10625 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → 1 ∈ ℂ)
37 2cnne0 11835 . . . . . . . . . . . . 13 (2 ∈ ℂ ∧ 2 ≠ 0)
3837a1i 11 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → (2 ∈ ℂ ∧ 2 ≠ 0))
39 muldivdir 11322 . . . . . . . . . . . 12 ((𝑛 ∈ ℂ ∧ 1 ∈ ℂ ∧ (2 ∈ ℂ ∧ 2 ≠ 0)) → (((2 · 𝑛) + 1) / 2) = (𝑛 + (1 / 2)))
4035, 36, 38, 39syl3anc 1368 . . . . . . . . . . 11 (𝑛 ∈ ℤ → (((2 · 𝑛) + 1) / 2) = (𝑛 + (1 / 2)))
4140breq2d 5042 . . . . . . . . . 10 (𝑛 ∈ ℤ → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑛 + (1 / 2))))
4241adantr 484 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑛 + (1 / 2))))
43 2z 12002 . . . . . . . . . . . . . . . . 17 2 ∈ ℤ
4443a1i 11 . . . . . . . . . . . . . . . 16 (𝑛 ∈ ℤ → 2 ∈ ℤ)
45 id 22 . . . . . . . . . . . . . . . 16 (𝑛 ∈ ℤ → 𝑛 ∈ ℤ)
4644, 45zmulcld 12081 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (2 · 𝑛) ∈ ℤ)
4746zcnd 12076 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (2 · 𝑛) ∈ ℂ)
4847adantr 484 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (2 · 𝑛) ∈ ℂ)
49 pncan1 11053 . . . . . . . . . . . . 13 ((2 · 𝑛) ∈ ℂ → (((2 · 𝑛) + 1) − 1) = (2 · 𝑛))
5048, 49syl 17 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (((2 · 𝑛) + 1) − 1) = (2 · 𝑛))
5150oveq1d 7150 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((((2 · 𝑛) + 1) − 1) / 2) = ((2 · 𝑛) / 2))
52 2cnd 11703 . . . . . . . . . . . . 13 (𝑛 ∈ ℤ → 2 ∈ ℂ)
53 2ne0 11729 . . . . . . . . . . . . . 14 2 ≠ 0
5453a1i 11 . . . . . . . . . . . . 13 (𝑛 ∈ ℤ → 2 ≠ 0)
5535, 52, 54divcan3d 11410 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → ((2 · 𝑛) / 2) = 𝑛)
5655adantr 484 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((2 · 𝑛) / 2) = 𝑛)
5751, 56eqtrd 2833 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((((2 · 𝑛) + 1) − 1) / 2) = 𝑛)
5857breq2d 5042 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2) ↔ 𝑀𝑛))
5934, 42, 583bitr4d 314 . . . . . . . 8 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2)))
60 oveq1 7142 . . . . . . . . . 10 (((2 · 𝑛) + 1) = 𝑁 → (((2 · 𝑛) + 1) / 2) = (𝑁 / 2))
6160breq2d 5042 . . . . . . . . 9 (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑁 / 2)))
62 oveq1 7142 . . . . . . . . . . 11 (((2 · 𝑛) + 1) = 𝑁 → (((2 · 𝑛) + 1) − 1) = (𝑁 − 1))
6362oveq1d 7150 . . . . . . . . . 10 (((2 · 𝑛) + 1) = 𝑁 → ((((2 · 𝑛) + 1) − 1) / 2) = ((𝑁 − 1) / 2))
6463breq2d 5042 . . . . . . . . 9 (((2 · 𝑛) + 1) = 𝑁 → (𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))
6561, 64bibi12d 349 . . . . . . . 8 (((2 · 𝑛) + 1) = 𝑁 → ((𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2)) ↔ (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2))))
6659, 65syl5ibcom 248 . . . . . . 7 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2))))
6766ex 416 . . . . . 6 (𝑛 ∈ ℤ → (𝑀 ∈ ℤ → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
6867adantl 485 . . . . 5 ((𝑁 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (𝑀 ∈ ℤ → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
6968com23 86 . . . 4 ((𝑁 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
7069rexlimdva 3243 . . 3 (𝑁 ∈ ℤ → (∃𝑛 ∈ ℤ ((2 · 𝑛) + 1) = 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
711, 70sylbid 243 . 2 (𝑁 ∈ ℤ → (¬ 2 ∥ 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
72713imp 1108 1 ((𝑁 ∈ ℤ ∧ ¬ 2 ∥ 𝑁𝑀 ∈ ℤ) → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))
Colors of variables: wff setvar class
Syntax hints:  ¬ wn 3  wi 4  wb 209  wa 399  w3a 1084   = wceq 1538  wcel 2111  wne 2987  wrex 3107   class class class wbr 5030  (class class class)co 7135  cc 10524  cr 10525  0cc0 10526  1c1 10527   + caddc 10529   · cmul 10531   < clt 10664  cle 10665  cmin 10859   / cdiv 11286  2c2 11680  cz 11969  cdvds 15599
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 1911  ax-6 1970  ax-7 2015  ax-8 2113  ax-9 2121  ax-10 2142  ax-11 2158  ax-12 2175  ax-ext 2770  ax-sep 5167  ax-nul 5174  ax-pow 5231  ax-pr 5295  ax-un 7441  ax-resscn 10583  ax-1cn 10584  ax-icn 10585  ax-addcl 10586  ax-addrcl 10587  ax-mulcl 10588  ax-mulrcl 10589  ax-mulcom 10590  ax-addass 10591  ax-mulass 10592  ax-distr 10593  ax-i2m1 10594  ax-1ne0 10595  ax-1rid 10596  ax-rnegex 10597  ax-rrecex 10598  ax-cnre 10599  ax-pre-lttri 10600  ax-pre-lttrn 10601  ax-pre-ltadd 10602  ax-pre-mulgt0 10603
This theorem depends on definitions:  df-bi 210  df-an 400  df-or 845  df-3or 1085  df-3an 1086  df-tru 1541  df-ex 1782  df-nf 1786  df-sb 2070  df-mo 2598  df-eu 2629  df-clab 2777  df-cleq 2791  df-clel 2870  df-nfc 2938  df-ne 2988  df-nel 3092  df-ral 3111  df-rex 3112  df-reu 3113  df-rmo 3114  df-rab 3115  df-v 3443  df-sbc 3721  df-csb 3829  df-dif 3884  df-un 3886  df-in 3888  df-ss 3898  df-pss 3900  df-nul 4244  df-if 4426  df-pw 4499  df-sn 4526  df-pr 4528  df-tp 4530  df-op 4532  df-uni 4801  df-iun 4883  df-br 5031  df-opab 5093  df-mpt 5111  df-tr 5137  df-id 5425  df-eprel 5430  df-po 5438  df-so 5439  df-fr 5478  df-we 5480  df-xp 5525  df-rel 5526  df-cnv 5527  df-co 5528  df-dm 5529  df-rn 5530  df-res 5531  df-ima 5532  df-pred 6116  df-ord 6162  df-on 6163  df-lim 6164  df-suc 6165  df-iota 6283  df-fun 6326  df-fn 6327  df-f 6328  df-f1 6329  df-fo 6330  df-f1o 6331  df-fv 6332  df-riota 7093  df-ov 7138  df-oprab 7139  df-mpo 7140  df-om 7561  df-wrecs 7930  df-recs 7991  df-rdg 8029  df-er 8272  df-en 8493  df-dom 8494  df-sdom 8495  df-pnf 10666  df-mnf 10667  df-xr 10668  df-ltxr 10669  df-le 10670  df-sub 10861  df-neg 10862  df-div 11287  df-nn 11626  df-2 11688  df-n0 11886  df-z 11970  df-dvds 15600
This theorem is referenced by:  gausslemma2dlem1a  25949
  Copyright terms: Public domain W3C validator