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

Theorem nnmulcl 9005
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 5927 . . . . 5 (𝑥 = 1 → (𝐴 · 𝑥) = (𝐴 · 1))
21eleq1d 2262 . . . 4 (𝑥 = 1 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 1) ∈ ℕ))
32imbi2d 230 . . 3 (𝑥 = 1 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ)))
4 oveq2 5927 . . . . 5 (𝑥 = 𝑦 → (𝐴 · 𝑥) = (𝐴 · 𝑦))
54eleq1d 2262 . . . 4 (𝑥 = 𝑦 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 𝑦) ∈ ℕ))
65imbi2d 230 . . 3 (𝑥 = 𝑦 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 𝑦) ∈ ℕ)))
7 oveq2 5927 . . . . 5 (𝑥 = (𝑦 + 1) → (𝐴 · 𝑥) = (𝐴 · (𝑦 + 1)))
87eleq1d 2262 . . . 4 (𝑥 = (𝑦 + 1) → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · (𝑦 + 1)) ∈ ℕ))
98imbi2d 230 . . 3 (𝑥 = (𝑦 + 1) → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · (𝑦 + 1)) ∈ ℕ)))
10 oveq2 5927 . . . . 5 (𝑥 = 𝐵 → (𝐴 · 𝑥) = (𝐴 · 𝐵))
1110eleq1d 2262 . . . 4 (𝑥 = 𝐵 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 𝐵) ∈ ℕ))
1211imbi2d 230 . . 3 (𝑥 = 𝐵 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 𝐵) ∈ ℕ)))
13 nncn 8992 . . . 4 (𝐴 ∈ ℕ → 𝐴 ∈ ℂ)
14 mulrid 8018 . . . . . 6 (𝐴 ∈ ℂ → (𝐴 · 1) = 𝐴)
1514eleq1d 2262 . . . . 5 (𝐴 ∈ ℂ → ((𝐴 · 1) ∈ ℕ ↔ 𝐴 ∈ ℕ))
1615biimprd 158 . . . 4 (𝐴 ∈ ℂ → (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ))
1713, 16mpcom 36 . . 3 (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ)
18 nnaddcl 9004 . . . . . . . 8 (((𝐴 · 𝑦) ∈ ℕ ∧ 𝐴 ∈ ℕ) → ((𝐴 · 𝑦) + 𝐴) ∈ ℕ)
1918ancoms 268 . . . . . . 7 ((𝐴 ∈ ℕ ∧ (𝐴 · 𝑦) ∈ ℕ) → ((𝐴 · 𝑦) + 𝐴) ∈ ℕ)
20 nncn 8992 . . . . . . . . 9 (𝑦 ∈ ℕ → 𝑦 ∈ ℂ)
21 ax-1cn 7967 . . . . . . . . . . 11 1 ∈ ℂ
22 adddi 8006 . . . . . . . . . . 11 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ ∧ 1 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + (𝐴 · 1)))
2321, 22mp3an3 1337 . . . . . . . . . 10 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + (𝐴 · 1)))
2414oveq2d 5935 . . . . . . . . . . 11 (𝐴 ∈ ℂ → ((𝐴 · 𝑦) + (𝐴 · 1)) = ((𝐴 · 𝑦) + 𝐴))
2524adantr 276 . . . . . . . . . 10 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → ((𝐴 · 𝑦) + (𝐴 · 1)) = ((𝐴 · 𝑦) + 𝐴))
2623, 25eqtrd 2226 . . . . . . . . 9 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + 𝐴))
2713, 20, 26syl2an 289 . . . . . . . 8 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + 𝐴))
2827eleq1d 2262 . . . . . . 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 9000 . 2 (𝐵 ∈ ℕ → (𝐴 ∈ ℕ → (𝐴 · 𝐵) ∈ ℕ))
3433impcom 125 1 ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ) → (𝐴 · 𝐵) ∈ ℕ)
Colors of variables: wff set class
Syntax hints:  wi 4  wa 104   = wceq 1364  wcel 2164  (class class class)co 5919  cc 7872  1c1 7875   + caddc 7877   · cmul 7879  cn 8984
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 1458  ax-7 1459  ax-gen 1460  ax-ie1 1504  ax-ie2 1505  ax-8 1515  ax-10 1516  ax-11 1517  ax-i12 1518  ax-bndl 1520  ax-4 1521  ax-17 1537  ax-i9 1541  ax-ial 1545  ax-i5r 1546  ax-ext 2175  ax-sep 4148  ax-cnex 7965  ax-resscn 7966  ax-1cn 7967  ax-1re 7968  ax-icn 7969  ax-addcl 7970  ax-addrcl 7971  ax-mulcl 7972  ax-mulcom 7975  ax-addass 7976  ax-mulass 7977  ax-distr 7978  ax-1rid 7981  ax-cnre 7985
This theorem depends on definitions:  df-bi 117  df-3an 982  df-tru 1367  df-nf 1472  df-sb 1774  df-clab 2180  df-cleq 2186  df-clel 2189  df-nfc 2325  df-ral 2477  df-rex 2478  df-rab 2481  df-v 2762  df-un 3158  df-in 3160  df-ss 3167  df-sn 3625  df-pr 3626  df-op 3628  df-uni 3837  df-int 3872  df-br 4031  df-iota 5216  df-fv 5263  df-ov 5922  df-inn 8985
This theorem is referenced by:  nnmulcli  9006  nndivtr  9026  nnmulcld  9033  nn0mulcl  9279  qaddcl  9703  qmulcl  9705  modqmulnn  10416  nnexpcl  10626  nnsqcl  10683  faccl  10809  facdiv  10812  faclbnd3  10817  bcrpcl  10827  trirecip  11647  fprodnncl  11756  lcmgcdlem  12218  lcmgcdnn  12223  pcmptcl  12483  pcmpt  12484  4sqlem12  12543  mulgnnass  13230  lgseisenlem1  15227  lgseisenlem2  15228  lgseisenlem3  15229  lgseisenlem4  15230  lgsquadlem1  15234  lgsquadlem2  15235
  Copyright terms: Public domain W3C validator