MPE Home Metamath Proof Explorer < Previous   Next >
Nearby theorems
Mirrors  >  Home  >  MPE Home  >  Th. List  >  naddov2 Structured version   Visualization version   GIF version

Theorem naddov2 8722
Description: Alternate expression for natural addition. (Contributed by Scott Fenton, 26-Aug-2024.)
Assertion
Ref Expression
naddov2 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +no 𝐵) = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
Distinct variable groups:   𝑥,𝐴   𝑥,𝐵   𝑦,𝐴   𝑧,𝐴   𝑦,𝐵   𝑧,𝐵   𝑥,𝑦   𝑥,𝑧

Proof of Theorem naddov2
Dummy variable 𝑡 is distinct from all other variables.
StepHypRef Expression
1 naddov 8721 . 2 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +no 𝐵) = {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)})
2 snssi 4814 . . . . . . . . 9 (𝐴 ∈ On → {𝐴} ⊆ On)
3 onss 7808 . . . . . . . . 9 (𝐵 ∈ On → 𝐵 ⊆ On)
4 xpss12 5705 . . . . . . . . 9 (({𝐴} ⊆ On ∧ 𝐵 ⊆ On) → ({𝐴} × 𝐵) ⊆ (On × On))
52, 3, 4syl2an 596 . . . . . . . 8 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ({𝐴} × 𝐵) ⊆ (On × On))
6 naddfn 8718 . . . . . . . . 9 +no Fn (On × On)
76fndmi 6677 . . . . . . . 8 dom +no = (On × On)
85, 7sseqtrrdi 4048 . . . . . . 7 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ({𝐴} × 𝐵) ⊆ dom +no )
9 fnfun 6673 . . . . . . . . 9 ( +no Fn (On × On) → Fun +no )
106, 9ax-mp 5 . . . . . . . 8 Fun +no
11 funimassov 7614 . . . . . . . 8 ((Fun +no ∧ ({𝐴} × 𝐵) ⊆ dom +no ) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
1210, 11mpan 690 . . . . . . 7 (({𝐴} × 𝐵) ⊆ dom +no → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
138, 12syl 17 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
14 oveq1 7442 . . . . . . . . . 10 (𝑡 = 𝐴 → (𝑡 +no 𝑦) = (𝐴 +no 𝑦))
1514eleq1d 2825 . . . . . . . . 9 (𝑡 = 𝐴 → ((𝑡 +no 𝑦) ∈ 𝑥 ↔ (𝐴 +no 𝑦) ∈ 𝑥))
1615ralbidv 3177 . . . . . . . 8 (𝑡 = 𝐴 → (∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1716ralsng 4681 . . . . . . 7 (𝐴 ∈ On → (∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1817adantr 480 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1913, 18bitrd 279 . . . . 5 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
20 onss 7808 . . . . . . . . 9 (𝐴 ∈ On → 𝐴 ⊆ On)
21 snssi 4814 . . . . . . . . 9 (𝐵 ∈ On → {𝐵} ⊆ On)
22 xpss12 5705 . . . . . . . . 9 ((𝐴 ⊆ On ∧ {𝐵} ⊆ On) → (𝐴 × {𝐵}) ⊆ (On × On))
2320, 21, 22syl2an 596 . . . . . . . 8 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 × {𝐵}) ⊆ (On × On))
2423, 7sseqtrrdi 4048 . . . . . . 7 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 × {𝐵}) ⊆ dom +no )
25 funimassov 7614 . . . . . . . 8 ((Fun +no ∧ (𝐴 × {𝐵}) ⊆ dom +no ) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
2610, 25mpan 690 . . . . . . 7 ((𝐴 × {𝐵}) ⊆ dom +no → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
2724, 26syl 17 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
28 oveq2 7443 . . . . . . . . . 10 (𝑡 = 𝐵 → (𝑧 +no 𝑡) = (𝑧 +no 𝐵))
2928eleq1d 2825 . . . . . . . . 9 (𝑡 = 𝐵 → ((𝑧 +no 𝑡) ∈ 𝑥 ↔ (𝑧 +no 𝐵) ∈ 𝑥))
3029ralsng 4681 . . . . . . . 8 (𝐵 ∈ On → (∀𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ (𝑧 +no 𝐵) ∈ 𝑥))
3130ralbidv 3177 . . . . . . 7 (𝐵 ∈ On → (∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3231adantl 481 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3327, 32bitrd 279 . . . . 5 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3419, 33anbi12d 632 . . . 4 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ((( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥) ↔ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)))
3534rabbidv 3442 . . 3 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)} = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
3635inteqd 4957 . 2 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)} = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
371, 36eqtrd 2776 1 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +no 𝐵) = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 206  wa 395   = wceq 1538  wcel 2107  wral 3060  {crab 3434  wss 3964  {csn 4632   cint 4952   × cxp 5688  dom cdm 5690  cima 5693  Oncon0 6389  Fun wfun 6560   Fn wfn 6561  (class class class)co 7435   +no cnadd 8708
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1793  ax-4 1807  ax-5 1909  ax-6 1966  ax-7 2006  ax-8 2109  ax-9 2117  ax-10 2140  ax-11 2156  ax-12 2176  ax-ext 2707  ax-rep 5286  ax-sep 5303  ax-nul 5313  ax-pow 5372  ax-pr 5439  ax-un 7758
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 848  df-3or 1087  df-3an 1088  df-tru 1541  df-fal 1551  df-ex 1778  df-nf 1782  df-sb 2064  df-mo 2539  df-eu 2568  df-clab 2714  df-cleq 2728  df-clel 2815  df-nfc 2891  df-ne 2940  df-ral 3061  df-rex 3070  df-reu 3380  df-rab 3435  df-v 3481  df-sbc 3793  df-csb 3910  df-dif 3967  df-un 3969  df-in 3971  df-ss 3981  df-pss 3984  df-nul 4341  df-if 4533  df-pw 4608  df-sn 4633  df-pr 4635  df-op 4639  df-uni 4914  df-int 4953  df-iun 4999  df-br 5150  df-opab 5212  df-mpt 5233  df-tr 5267  df-id 5584  df-eprel 5590  df-po 5598  df-so 5599  df-fr 5642  df-se 5643  df-we 5644  df-xp 5696  df-rel 5697  df-cnv 5698  df-co 5699  df-dm 5700  df-rn 5701  df-res 5702  df-ima 5703  df-pred 6326  df-ord 6392  df-on 6393  df-suc 6395  df-iota 6519  df-fun 6568  df-fn 6569  df-f 6570  df-f1 6571  df-fo 6572  df-f1o 6573  df-fv 6574  df-ov 7438  df-oprab 7439  df-mpo 7440  df-1st 8019  df-2nd 8020  df-frecs 8311  df-nadd 8709
This theorem is referenced by:  naddcom  8725  naddrid  8726  naddssim  8728  naddelim  8729  naddsuc2  8744  naddov4  43387  nadd1suc  43396
  Copyright terms: Public domain W3C validator