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

Theorem divides 15965
Description: Define the divides relation. 𝑀𝑁 means 𝑀 divides into 𝑁 with no remainder. For example, 3 ∥ 6 (ex-dvds 28820). As proven in dvdsval3 15967, 𝑀𝑁 ↔ (𝑁 mod 𝑀) = 0. See divides 15965 and dvdsval2 15966 for other equivalent expressions. (Contributed by Paul Chapman, 21-Mar-2011.)
Assertion
Ref Expression
divides ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝑀𝑁 ↔ ∃𝑛 ∈ ℤ (𝑛 · 𝑀) = 𝑁))
Distinct variable groups:   𝑛,𝑀   𝑛,𝑁

Proof of Theorem divides
Dummy variables 𝑥 𝑦 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 df-br 5075 . . 3 (𝑀𝑁 ↔ ⟨𝑀, 𝑁⟩ ∈ ∥ )
2 df-dvds 15964 . . . 4 ∥ = {⟨𝑥, 𝑦⟩ ∣ ((𝑥 ∈ ℤ ∧ 𝑦 ∈ ℤ) ∧ ∃𝑛 ∈ ℤ (𝑛 · 𝑥) = 𝑦)}
32eleq2i 2830 . . 3 (⟨𝑀, 𝑁⟩ ∈ ∥ ↔ ⟨𝑀, 𝑁⟩ ∈ {⟨𝑥, 𝑦⟩ ∣ ((𝑥 ∈ ℤ ∧ 𝑦 ∈ ℤ) ∧ ∃𝑛 ∈ ℤ (𝑛 · 𝑥) = 𝑦)})
41, 3bitri 274 . 2 (𝑀𝑁 ↔ ⟨𝑀, 𝑁⟩ ∈ {⟨𝑥, 𝑦⟩ ∣ ((𝑥 ∈ ℤ ∧ 𝑦 ∈ ℤ) ∧ ∃𝑛 ∈ ℤ (𝑛 · 𝑥) = 𝑦)})
5 oveq2 7283 . . . . 5 (𝑥 = 𝑀 → (𝑛 · 𝑥) = (𝑛 · 𝑀))
65eqeq1d 2740 . . . 4 (𝑥 = 𝑀 → ((𝑛 · 𝑥) = 𝑦 ↔ (𝑛 · 𝑀) = 𝑦))
76rexbidv 3226 . . 3 (𝑥 = 𝑀 → (∃𝑛 ∈ ℤ (𝑛 · 𝑥) = 𝑦 ↔ ∃𝑛 ∈ ℤ (𝑛 · 𝑀) = 𝑦))
8 eqeq2 2750 . . . 4 (𝑦 = 𝑁 → ((𝑛 · 𝑀) = 𝑦 ↔ (𝑛 · 𝑀) = 𝑁))
98rexbidv 3226 . . 3 (𝑦 = 𝑁 → (∃𝑛 ∈ ℤ (𝑛 · 𝑀) = 𝑦 ↔ ∃𝑛 ∈ ℤ (𝑛 · 𝑀) = 𝑁))
107, 9opelopab2 5454 . 2 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (⟨𝑀, 𝑁⟩ ∈ {⟨𝑥, 𝑦⟩ ∣ ((𝑥 ∈ ℤ ∧ 𝑦 ∈ ℤ) ∧ ∃𝑛 ∈ ℤ (𝑛 · 𝑥) = 𝑦)} ↔ ∃𝑛 ∈ ℤ (𝑛 · 𝑀) = 𝑁))
114, 10bitrid 282 1 ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝑀𝑁 ↔ ∃𝑛 ∈ ℤ (𝑛 · 𝑀) = 𝑁))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 205  wa 396   = wceq 1539  wcel 2106  wrex 3065  cop 4567   class class class wbr 5074  {copab 5136  (class class class)co 7275   · cmul 10876  cz 12319  cdvds 15963
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-ext 2709  ax-sep 5223  ax-nul 5230  ax-pr 5352
This theorem depends on definitions:  df-bi 206  df-an 397  df-or 845  df-3an 1088  df-tru 1542  df-fal 1552  df-ex 1783  df-sb 2068  df-clab 2716  df-cleq 2730  df-clel 2816  df-rex 3070  df-rab 3073  df-v 3434  df-dif 3890  df-un 3892  df-in 3894  df-ss 3904  df-nul 4257  df-if 4460  df-sn 4562  df-pr 4564  df-op 4568  df-uni 4840  df-br 5075  df-opab 5137  df-iota 6391  df-fv 6441  df-ov 7278  df-dvds 15964
This theorem is referenced by:  dvdsval2  15966  dvds0lem  15976  dvds1lem  15977  dvds2lem  15978  0dvds  15986  dvdsle  16019  divconjdvds  16024  dvdsexp2im  16036  odd2np1  16050  even2n  16051  oddm1even  16052  opeo  16074  omeo  16075  m1exp1  16085  divalglem4  16105  divalglem9  16110  divalgb  16113  modremain  16117  zeqzmulgcd  16217  bezoutlem4  16250  gcddiv  16259  dvdssqim  16264  coprmdvds2  16359  congr  16369  divgcdcoprm0  16370  cncongr2  16373  dvdsnprmd  16395  prmpwdvds  16605  odmulg  19163  gexdvdsi  19188  lgsquadlem2  26529  dvdsexpim  40328  dvdsrabdioph  40632  jm2.26a  40822  coskpi2  43407  cosknegpi  43410  fourierswlem  43771  dfeven2  45101
  Copyright terms: Public domain W3C validator