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

Theorem gcdabsOLD 16480
Description: Obsolete version of gcdabs 16479 as of 15-Sep-2024. (Contributed by Paul Chapman, 31-Mar-2011.) (New usage is discouraged.) (Proof modification is discouraged.)
Assertion
Ref Expression
gcdabsOLD ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁))

Proof of Theorem gcdabsOLD
StepHypRef Expression
1 zre 12566 . . 3 (𝑀 ∈ ℤ → 𝑀 ∈ ℝ)
2 zre 12566 . . 3 (𝑁 ∈ ℤ → 𝑁 ∈ ℝ)
3 absor 15253 . . . 4 (𝑀 ∈ ℝ → ((abs‘𝑀) = 𝑀 ∨ (abs‘𝑀) = -𝑀))
4 absor 15253 . . . 4 (𝑁 ∈ ℝ → ((abs‘𝑁) = 𝑁 ∨ (abs‘𝑁) = -𝑁))
53, 4anim12i 612 . . 3 ((𝑀 ∈ ℝ ∧ 𝑁 ∈ ℝ) → (((abs‘𝑀) = 𝑀 ∨ (abs‘𝑀) = -𝑀) ∧ ((abs‘𝑁) = 𝑁 ∨ (abs‘𝑁) = -𝑁)))
61, 2, 5syl2an 595 . 2 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (((abs‘𝑀) = 𝑀 ∨ (abs‘𝑀) = -𝑀) ∧ ((abs‘𝑁) = 𝑁 ∨ (abs‘𝑁) = -𝑁)))
7 oveq12 7414 . . . 4 (((abs‘𝑀) = 𝑀 ∧ (abs‘𝑁) = 𝑁) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁))
87a1i 11 . . 3 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (((abs‘𝑀) = 𝑀 ∧ (abs‘𝑁) = 𝑁) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁)))
9 oveq12 7414 . . . . 5 (((abs‘𝑀) = -𝑀 ∧ (abs‘𝑁) = 𝑁) → ((abs‘𝑀) gcd (abs‘𝑁)) = (-𝑀 gcd 𝑁))
10 neggcd 16471 . . . . 5 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (-𝑀 gcd 𝑁) = (𝑀 gcd 𝑁))
119, 10sylan9eqr 2788 . . . 4 (((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) ∧ ((abs‘𝑀) = -𝑀 ∧ (abs‘𝑁) = 𝑁)) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁))
1211ex 412 . . 3 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (((abs‘𝑀) = -𝑀 ∧ (abs‘𝑁) = 𝑁) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁)))
13 oveq12 7414 . . . . 5 (((abs‘𝑀) = 𝑀 ∧ (abs‘𝑁) = -𝑁) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd -𝑁))
14 gcdneg 16470 . . . . 5 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝑀 gcd -𝑁) = (𝑀 gcd 𝑁))
1513, 14sylan9eqr 2788 . . . 4 (((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) ∧ ((abs‘𝑀) = 𝑀 ∧ (abs‘𝑁) = -𝑁)) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁))
1615ex 412 . . 3 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (((abs‘𝑀) = 𝑀 ∧ (abs‘𝑁) = -𝑁) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁)))
17 oveq12 7414 . . . . 5 (((abs‘𝑀) = -𝑀 ∧ (abs‘𝑁) = -𝑁) → ((abs‘𝑀) gcd (abs‘𝑁)) = (-𝑀 gcd -𝑁))
18 znegcl 12601 . . . . . . 7 (𝑀 ∈ ℤ → -𝑀 ∈ ℤ)
19 gcdneg 16470 . . . . . . 7 ((-𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (-𝑀 gcd -𝑁) = (-𝑀 gcd 𝑁))
2018, 19sylan 579 . . . . . 6 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (-𝑀 gcd -𝑁) = (-𝑀 gcd 𝑁))
2120, 10eqtrd 2766 . . . . 5 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (-𝑀 gcd -𝑁) = (𝑀 gcd 𝑁))
2217, 21sylan9eqr 2788 . . . 4 (((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) ∧ ((abs‘𝑀) = -𝑀 ∧ (abs‘𝑁) = -𝑁)) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁))
2322ex 412 . . 3 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (((abs‘𝑀) = -𝑀 ∧ (abs‘𝑁) = -𝑁) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁)))
248, 12, 16, 23ccased 1035 . 2 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → ((((abs‘𝑀) = 𝑀 ∨ (abs‘𝑀) = -𝑀) ∧ ((abs‘𝑁) = 𝑁 ∨ (abs‘𝑁) = -𝑁)) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁)))
256, 24mpd 15 1 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → ((abs‘𝑀) gcd (abs‘𝑁)) = (𝑀 gcd 𝑁))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 395  wo 844   = wceq 1533  wcel 2098  cfv 6537  (class class class)co 7405  cr 11111  -cneg 11449  cz 12562  abscabs 15187   gcd cgcd 16442
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 2163  ax-ext 2697  ax-sep 5292  ax-nul 5299  ax-pow 5356  ax-pr 5420  ax-un 7722  ax-cnex 11168  ax-resscn 11169  ax-1cn 11170  ax-icn 11171  ax-addcl 11172  ax-addrcl 11173  ax-mulcl 11174  ax-mulrcl 11175  ax-mulcom 11176  ax-addass 11177  ax-mulass 11178  ax-distr 11179  ax-i2m1 11180  ax-1ne0 11181  ax-1rid 11182  ax-rnegex 11183  ax-rrecex 11184  ax-cnre 11185  ax-pre-lttri 11186  ax-pre-lttrn 11187  ax-pre-ltadd 11188  ax-pre-mulgt0 11189  ax-pre-sup 11190
This theorem depends on definitions:  df-bi 206  df-an 396  df-or 845  df-3or 1085  df-3an 1086  df-tru 1536  df-fal 1546  df-ex 1774  df-nf 1778  df-sb 2060  df-mo 2528  df-eu 2557  df-clab 2704  df-cleq 2718  df-clel 2804  df-nfc 2879  df-ne 2935  df-nel 3041  df-ral 3056  df-rex 3065  df-rmo 3370  df-reu 3371  df-rab 3427  df-v 3470  df-sbc 3773  df-csb 3889  df-dif 3946  df-un 3948  df-in 3950  df-ss 3960  df-pss 3962  df-nul 4318  df-if 4524  df-pw 4599  df-sn 4624  df-pr 4626  df-op 4630  df-uni 4903  df-iun 4992  df-br 5142  df-opab 5204  df-mpt 5225  df-tr 5259  df-id 5567  df-eprel 5573  df-po 5581  df-so 5582  df-fr 5624  df-we 5626  df-xp 5675  df-rel 5676  df-cnv 5677  df-co 5678  df-dm 5679  df-rn 5680  df-res 5681  df-ima 5682  df-pred 6294  df-ord 6361  df-on 6362  df-lim 6363  df-suc 6364  df-iota 6489  df-fun 6539  df-fn 6540  df-f 6541  df-f1 6542  df-fo 6543  df-f1o 6544  df-fv 6545  df-riota 7361  df-ov 7408  df-oprab 7409  df-mpo 7410  df-om 7853  df-2nd 7975  df-frecs 8267  df-wrecs 8298  df-recs 8372  df-rdg 8411  df-er 8705  df-en 8942  df-dom 8943  df-sdom 8944  df-sup 9439  df-inf 9440  df-pnf 11254  df-mnf 11255  df-xr 11256  df-ltxr 11257  df-le 11258  df-sub 11450  df-neg 11451  df-div 11876  df-nn 12217  df-2 12279  df-3 12280  df-n0 12477  df-z 12563  df-uz 12827  df-rp 12981  df-seq 13973  df-exp 14033  df-cj 15052  df-re 15053  df-im 15054  df-sqrt 15188  df-abs 15189  df-dvds 16205  df-gcd 16443
This theorem is referenced by: (None)
  Copyright terms: Public domain W3C validator