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

Theorem nnaddcl 8877
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 5850 . . . . 5 (𝑥 = 1 → (𝐴 + 𝑥) = (𝐴 + 1))
21eleq1d 2235 . . . 4 (𝑥 = 1 → ((𝐴 + 𝑥) ∈ ℕ ↔ (𝐴 + 1) ∈ ℕ))
32imbi2d 229 . . 3 (𝑥 = 1 → ((𝐴 ∈ ℕ → (𝐴 + 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 + 1) ∈ ℕ)))
4 oveq2 5850 . . . . 5 (𝑥 = 𝑦 → (𝐴 + 𝑥) = (𝐴 + 𝑦))
54eleq1d 2235 . . . 4 (𝑥 = 𝑦 → ((𝐴 + 𝑥) ∈ ℕ ↔ (𝐴 + 𝑦) ∈ ℕ))
65imbi2d 229 . . 3 (𝑥 = 𝑦 → ((𝐴 ∈ ℕ → (𝐴 + 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 + 𝑦) ∈ ℕ)))
7 oveq2 5850 . . . . 5 (𝑥 = (𝑦 + 1) → (𝐴 + 𝑥) = (𝐴 + (𝑦 + 1)))
87eleq1d 2235 . . . 4 (𝑥 = (𝑦 + 1) → ((𝐴 + 𝑥) ∈ ℕ ↔ (𝐴 + (𝑦 + 1)) ∈ ℕ))
98imbi2d 229 . . 3 (𝑥 = (𝑦 + 1) → ((𝐴 ∈ ℕ → (𝐴 + 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 + (𝑦 + 1)) ∈ ℕ)))
10 oveq2 5850 . . . . 5 (𝑥 = 𝐵 → (𝐴 + 𝑥) = (𝐴 + 𝐵))
1110eleq1d 2235 . . . 4 (𝑥 = 𝐵 → ((𝐴 + 𝑥) ∈ ℕ ↔ (𝐴 + 𝐵) ∈ ℕ))
1211imbi2d 229 . . 3 (𝑥 = 𝐵 → ((𝐴 ∈ ℕ → (𝐴 + 𝑥) ∈ ℕ) ↔ (𝐴 ∈ ℕ → (𝐴 + 𝐵) ∈ ℕ)))
13 peano2nn 8869 . . 3 (𝐴 ∈ ℕ → (𝐴 + 1) ∈ ℕ)
14 peano2nn 8869 . . . . . 6 ((𝐴 + 𝑦) ∈ ℕ → ((𝐴 + 𝑦) + 1) ∈ ℕ)
15 nncn 8865 . . . . . . . 8 (𝐴 ∈ ℕ → 𝐴 ∈ ℂ)
16 nncn 8865 . . . . . . . 8 (𝑦 ∈ ℕ → 𝑦 ∈ ℂ)
17 ax-1cn 7846 . . . . . . . . 9 1 ∈ ℂ
18 addass 7883 . . . . . . . . 9 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ ∧ 1 ∈ ℂ) → ((𝐴 + 𝑦) + 1) = (𝐴 + (𝑦 + 1)))
1917, 18mp3an3 1316 . . . . . . . 8 ((𝐴 ∈ ℂ ∧ 𝑦 ∈ ℂ) → ((𝐴 + 𝑦) + 1) = (𝐴 + (𝑦 + 1)))
2015, 16, 19syl2an 287 . . . . . . 7 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → ((𝐴 + 𝑦) + 1) = (𝐴 + (𝑦 + 1)))
2120eleq1d 2235 . . . . . 6 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → (((𝐴 + 𝑦) + 1) ∈ ℕ ↔ (𝐴 + (𝑦 + 1)) ∈ ℕ))
2214, 21syl5ib 153 . . . . 5 ((𝐴 ∈ ℕ ∧ 𝑦 ∈ ℕ) → ((𝐴 + 𝑦) ∈ ℕ → (𝐴 + (𝑦 + 1)) ∈ ℕ))
2322expcom 115 . . . 4 (𝑦 ∈ ℕ → (𝐴 ∈ ℕ → ((𝐴 + 𝑦) ∈ ℕ → (𝐴 + (𝑦 + 1)) ∈ ℕ)))
2423a2d 26 . . 3 (𝑦 ∈ ℕ → ((𝐴 ∈ ℕ → (𝐴 + 𝑦) ∈ ℕ) → (𝐴 ∈ ℕ → (𝐴 + (𝑦 + 1)) ∈ ℕ)))
253, 6, 9, 12, 13, 24nnind 8873 . 2 (𝐵 ∈ ℕ → (𝐴 ∈ ℕ → (𝐴 + 𝐵) ∈ ℕ))
2625impcom 124 1 ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ) → (𝐴 + 𝐵) ∈ ℕ)
Colors of variables: wff set class
Syntax hints:  wi 4  wa 103   = wceq 1343  wcel 2136  (class class class)co 5842  cc 7751  1c1 7754   + caddc 7756  cn 8857
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-ia1 105  ax-ia2 106  ax-ia3 107  ax-io 699  ax-5 1435  ax-7 1436  ax-gen 1437  ax-ie1 1481  ax-ie2 1482  ax-8 1492  ax-10 1493  ax-11 1494  ax-i12 1495  ax-bndl 1497  ax-4 1498  ax-17 1514  ax-i9 1518  ax-ial 1522  ax-i5r 1523  ax-ext 2147  ax-sep 4100  ax-cnex 7844  ax-resscn 7845  ax-1cn 7846  ax-1re 7847  ax-addrcl 7850  ax-addass 7855
This theorem depends on definitions:  df-bi 116  df-3an 970  df-tru 1346  df-nf 1449  df-sb 1751  df-clab 2152  df-cleq 2158  df-clel 2161  df-nfc 2297  df-ral 2449  df-rex 2450  df-rab 2453  df-v 2728  df-un 3120  df-in 3122  df-ss 3129  df-sn 3582  df-pr 3583  df-op 3585  df-uni 3790  df-int 3825  df-br 3983  df-iota 5153  df-fv 5196  df-ov 5845  df-inn 8858
This theorem is referenced by:  nnmulcl  8878  nn2ge  8890  nnaddcld  8905  nnnn0addcl  9144  nn0addcl  9149  9p1e10  9324  pythagtriplem4  12200
  Copyright terms: Public domain W3C validator