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

Theorem nnmulcl 8934
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 5878 . . . . 5 (𝑥 = 1 → (𝐴 · 𝑥) = (𝐴 · 1))
21eleq1d 2246 . . . 4 (𝑥 = 1 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 1) ∈ ℕ))
32imbi2d 230 . . 3 (𝑥 = 1 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ)))
4 oveq2 5878 . . . . 5 (𝑥 = 𝑦 → (𝐴 · 𝑥) = (𝐴 · 𝑦))
54eleq1d 2246 . . . 4 (𝑥 = 𝑦 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 𝑦) ∈ ℕ))
65imbi2d 230 . . 3 (𝑥 = 𝑦 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 𝑦) ∈ ℕ)))
7 oveq2 5878 . . . . 5 (𝑥 = (𝑦 + 1) → (𝐴 · 𝑥) = (𝐴 · (𝑦 + 1)))
87eleq1d 2246 . . . 4 (𝑥 = (𝑦 + 1) → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · (𝑦 + 1)) ∈ ℕ))
98imbi2d 230 . . 3 (𝑥 = (𝑦 + 1) → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · (𝑦 + 1)) ∈ ℕ)))
10 oveq2 5878 . . . . 5 (𝑥 = 𝐵 → (𝐴 · 𝑥) = (𝐴 · 𝐵))
1110eleq1d 2246 . . . 4 (𝑥 = 𝐵 → ((𝐴 · 𝑥) ∈ ℕ ↔ (𝐴 · 𝐵) ∈ ℕ))
1211imbi2d 230 . . 3 (𝑥 = 𝐵 → ((𝐴 ∈ ℕ → (𝐴 · 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 · 𝐵) ∈ ℕ)))
13 nncn 8921 . . . 4 (𝐴 ∈ ℕ → 𝐴 ∈ ℂ)
14 mulrid 7949 . . . . . 6 (𝐴 ∈ ℂ → (𝐴 · 1) = 𝐴)
1514eleq1d 2246 . . . . 5 (𝐴 ∈ ℂ → ((𝐴 · 1) ∈ ℕ ↔ 𝐴 ∈ ℕ))
1615biimprd 158 . . . 4 (𝐴 ∈ ℂ → (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ))
1713, 16mpcom 36 . . 3 (𝐴 ∈ ℕ → (𝐴 · 1) ∈ ℕ)
18 nnaddcl 8933 . . . . . . . 8 (((𝐴 · 𝑦) ∈ ℕ ∧ 𝐴 ∈ ℕ) → ((𝐴 · 𝑦) + 𝐴) ∈ ℕ)
1918ancoms 268 . . . . . . 7 ((𝐴 ∈ ℕ ∧ (𝐴 · 𝑦) ∈ ℕ) → ((𝐴 · 𝑦) + 𝐴) ∈ ℕ)
20 nncn 8921 . . . . . . . . 9 (𝑦 ∈ ℕ → 𝑦 ∈ ℂ)
21 ax-1cn 7899 . . . . . . . . . . 11 1 ∈ ℂ
22 adddi 7938 . . . . . . . . . . 11 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ ∧ 1 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + (𝐴 · 1)))
2321, 22mp3an3 1326 . . . . . . . . . 10 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + (𝐴 · 1)))
2414oveq2d 5886 . . . . . . . . . . 11 (𝐴 ∈ ℂ → ((𝐴 · 𝑦) + (𝐴 · 1)) = ((𝐴 · 𝑦) + 𝐴))
2524adantr 276 . . . . . . . . . 10 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → ((𝐴 · 𝑦) + (𝐴 · 1)) = ((𝐴 · 𝑦) + 𝐴))
2623, 25eqtrd 2210 . . . . . . . . 9 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + 𝐴))
2713, 20, 26syl2an 289 . . . . . . . 8 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → (𝐴 · (𝑦 + 1)) = ((𝐴 · 𝑦) + 𝐴))
2827eleq1d 2246 . . . . . . 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 8929 . 2 (𝐵 ∈ ℕ → (𝐴 ∈ ℕ → (𝐴 · 𝐵) ∈ ℕ))
3433impcom 125 1 ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ) → (𝐴 · 𝐵) ∈ ℕ)
Colors of variables: wff set class
Syntax hints:  wi 4  wa 104   = wceq 1353  wcel 2148  (class class class)co 5870  cc 7804  1c1 7807   + caddc 7809   · cmul 7811  cn 8913
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 709  ax-5 1447  ax-7 1448  ax-gen 1449  ax-ie1 1493  ax-ie2 1494  ax-8 1504  ax-10 1505  ax-11 1506  ax-i12 1507  ax-bndl 1509  ax-4 1510  ax-17 1526  ax-i9 1530  ax-ial 1534  ax-i5r 1535  ax-ext 2159  ax-sep 4119  ax-cnex 7897  ax-resscn 7898  ax-1cn 7899  ax-1re 7900  ax-icn 7901  ax-addcl 7902  ax-addrcl 7903  ax-mulcl 7904  ax-mulcom 7907  ax-addass 7908  ax-mulass 7909  ax-distr 7910  ax-1rid 7913  ax-cnre 7917
This theorem depends on definitions:  df-bi 117  df-3an 980  df-tru 1356  df-nf 1461  df-sb 1763  df-clab 2164  df-cleq 2170  df-clel 2173  df-nfc 2308  df-ral 2460  df-rex 2461  df-rab 2464  df-v 2739  df-un 3133  df-in 3135  df-ss 3142  df-sn 3598  df-pr 3599  df-op 3601  df-uni 3809  df-int 3844  df-br 4002  df-iota 5175  df-fv 5221  df-ov 5873  df-inn 8914
This theorem is referenced by:  nnmulcli  8935  nndivtr  8955  nnmulcld  8962  nn0mulcl  9206  qaddcl  9629  qmulcl  9631  modqmulnn  10335  nnexpcl  10526  nnsqcl  10582  faccl  10706  facdiv  10709  faclbnd3  10714  bcrpcl  10724  trirecip  11500  fprodnncl  11609  lcmgcdlem  12067  lcmgcdnn  12072  pcmptcl  12330  pcmpt  12331  mulgnnass  12945
  Copyright terms: Public domain W3C validator