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

Theorem ltoddhalfle 16080
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 16060 . . 3 (𝑁 ∈ ℤ → (¬ 2 ∥ 𝑁 ↔ ∃𝑛 ∈ ℤ ((2 · 𝑛) + 1) = 𝑁))
2 halfre 12197 . . . . . . . . . . . . . . . 16 (1 / 2) ∈ ℝ
32a1i 11 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (1 / 2) ∈ ℝ)
4 1red 10986 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → 1 ∈ ℝ)
5 zre 12333 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → 𝑛 ∈ ℝ)
63, 4, 53jca 1127 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → ((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ))
76adantr 481 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ))
8 halflt1 12201 . . . . . . . . . . . . 13 (1 / 2) < 1
9 axltadd 11058 . . . . . . . . . . . . 13 (((1 / 2) ∈ ℝ ∧ 1 ∈ ℝ ∧ 𝑛 ∈ ℝ) → ((1 / 2) < 1 → (𝑛 + (1 / 2)) < (𝑛 + 1)))
107, 8, 9mpisyl 21 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + (1 / 2)) < (𝑛 + 1))
11 zre 12333 . . . . . . . . . . . . . 14 (𝑀 ∈ ℤ → 𝑀 ∈ ℝ)
1211adantl 482 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑀 ∈ ℝ)
135, 3readdcld 11014 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (𝑛 + (1 / 2)) ∈ ℝ)
1413adantr 481 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + (1 / 2)) ∈ ℝ)
15 peano2z 12371 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (𝑛 + 1) ∈ ℤ)
1615zred 12436 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (𝑛 + 1) ∈ ℝ)
1716adantr 481 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑛 + 1) ∈ ℝ)
18 lttr 11061 . . . . . . . . . . . . 13 ((𝑀 ∈ ℝ ∧ (𝑛 + (1 / 2)) ∈ ℝ ∧ (𝑛 + 1) ∈ ℝ) → ((𝑀 < (𝑛 + (1 / 2)) ∧ (𝑛 + (1 / 2)) < (𝑛 + 1)) → 𝑀 < (𝑛 + 1)))
1912, 14, 17, 18syl3anc 1370 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((𝑀 < (𝑛 + (1 / 2)) ∧ (𝑛 + (1 / 2)) < (𝑛 + 1)) → 𝑀 < (𝑛 + 1)))
2010, 19mpan2d 691 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) → 𝑀 < (𝑛 + 1)))
21 zleltp1 12381 . . . . . . . . . . . 12 ((𝑀 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + 1)))
2221ancoms 459 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + 1)))
2320, 22sylibrd 258 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) → 𝑀𝑛))
24 halfgt0 12199 . . . . . . . . . . . 12 0 < (1 / 2)
253, 5jca 512 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → ((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ))
2625adantr 481 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ))
27 ltaddpos 11475 . . . . . . . . . . . . 13 (((1 / 2) ∈ ℝ ∧ 𝑛 ∈ ℝ) → (0 < (1 / 2) ↔ 𝑛 < (𝑛 + (1 / 2))))
2826, 27syl 17 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (0 < (1 / 2) ↔ 𝑛 < (𝑛 + (1 / 2))))
2924, 28mpbii 232 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑛 < (𝑛 + (1 / 2)))
305adantr 481 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → 𝑛 ∈ ℝ)
31 lelttr 11075 . . . . . . . . . . . 12 ((𝑀 ∈ ℝ ∧ 𝑛 ∈ ℝ ∧ (𝑛 + (1 / 2)) ∈ ℝ) → ((𝑀𝑛𝑛 < (𝑛 + (1 / 2))) → 𝑀 < (𝑛 + (1 / 2))))
3212, 30, 14, 31syl3anc 1370 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((𝑀𝑛𝑛 < (𝑛 + (1 / 2))) → 𝑀 < (𝑛 + (1 / 2))))
3329, 32mpan2d 691 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀𝑛𝑀 < (𝑛 + (1 / 2))))
3423, 33impbid 211 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (𝑛 + (1 / 2)) ↔ 𝑀𝑛))
35 zcn 12334 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → 𝑛 ∈ ℂ)
36 1cnd 10980 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → 1 ∈ ℂ)
37 2cnne0 12193 . . . . . . . . . . . . 13 (2 ∈ ℂ ∧ 2 ≠ 0)
3837a1i 11 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → (2 ∈ ℂ ∧ 2 ≠ 0))
39 muldivdir 11678 . . . . . . . . . . . 12 ((𝑛 ∈ ℂ ∧ 1 ∈ ℂ ∧ (2 ∈ ℂ ∧ 2 ≠ 0)) → (((2 · 𝑛) + 1) / 2) = (𝑛 + (1 / 2)))
4035, 36, 38, 39syl3anc 1370 . . . . . . . . . . 11 (𝑛 ∈ ℤ → (((2 · 𝑛) + 1) / 2) = (𝑛 + (1 / 2)))
4140breq2d 5085 . . . . . . . . . 10 (𝑛 ∈ ℤ → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑛 + (1 / 2))))
4241adantr 481 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑛 + (1 / 2))))
43 2z 12362 . . . . . . . . . . . . . . . . 17 2 ∈ ℤ
4443a1i 11 . . . . . . . . . . . . . . . 16 (𝑛 ∈ ℤ → 2 ∈ ℤ)
45 id 22 . . . . . . . . . . . . . . . 16 (𝑛 ∈ ℤ → 𝑛 ∈ ℤ)
4644, 45zmulcld 12442 . . . . . . . . . . . . . . 15 (𝑛 ∈ ℤ → (2 · 𝑛) ∈ ℤ)
4746zcnd 12437 . . . . . . . . . . . . . 14 (𝑛 ∈ ℤ → (2 · 𝑛) ∈ ℂ)
4847adantr 481 . . . . . . . . . . . . 13 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (2 · 𝑛) ∈ ℂ)
49 pncan1 11409 . . . . . . . . . . . . 13 ((2 · 𝑛) ∈ ℂ → (((2 · 𝑛) + 1) − 1) = (2 · 𝑛))
5048, 49syl 17 . . . . . . . . . . . 12 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (((2 · 𝑛) + 1) − 1) = (2 · 𝑛))
5150oveq1d 7282 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((((2 · 𝑛) + 1) − 1) / 2) = ((2 · 𝑛) / 2))
52 2cnd 12061 . . . . . . . . . . . . 13 (𝑛 ∈ ℤ → 2 ∈ ℂ)
53 2ne0 12087 . . . . . . . . . . . . . 14 2 ≠ 0
5453a1i 11 . . . . . . . . . . . . 13 (𝑛 ∈ ℤ → 2 ≠ 0)
5535, 52, 54divcan3d 11766 . . . . . . . . . . . 12 (𝑛 ∈ ℤ → ((2 · 𝑛) / 2) = 𝑛)
5655adantr 481 . . . . . . . . . . 11 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((2 · 𝑛) / 2) = 𝑛)
5751, 56eqtrd 2778 . . . . . . . . . 10 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → ((((2 · 𝑛) + 1) − 1) / 2) = 𝑛)
5857breq2d 5085 . . . . . . . . 9 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2) ↔ 𝑀𝑛))
5934, 42, 583bitr4d 311 . . . . . . . 8 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2)))
60 oveq1 7274 . . . . . . . . . 10 (((2 · 𝑛) + 1) = 𝑁 → (((2 · 𝑛) + 1) / 2) = (𝑁 / 2))
6160breq2d 5085 . . . . . . . . 9 (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 < (𝑁 / 2)))
62 oveq1 7274 . . . . . . . . . . 11 (((2 · 𝑛) + 1) = 𝑁 → (((2 · 𝑛) + 1) − 1) = (𝑁 − 1))
6362oveq1d 7282 . . . . . . . . . 10 (((2 · 𝑛) + 1) = 𝑁 → ((((2 · 𝑛) + 1) − 1) / 2) = ((𝑁 − 1) / 2))
6463breq2d 5085 . . . . . . . . 9 (((2 · 𝑛) + 1) = 𝑁 → (𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))
6561, 64bibi12d 346 . . . . . . . 8 (((2 · 𝑛) + 1) = 𝑁 → ((𝑀 < (((2 · 𝑛) + 1) / 2) ↔ 𝑀 ≤ ((((2 · 𝑛) + 1) − 1) / 2)) ↔ (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2))))
6659, 65syl5ibcom 244 . . . . . . 7 ((𝑛 ∈ ℤ ∧ 𝑀 ∈ ℤ) → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2))))
6766ex 413 . . . . . 6 (𝑛 ∈ ℤ → (𝑀 ∈ ℤ → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
6867adantl 482 . . . . 5 ((𝑁 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (𝑀 ∈ ℤ → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
6968com23 86 . . . 4 ((𝑁 ∈ ℤ ∧ 𝑛 ∈ ℤ) → (((2 · 𝑛) + 1) = 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
7069rexlimdva 3211 . . 3 (𝑁 ∈ ℤ → (∃𝑛 ∈ ℤ ((2 · 𝑛) + 1) = 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
711, 70sylbid 239 . 2 (𝑁 ∈ ℤ → (¬ 2 ∥ 𝑁 → (𝑀 ∈ ℤ → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))))
72713imp 1110 1 ((𝑁 ∈ ℤ ∧ ¬ 2 ∥ 𝑁𝑀 ∈ ℤ) → (𝑀 < (𝑁 / 2) ↔ 𝑀 ≤ ((𝑁 − 1) / 2)))
Colors of variables: wff setvar class
Syntax hints:  ¬ wn 3  wi 4  wb 205  wa 396  w3a 1086   = wceq 1539  wcel 2106  wne 2943  wrex 3065   class class class wbr 5073  (class class class)co 7267  cc 10879  cr 10880  0cc0 10881  1c1 10882   + caddc 10884   · cmul 10886   < clt 11019  cle 11020  cmin 11215   / cdiv 11642  2c2 12038  cz 12329  cdvds 15973
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1798  ax-4 1812  ax-5 1913  ax-6 1971  ax-7 2011  ax-8 2108  ax-9 2116  ax-10 2137  ax-11 2154  ax-12 2171  ax-ext 2709  ax-sep 5221  ax-nul 5228  ax-pow 5286  ax-pr 5350  ax-un 7578  ax-resscn 10938  ax-1cn 10939  ax-icn 10940  ax-addcl 10941  ax-addrcl 10942  ax-mulcl 10943  ax-mulrcl 10944  ax-mulcom 10945  ax-addass 10946  ax-mulass 10947  ax-distr 10948  ax-i2m1 10949  ax-1ne0 10950  ax-1rid 10951  ax-rnegex 10952  ax-rrecex 10953  ax-cnre 10954  ax-pre-lttri 10955  ax-pre-lttrn 10956  ax-pre-ltadd 10957  ax-pre-mulgt0 10958
This theorem depends on definitions:  df-bi 206  df-an 397  df-or 845  df-3or 1087  df-3an 1088  df-tru 1542  df-fal 1552  df-ex 1783  df-nf 1787  df-sb 2068  df-mo 2540  df-eu 2569  df-clab 2716  df-cleq 2730  df-clel 2816  df-nfc 2889  df-ne 2944  df-nel 3050  df-ral 3069  df-rex 3070  df-reu 3071  df-rmo 3072  df-rab 3073  df-v 3431  df-sbc 3716  df-csb 3832  df-dif 3889  df-un 3891  df-in 3893  df-ss 3903  df-pss 3905  df-nul 4257  df-if 4460  df-pw 4535  df-sn 4562  df-pr 4564  df-op 4568  df-uni 4840  df-iun 4926  df-br 5074  df-opab 5136  df-mpt 5157  df-tr 5191  df-id 5484  df-eprel 5490  df-po 5498  df-so 5499  df-fr 5539  df-we 5541  df-xp 5590  df-rel 5591  df-cnv 5592  df-co 5593  df-dm 5594  df-rn 5595  df-res 5596  df-ima 5597  df-pred 6195  df-ord 6262  df-on 6263  df-lim 6264  df-suc 6265  df-iota 6384  df-fun 6428  df-fn 6429  df-f 6430  df-f1 6431  df-fo 6432  df-f1o 6433  df-fv 6434  df-riota 7224  df-ov 7270  df-oprab 7271  df-mpo 7272  df-om 7703  df-2nd 7821  df-frecs 8084  df-wrecs 8115  df-recs 8189  df-rdg 8228  df-er 8485  df-en 8721  df-dom 8722  df-sdom 8723  df-pnf 11021  df-mnf 11022  df-xr 11023  df-ltxr 11024  df-le 11025  df-sub 11217  df-neg 11218  df-div 11643  df-nn 11984  df-2 12046  df-n0 12244  df-z 12330  df-dvds 15974
This theorem is referenced by:  gausslemma2dlem1a  26523
  Copyright terms: Public domain W3C validator