ILE Home Intuitionistic Logic Explorer < Previous   Next >
Nearby theorems
Mirrors  >  Home  >  ILE Home  >  Th. List  >  nnmulcl GIF version

Theorem nnmulcl 9011
Description: Closure of multiplication of positive integers. (Contributed by NM, 12-Jan-1997.)
Assertion
Ref Expression
nnmulcl ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ) → (𝐴 · 𝐵) ∈ ℕ)

Proof of Theorem nnmulcl
Dummy variables 𝑥 𝑦 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 oveq2 5930 . . . . 5 (𝑥 = 1 → (𝐴 · 𝑥) = (𝐴 · 1))
21eleq1d 2265 . . . 4 (𝑥 = 1 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 1) ∈ ℕ))
32imbi2d 230 . . 3 (𝑥 = 1 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ)))
4 oveq2 5930 . . . . 5 (𝑥 = 𝑦 → (𝐴 · 𝑥) = (𝐴 · 𝑦))
54eleq1d 2265 . . . 4 (𝑥 = 𝑦 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 𝑦) ∈ ℕ))
65imbi2d 230 . . 3 (𝑥 = 𝑦 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 𝑦) ∈ ℕ)))
7 oveq2 5930 . . . . 5 (𝑥 = (𝑦 + 1) → (𝐴 · 𝑥) = (𝐴 · (𝑦 + 1)))
87eleq1d 2265 . . . 4 (𝑥 = (𝑦 + 1) → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · (𝑦 + 1)) ∈ ℕ))
98imbi2d 230 . . 3 (𝑥 = (𝑦 + 1) → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · (𝑦 + 1)) ∈ ℕ)))
10 oveq2 5930 . . . . 5 (𝑥 = 𝐵 → (𝐴 · 𝑥) = (𝐴 · 𝐵))
1110eleq1d 2265 . . . 4 (𝑥 = 𝐵 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 𝐵) ∈ ℕ))
1211imbi2d 230 . . 3 (𝑥 = 𝐵 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 𝐵) ∈ ℕ)))
13 nncn 8998 . . . 4 (𝐴 ∈ ℕ → 𝐴 ∈ ℂ)
14 mulrid 8023 . . . . . 6 (𝐴 ∈ ℂ → (𝐴 · 1) = 𝐴)
1514eleq1d 2265 . . . . 5 (𝐴 ∈ ℂ → ((𝐴 · 1) ∈ ℕ ↔ 𝐴 ∈ ℕ))
1615biimprd 158 . . . 4 (𝐴 ∈ ℂ → (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ))
1713, 16mpcom 36 . . 3 (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ)
18 nnaddcl 9010 . . . . . . . 8 (((𝐴 · 𝑦) ∈ ℕ ∧ 𝐴 ∈ ℕ) → ((𝐴 · 𝑦) + 𝐴) ∈ ℕ)
1918ancoms 268 . . . . . . 7 ((𝐴 ∈ ℕ ∧ (𝐴 · 𝑦) ∈ ℕ) → ((𝐴 · 𝑦) + 𝐴) ∈ ℕ)
20 nncn 8998 . . . . . . . . 9 (𝑦 ∈ ℕ → 𝑦 ∈ ℂ)
21 ax-1cn 7972 . . . . . . . . . . 11 1 ∈ ℂ
22 adddi 8011 . . . . . . . . . . 11 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ ∧ 1 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + (𝐴 · 1)))
2321, 22mp3an3 1337 . . . . . . . . . 10 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + (𝐴 · 1)))
2414oveq2d 5938 . . . . . . . . . . 11 (𝐴 ∈ ℂ → ((𝐴 · 𝑦) + (𝐴 · 1)) = ((𝐴 · 𝑦) + 𝐴))
2524adantr 276 . . . . . . . . . 10 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → ((𝐴 · 𝑦) + (𝐴 · 1)) = ((𝐴 · 𝑦) + 𝐴))
2623, 25eqtrd 2229 . . . . . . . . 9 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + 𝐴))
2713, 20, 26syl2an 289 . . . . . . . 8 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + 𝐴))
2827eleq1d 2265 . . . . . . 7 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → ((𝐴 · (𝑦 + 1)) ∈ ℕ ↔ ((𝐴 · 𝑦) + 𝐴) ∈ ℕ))
2919, 28imbitrrid 156 . . . . . 6 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → ((𝐴 ∈ ℕ ∧ (𝐴 · 𝑦) ∈ ℕ) → (𝐴 · (𝑦 + 1)) ∈ ℕ))
3029exp4b 367 . . . . 5 (𝐴 ∈ ℕ → (𝑦 ∈ ℕ → (𝐴 ∈ ℕ → ((𝐴 · 𝑦) ∈ ℕ → (𝐴 · (𝑦 + 1)) ∈ ℕ))))
3130pm2.43b 52 . . . 4 (𝑦 ∈ ℕ → (𝐴 ∈ ℕ → ((𝐴 · 𝑦) ∈ ℕ → (𝐴 · (𝑦 + 1)) ∈ ℕ)))
3231a2d 26 . . 3 (𝑦 ∈ ℕ → ((𝐴 ∈ ℕ → (𝐴 · 𝑦) ∈ ℕ) → (𝐴 ∈ ℕ → (𝐴 · (𝑦 + 1)) ∈ ℕ)))
333, 6, 9, 12, 17, 32nnind 9006 . 2 (𝐵 ∈ ℕ → (𝐴 ∈ ℕ → (𝐴 · 𝐵) ∈ ℕ))
3433impcom 125 1 ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ) → (𝐴 · 𝐵) ∈ ℕ)
Colors of variables: wff set class
Syntax hints:  wi 4  wa 104   = wceq 1364  wcel 2167  (class class class)co 5922  cc 7877  1c1 7880   + caddc 7882   · cmul 7884  cn 8990
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-ia1 106  ax-ia2 107  ax-ia3 108  ax-io 710  ax-5 1461  ax-7 1462  ax-gen 1463  ax-ie1 1507  ax-ie2 1508  ax-8 1518  ax-10 1519  ax-11 1520  ax-i12 1521  ax-bndl 1523  ax-4 1524  ax-17 1540  ax-i9 1544  ax-ial 1548  ax-i5r 1549  ax-ext 2178  ax-sep 4151  ax-cnex 7970  ax-resscn 7971  ax-1cn 7972  ax-1re 7973  ax-icn 7974  ax-addcl 7975  ax-addrcl 7976  ax-mulcl 7977  ax-mulcom 7980  ax-addass 7981  ax-mulass 7982  ax-distr 7983  ax-1rid 7986  ax-cnre 7990
This theorem depends on definitions:  df-bi 117  df-3an 982  df-tru 1367  df-nf 1475  df-sb 1777  df-clab 2183  df-cleq 2189  df-clel 2192  df-nfc 2328  df-ral 2480  df-rex 2481  df-rab 2484  df-v 2765  df-un 3161  df-in 3163  df-ss 3170  df-sn 3628  df-pr 3629  df-op 3631  df-uni 3840  df-int 3875  df-br 4034  df-iota 5219  df-fv 5266  df-ov 5925  df-inn 8991
This theorem is referenced by:  nnmulcli  9012  nndivtr  9032  nnmulcld  9039  nn0mulcl  9285  qaddcl  9709  qmulcl  9711  modqmulnn  10434  nnexpcl  10644  nnsqcl  10701  faccl  10827  facdiv  10830  faclbnd3  10835  bcrpcl  10845  trirecip  11666  fprodnncl  11775  lcmgcdlem  12245  lcmgcdnn  12250  pcmptcl  12511  pcmpt  12512  4sqlem12  12571  mulgnnass  13287  lgseisenlem1  15311  lgseisenlem2  15312  lgseisenlem3  15313  lgseisenlem4  15314  lgsquadlem1  15318  lgsquadlem2  15319
  Copyright terms: Public domain W3C validator