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

Theorem naddov2 8700
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 8699 . 2 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +no 𝐵) = {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)})
2 snssi 4813 . . . . . . . . 9 (𝐴 ∈ On → {𝐴} ⊆ On)
3 onss 7788 . . . . . . . . 9 (𝐵 ∈ On → 𝐵 ⊆ On)
4 xpss12 5693 . . . . . . . . 9 (({𝐴} ⊆ On ∧ 𝐵 ⊆ On) → ({𝐴} × 𝐵) ⊆ (On × On))
52, 3, 4syl2an 594 . . . . . . . 8 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ({𝐴} × 𝐵) ⊆ (On × On))
6 naddfn 8696 . . . . . . . . 9 +no Fn (On × On)
76fndmi 6659 . . . . . . . 8 dom +no = (On × On)
85, 7sseqtrrdi 4028 . . . . . . 7 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ({𝐴} × 𝐵) ⊆ dom +no )
9 fnfun 6655 . . . . . . . . 9 ( +no Fn (On × On) → Fun +no )
106, 9ax-mp 5 . . . . . . . 8 Fun +no
11 funimassov 7598 . . . . . . . 8 ((Fun +no ∧ ({𝐴} × 𝐵) ⊆ dom +no ) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
1210, 11mpan 688 . . . . . . 7 (({𝐴} × 𝐵) ⊆ dom +no → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
138, 12syl 17 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
14 oveq1 7426 . . . . . . . . . 10 (𝑡 = 𝐴 → (𝑡 +no 𝑦) = (𝐴 +no 𝑦))
1514eleq1d 2810 . . . . . . . . 9 (𝑡 = 𝐴 → ((𝑡 +no 𝑦) ∈ 𝑥 ↔ (𝐴 +no 𝑦) ∈ 𝑥))
1615ralbidv 3167 . . . . . . . 8 (𝑡 = 𝐴 → (∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1716ralsng 4679 . . . . . . 7 (𝐴 ∈ On → (∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1817adantr 479 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1913, 18bitrd 278 . . . . 5 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
20 onss 7788 . . . . . . . . 9 (𝐴 ∈ On → 𝐴 ⊆ On)
21 snssi 4813 . . . . . . . . 9 (𝐵 ∈ On → {𝐵} ⊆ On)
22 xpss12 5693 . . . . . . . . 9 ((𝐴 ⊆ On ∧ {𝐵} ⊆ On) → (𝐴 × {𝐵}) ⊆ (On × On))
2320, 21, 22syl2an 594 . . . . . . . 8 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 × {𝐵}) ⊆ (On × On))
2423, 7sseqtrrdi 4028 . . . . . . 7 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 × {𝐵}) ⊆ dom +no )
25 funimassov 7598 . . . . . . . 8 ((Fun +no ∧ (𝐴 × {𝐵}) ⊆ dom +no ) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
2610, 25mpan 688 . . . . . . 7 ((𝐴 × {𝐵}) ⊆ dom +no → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
2724, 26syl 17 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
28 oveq2 7427 . . . . . . . . . 10 (𝑡 = 𝐵 → (𝑧 +no 𝑡) = (𝑧 +no 𝐵))
2928eleq1d 2810 . . . . . . . . 9 (𝑡 = 𝐵 → ((𝑧 +no 𝑡) ∈ 𝑥 ↔ (𝑧 +no 𝐵) ∈ 𝑥))
3029ralsng 4679 . . . . . . . 8 (𝐵 ∈ On → (∀𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ (𝑧 +no 𝐵) ∈ 𝑥))
3130ralbidv 3167 . . . . . . 7 (𝐵 ∈ On → (∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3231adantl 480 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3327, 32bitrd 278 . . . . 5 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3419, 33anbi12d 630 . . . 4 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ((( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥) ↔ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)))
3534rabbidv 3426 . . 3 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)} = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
3635inteqd 4955 . 2 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)} = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
371, 36eqtrd 2765 1 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +no 𝐵) = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 205  wa 394   = wceq 1533  wcel 2098  wral 3050  {crab 3418  wss 3944  {csn 4630   cint 4950   × cxp 5676  dom cdm 5678  cima 5681  Oncon0 6371  Fun wfun 6543   Fn wfn 6544  (class class class)co 7419   +no cnadd 8686
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1789  ax-4 1803  ax-5 1905  ax-6 1963  ax-7 2003  ax-8 2100  ax-9 2108  ax-10 2129  ax-11 2146  ax-12 2166  ax-ext 2696  ax-rep 5286  ax-sep 5300  ax-nul 5307  ax-pow 5365  ax-pr 5429  ax-un 7741
This theorem depends on definitions:  df-bi 206  df-an 395  df-or 846  df-3or 1085  df-3an 1086  df-tru 1536  df-fal 1546  df-ex 1774  df-nf 1778  df-sb 2060  df-mo 2528  df-eu 2557  df-clab 2703  df-cleq 2717  df-clel 2802  df-nfc 2877  df-ne 2930  df-ral 3051  df-rex 3060  df-reu 3364  df-rab 3419  df-v 3463  df-sbc 3774  df-csb 3890  df-dif 3947  df-un 3949  df-in 3951  df-ss 3961  df-pss 3964  df-nul 4323  df-if 4531  df-pw 4606  df-sn 4631  df-pr 4633  df-op 4637  df-uni 4910  df-int 4951  df-iun 4999  df-br 5150  df-opab 5212  df-mpt 5233  df-tr 5267  df-id 5576  df-eprel 5582  df-po 5590  df-so 5591  df-fr 5633  df-se 5634  df-we 5635  df-xp 5684  df-rel 5685  df-cnv 5686  df-co 5687  df-dm 5688  df-rn 5689  df-res 5690  df-ima 5691  df-pred 6307  df-ord 6374  df-on 6375  df-suc 6377  df-iota 6501  df-fun 6551  df-fn 6552  df-f 6553  df-f1 6554  df-fo 6555  df-f1o 6556  df-fv 6557  df-ov 7422  df-oprab 7423  df-mpo 7424  df-1st 7994  df-2nd 7995  df-frecs 8287  df-nadd 8687
This theorem is referenced by:  naddcom  8703  naddrid  8704  naddssim  8706  naddelim  8707  naddov4  42951  nadd1suc  42960  naddsuc2  42961
  Copyright terms: Public domain W3C validator