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

Theorem lemul2a 12065
Description: Multiplication of both sides of 'less than or equal to' by a nonnegative number. (Contributed by Paul Chapman, 7-Sep-2007.)
Assertion
Ref Expression
lemul2a (((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) ∧ 𝐴𝐵) → (𝐶 · 𝐴) ≤ (𝐶 · 𝐵))

Proof of Theorem lemul2a
StepHypRef Expression
1 lemul1a 12064 . 2 (((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) ∧ 𝐴𝐵) → (𝐴 · 𝐶) ≤ (𝐵 · 𝐶))
2 recn 11196 . . . . . 6 (𝐴 ∈ ℝ → 𝐴 ∈ ℂ)
3 recn 11196 . . . . . 6 (𝐶 ∈ ℝ → 𝐶 ∈ ℂ)
4 mulcom 11192 . . . . . 6 ((𝐴 ∈ ℂ ∧ 𝐶 ∈ ℂ) → (𝐴 · 𝐶) = (𝐶 · 𝐴))
52, 3, 4syl2an 597 . . . . 5 ((𝐴 ∈ ℝ ∧ 𝐶 ∈ ℝ) → (𝐴 · 𝐶) = (𝐶 · 𝐴))
65adantrr 716 . . . 4 ((𝐴 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) → (𝐴 · 𝐶) = (𝐶 · 𝐴))
763adant2 1132 . . 3 ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) → (𝐴 · 𝐶) = (𝐶 · 𝐴))
87adantr 482 . 2 (((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) ∧ 𝐴𝐵) → (𝐴 · 𝐶) = (𝐶 · 𝐴))
9 recn 11196 . . . . . 6 (𝐵 ∈ ℝ → 𝐵 ∈ ℂ)
10 mulcom 11192 . . . . . 6 ((𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ) → (𝐵 · 𝐶) = (𝐶 · 𝐵))
119, 3, 10syl2an 597 . . . . 5 ((𝐵 ∈ ℝ ∧ 𝐶 ∈ ℝ) → (𝐵 · 𝐶) = (𝐶 · 𝐵))
1211adantrr 716 . . . 4 ((𝐵 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) → (𝐵 · 𝐶) = (𝐶 · 𝐵))
13123adant1 1131 . . 3 ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) → (𝐵 · 𝐶) = (𝐶 · 𝐵))
1413adantr 482 . 2 (((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) ∧ 𝐴𝐵) → (𝐵 · 𝐶) = (𝐶 · 𝐵))
151, 8, 143brtr3d 5178 1 (((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ (𝐶 ∈ ℝ ∧ 0 ≤ 𝐶)) ∧ 𝐴𝐵) → (𝐶 · 𝐴) ≤ (𝐶 · 𝐵))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 397  w3a 1088   = wceq 1542  wcel 2107   class class class wbr 5147  (class class class)co 7404  cc 11104  cr 11105  0cc0 11106   · cmul 11111  cle 11245
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 1914  ax-6 1972  ax-7 2012  ax-8 2109  ax-9 2117  ax-10 2138  ax-11 2155  ax-12 2172  ax-ext 2704  ax-sep 5298  ax-nul 5305  ax-pow 5362  ax-pr 5426  ax-un 7720  ax-resscn 11163  ax-1cn 11164  ax-icn 11165  ax-addcl 11166  ax-addrcl 11167  ax-mulcl 11168  ax-mulrcl 11169  ax-mulcom 11170  ax-addass 11171  ax-mulass 11172  ax-distr 11173  ax-i2m1 11174  ax-1ne0 11175  ax-1rid 11176  ax-rnegex 11177  ax-rrecex 11178  ax-cnre 11179  ax-pre-lttri 11180  ax-pre-lttrn 11181  ax-pre-ltadd 11182  ax-pre-mulgt0 11183
This theorem depends on definitions:  df-bi 206  df-an 398  df-or 847  df-3or 1089  df-3an 1090  df-tru 1545  df-fal 1555  df-ex 1783  df-nf 1787  df-sb 2069  df-mo 2535  df-eu 2564  df-clab 2711  df-cleq 2725  df-clel 2811  df-nfc 2886  df-ne 2942  df-nel 3048  df-ral 3063  df-rex 3072  df-reu 3378  df-rab 3434  df-v 3477  df-sbc 3777  df-csb 3893  df-dif 3950  df-un 3952  df-in 3954  df-ss 3964  df-nul 4322  df-if 4528  df-pw 4603  df-sn 4628  df-pr 4630  df-op 4634  df-uni 4908  df-br 5148  df-opab 5210  df-mpt 5231  df-id 5573  df-po 5587  df-so 5588  df-xp 5681  df-rel 5682  df-cnv 5683  df-co 5684  df-dm 5685  df-rn 5686  df-res 5687  df-ima 5688  df-iota 6492  df-fun 6542  df-fn 6543  df-f 6544  df-f1 6545  df-fo 6546  df-f1o 6547  df-fv 6548  df-riota 7360  df-ov 7407  df-oprab 7408  df-mpo 7409  df-er 8699  df-en 8936  df-dom 8937  df-sdom 8938  df-pnf 11246  df-mnf 11247  df-xr 11248  df-ltxr 11249  df-le 11250  df-sub 11442  df-neg 11443
This theorem is referenced by:  lemul12b  12067  ledivp1  12112  ledivp1i  12135  ltdivp1i  12136  lemul2ad  12150  supmul1  12179  facavg  14257  mulcn2  15536  cvgrat  15825  mertenslem1  15826  prmreclem3  16847  nmoco  24236  blcvx  24296  fsumharmonic  26496  bposlem1  26767  dchrvmasumiflem1  26984  nmoub3i  30004  htthlem  30148  nmopub2tALT  31140  nmfnleub2  31157  nmophmi  31262  nmopadjlem  31320  nmopcoadji  31332  lediv2aALT  34600  stoweidlem24  44675
  Copyright terms: Public domain W3C validator