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

Theorem divass 11928
Description: An associative law for division. (Contributed by NM, 2-Aug-2004.)
Assertion
Ref Expression
divass ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 · 𝐵) / 𝐶) = (𝐴 · (𝐵 / 𝐶)))

Proof of Theorem divass
StepHypRef Expression
1 reccl 11917 . . 3 ((𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) → (1 / 𝐶) ∈ ℂ)
2 mulass 11234 . . 3 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (1 / 𝐶) ∈ ℂ) → ((𝐴 · 𝐵) · (1 / 𝐶)) = (𝐴 · (𝐵 · (1 / 𝐶))))
31, 2syl3an3 1162 . 2 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 · 𝐵) · (1 / 𝐶)) = (𝐴 · (𝐵 · (1 / 𝐶))))
4 mulcl 11230 . . . 4 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ) → (𝐴 · 𝐵) ∈ ℂ)
543adant3 1129 . . 3 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → (𝐴 · 𝐵) ∈ ℂ)
6 simp3l 1198 . . 3 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → 𝐶 ∈ ℂ)
7 simp3r 1199 . . 3 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → 𝐶 ≠ 0)
8 divrec 11926 . . 3 (((𝐴 · 𝐵) ∈ ℂ ∧ 𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) → ((𝐴 · 𝐵) / 𝐶) = ((𝐴 · 𝐵) · (1 / 𝐶)))
95, 6, 7, 8syl3anc 1368 . 2 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 · 𝐵) / 𝐶) = ((𝐴 · 𝐵) · (1 / 𝐶)))
10 simp2 1134 . . . 4 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → 𝐵 ∈ ℂ)
11 divrec 11926 . . . 4 ((𝐵 ∈ ℂ ∧ 𝐶 ∈ ℂ ∧ 𝐶 ≠ 0) → (𝐵 / 𝐶) = (𝐵 · (1 / 𝐶)))
1210, 6, 7, 11syl3anc 1368 . . 3 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → (𝐵 / 𝐶) = (𝐵 · (1 / 𝐶)))
1312oveq2d 7442 . 2 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → (𝐴 · (𝐵 / 𝐶)) = (𝐴 · (𝐵 · (1 / 𝐶))))
143, 9, 133eqtr4d 2778 1 ((𝐴 ∈ ℂ ∧ 𝐵 ∈ ℂ ∧ (𝐶 ∈ ℂ ∧ 𝐶 ≠ 0)) → ((𝐴 · 𝐵) / 𝐶) = (𝐴 · (𝐵 / 𝐶)))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 394  w3a 1084   = wceq 1533  wcel 2098  wne 2937  (class class class)co 7426  cc 11144  0cc0 11146  1c1 11147   · cmul 11151   / cdiv 11909
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1789  ax-4 1803  ax-5 1905  ax-6 1963  ax-7 2003  ax-8 2100  ax-9 2108  ax-10 2129  ax-11 2146  ax-12 2166  ax-ext 2699  ax-sep 5303  ax-nul 5310  ax-pow 5369  ax-pr 5433  ax-un 7746  ax-resscn 11203  ax-1cn 11204  ax-icn 11205  ax-addcl 11206  ax-addrcl 11207  ax-mulcl 11208  ax-mulrcl 11209  ax-mulcom 11210  ax-addass 11211  ax-mulass 11212  ax-distr 11213  ax-i2m1 11214  ax-1ne0 11215  ax-1rid 11216  ax-rnegex 11217  ax-rrecex 11218  ax-cnre 11219  ax-pre-lttri 11220  ax-pre-lttrn 11221  ax-pre-ltadd 11222  ax-pre-mulgt0 11223
This theorem depends on definitions:  df-bi 206  df-an 395  df-or 846  df-3or 1085  df-3an 1086  df-tru 1536  df-fal 1546  df-ex 1774  df-nf 1778  df-sb 2060  df-mo 2529  df-eu 2558  df-clab 2706  df-cleq 2720  df-clel 2806  df-nfc 2881  df-ne 2938  df-nel 3044  df-ral 3059  df-rex 3068  df-rmo 3374  df-reu 3375  df-rab 3431  df-v 3475  df-sbc 3779  df-csb 3895  df-dif 3952  df-un 3954  df-in 3956  df-ss 3966  df-nul 4327  df-if 4533  df-pw 4608  df-sn 4633  df-pr 4635  df-op 4639  df-uni 4913  df-br 5153  df-opab 5215  df-mpt 5236  df-id 5580  df-po 5594  df-so 5595  df-xp 5688  df-rel 5689  df-cnv 5690  df-co 5691  df-dm 5692  df-rn 5693  df-res 5694  df-ima 5695  df-iota 6505  df-fun 6555  df-fn 6556  df-f 6557  df-f1 6558  df-fo 6559  df-f1o 6560  df-fv 6561  df-riota 7382  df-ov 7429  df-oprab 7430  df-mpo 7431  df-er 8731  df-en 8971  df-dom 8972  df-sdom 8973  df-pnf 11288  df-mnf 11289  df-xr 11290  df-ltxr 11291  df-le 11292  df-sub 11484  df-neg 11485  df-div 11910
This theorem is referenced by:  div23  11929  div32  11930  divmulass  11933  divmulasscom  11934  divasszi  12002  divassd  12063  lt2mul2div  12130  zdivmul  12672  mertenslem1  15870  efi4p  16121  mulsucdiv2z  16337  relogbreexp  26727  divsqrtsumlem  26932  basellem8  27040  logexprlim  27178  bposlem6  27242  lgsquadlem2  27334  chebbnd1lem3  27424  vmadivsum  27435  dchrmusum2  27447  dchrisum0lem1b  27468  dchrisum0lem2  27471  mudivsum  27483  mulog2sumlem2  27488  selberglem1  27498  selberglem2  27499  pntlemb  27550  pntlemr  27555  pntlemj  27556  pntlemf  27558  pntlemk  27559  pntlemo  27560  dvasin  37210  stoweidlem24  45441
  Copyright terms: Public domain W3C validator