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

Theorem nnaddcl 8059
Description: Closure of addition of positive integers, proved by induction on the second addend. (Contributed by NM, 12-Jan-1997.)
Assertion
Ref Expression
nnaddcl ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ) → (𝐴 + 𝐵) ∈ ℕ)

Proof of Theorem nnaddcl
Dummy variables 𝑥 𝑦 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 oveq2 5540 . . . . 5 (𝑥 = 1 → (𝐴 + 𝑥) = (𝐴 + 1))
21eleq1d 2147 . . . 4 (𝑥 = 1 → ((𝐴 + 𝑥) ∈ ℕ ↔ (𝐴 + 1) ∈ ℕ))
32imbi2d 228 . . 3 (𝑥 = 1 → ((𝐴 ∈ ℕ → (𝐴 + 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 + 1) ∈ ℕ)))
4 oveq2 5540 . . . . 5 (𝑥 = 𝑦 → (𝐴 + 𝑥) = (𝐴 + 𝑦))
54eleq1d 2147 . . . 4 (𝑥 = 𝑦 → ((𝐴 + 𝑥) ∈ ℕ ↔ (𝐴 + 𝑦) ∈ ℕ))
65imbi2d 228 . . 3 (𝑥 = 𝑦 → ((𝐴 ∈ ℕ → (𝐴 + 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 + 𝑦) ∈ ℕ)))
7 oveq2 5540 . . . . 5 (𝑥 = (𝑦 + 1) → (𝐴 + 𝑥) = (𝐴 + (𝑦 + 1)))
87eleq1d 2147 . . . 4 (𝑥 = (𝑦 + 1) → ((𝐴 + 𝑥) ∈ ℕ ↔ (𝐴 + (𝑦 + 1)) ∈ ℕ))
98imbi2d 228 . . 3 (𝑥 = (𝑦 + 1) → ((𝐴 ∈ ℕ → (𝐴 + 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 + (𝑦 + 1)) ∈ ℕ)))
10 oveq2 5540 . . . . 5 (𝑥 = 𝐵 → (𝐴 + 𝑥) = (𝐴 + 𝐵))
1110eleq1d 2147 . . . 4 (𝑥 = 𝐵 → ((𝐴 + 𝑥) ∈ ℕ ↔ (𝐴 + 𝐵) ∈ ℕ))
1211imbi2d 228 . . 3 (𝑥 = 𝐵 → ((𝐴 ∈ ℕ → (𝐴 + 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 + 𝐵) ∈ ℕ)))
13 peano2nn 8051 . . 3 (𝐴 ∈ ℕ → (𝐴 + 1) ∈ ℕ)
14 peano2nn 8051 . . . . . 6 ((𝐴 + 𝑦) ∈ ℕ → ((𝐴 + 𝑦) + 1) ∈ ℕ)
15 nncn 8047 . . . . . . . 8 (𝐴 ∈ ℕ → 𝐴 ∈ ℂ)
16 nncn 8047 . . . . . . . 8 (𝑦 ∈ ℕ → 𝑦 ∈ ℂ)
17 ax-1cn 7069 . . . . . . . . 9 1 ∈ ℂ
18 addass 7103 . . . . . . . . 9 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ ∧ 1 ∈ ℂ) → ((𝐴 + 𝑦) + 1) = (𝐴 + (𝑦 + 1)))
1917, 18mp3an3 1257 . . . . . . . 8 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → ((𝐴 + 𝑦) + 1) = (𝐴 + (𝑦 + 1)))
2015, 16, 19syl2an 283 . . . . . . 7 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → ((𝐴 + 𝑦) + 1) = (𝐴 + (𝑦 + 1)))
2120eleq1d 2147 . . . . . 6 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → (((𝐴 + 𝑦) + 1) ∈ ℕ ↔ (𝐴 + (𝑦 + 1)) ∈ ℕ))
2214, 21syl5ib 152 . . . . 5 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → ((𝐴 + 𝑦) ∈ ℕ → (𝐴 + (𝑦 + 1)) ∈ ℕ))
2322expcom 114 . . . 4 (𝑦 ∈ ℕ → (𝐴 ∈ ℕ → ((𝐴 + 𝑦) ∈ ℕ → (𝐴 + (𝑦 + 1)) ∈ ℕ)))
2423a2d 26 . . 3 (𝑦 ∈ ℕ → ((𝐴 ∈ ℕ → (𝐴 + 𝑦) ∈ ℕ) → (𝐴 ∈ ℕ → (𝐴 + (𝑦 + 1)) ∈ ℕ)))
253, 6, 9, 12, 13, 24nnind 8055 . 2 (𝐵 ∈ ℕ → (𝐴 ∈ ℕ → (𝐴 + 𝐵) ∈ ℕ))
2625impcom 123 1 ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ) → (𝐴 + 𝐵) ∈ ℕ)
Colors of variables: wff set class
Syntax hints:  wi 4  wa 102   = wceq 1284  wcel 1433  (class class class)co 5532  cc 6979  1c1 6982   + caddc 6984  cn 8039
This theorem was proved from axioms:  ax-1 5  ax-2 6  ax-mp 7  ax-ia1 104  ax-ia2 105  ax-ia3 106  ax-io 662  ax-5 1376  ax-7 1377  ax-gen 1378  ax-ie1 1422  ax-ie2 1423  ax-8 1435  ax-10 1436  ax-11 1437  ax-i12 1438  ax-bndl 1439  ax-4 1440  ax-17 1459  ax-i9 1463  ax-ial 1467  ax-i5r 1468  ax-ext 2063  ax-sep 3896  ax-cnex 7067  ax-resscn 7068  ax-1cn 7069  ax-1re 7070  ax-addrcl 7073  ax-addass 7078
This theorem depends on definitions:  df-bi 115  df-3an 921  df-tru 1287  df-nf 1390  df-sb 1686  df-clab 2068  df-cleq 2074  df-clel 2077  df-nfc 2208  df-ral 2353  df-rex 2354  df-rab 2357  df-v 2603  df-un 2977  df-in 2979  df-ss 2986  df-sn 3404  df-pr 3405  df-op 3407  df-uni 3602  df-int 3637  df-br 3786  df-iota 4887  df-fv 4930  df-ov 5535  df-inn 8040
This theorem is referenced by:  nnmulcl  8060  nn2ge  8071  nnaddcld  8086  nnnn0addcl  8318  nn0addcl  8323  9p1e10  8479
  Copyright terms: Public domain W3C validator