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

Theorem naddov2 8737
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 8736 . 2 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +no 𝐵) = {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)})
2 snssi 4833 . . . . . . . . 9 (𝐴 ∈ On → {𝐴} ⊆ On)
3 onss 7822 . . . . . . . . 9 (𝐵 ∈ On → 𝐵 ⊆ On)
4 xpss12 5715 . . . . . . . . 9 (({𝐴} ⊆ On ∧ 𝐵 ⊆ On) → ({𝐴} × 𝐵) ⊆ (On × On))
52, 3, 4syl2an 595 . . . . . . . 8 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ({𝐴} × 𝐵) ⊆ (On × On))
6 naddfn 8733 . . . . . . . . 9 +no Fn (On × On)
76fndmi 6685 . . . . . . . 8 dom +no = (On × On)
85, 7sseqtrrdi 4060 . . . . . . 7 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ({𝐴} × 𝐵) ⊆ dom +no )
9 fnfun 6681 . . . . . . . . 9 ( +no Fn (On × On) → Fun +no )
106, 9ax-mp 5 . . . . . . . 8 Fun +no
11 funimassov 7629 . . . . . . . 8 ((Fun +no ∧ ({𝐴} × 𝐵) ⊆ dom +no ) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
1210, 11mpan 689 . . . . . . 7 (({𝐴} × 𝐵) ⊆ dom +no → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
138, 12syl 17 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥))
14 oveq1 7457 . . . . . . . . . 10 (𝑡 = 𝐴 → (𝑡 +no 𝑦) = (𝐴 +no 𝑦))
1514eleq1d 2829 . . . . . . . . 9 (𝑡 = 𝐴 → ((𝑡 +no 𝑦) ∈ 𝑥 ↔ (𝐴 +no 𝑦) ∈ 𝑥))
1615ralbidv 3184 . . . . . . . 8 (𝑡 = 𝐴 → (∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1716ralsng 4697 . . . . . . 7 (𝐴 ∈ On → (∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1817adantr 480 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (∀𝑡 ∈ {𝐴}∀𝑦𝐵 (𝑡 +no 𝑦) ∈ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
1913, 18bitrd 279 . . . . 5 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ↔ ∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥))
20 onss 7822 . . . . . . . . 9 (𝐴 ∈ On → 𝐴 ⊆ On)
21 snssi 4833 . . . . . . . . 9 (𝐵 ∈ On → {𝐵} ⊆ On)
22 xpss12 5715 . . . . . . . . 9 ((𝐴 ⊆ On ∧ {𝐵} ⊆ On) → (𝐴 × {𝐵}) ⊆ (On × On))
2320, 21, 22syl2an 595 . . . . . . . 8 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 × {𝐵}) ⊆ (On × On))
2423, 7sseqtrrdi 4060 . . . . . . 7 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 × {𝐵}) ⊆ dom +no )
25 funimassov 7629 . . . . . . . 8 ((Fun +no ∧ (𝐴 × {𝐵}) ⊆ dom +no ) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
2610, 25mpan 689 . . . . . . 7 ((𝐴 × {𝐵}) ⊆ dom +no → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
2724, 26syl 17 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥))
28 oveq2 7458 . . . . . . . . . 10 (𝑡 = 𝐵 → (𝑧 +no 𝑡) = (𝑧 +no 𝐵))
2928eleq1d 2829 . . . . . . . . 9 (𝑡 = 𝐵 → ((𝑧 +no 𝑡) ∈ 𝑥 ↔ (𝑧 +no 𝐵) ∈ 𝑥))
3029ralsng 4697 . . . . . . . 8 (𝐵 ∈ On → (∀𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ (𝑧 +no 𝐵) ∈ 𝑥))
3130ralbidv 3184 . . . . . . 7 (𝐵 ∈ On → (∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3231adantl 481 . . . . . 6 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (∀𝑧𝐴𝑡 ∈ {𝐵} (𝑧 +no 𝑡) ∈ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3327, 32bitrd 279 . . . . 5 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (( +no “ (𝐴 × {𝐵})) ⊆ 𝑥 ↔ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥))
3419, 33anbi12d 631 . . . 4 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → ((( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥) ↔ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)))
3534rabbidv 3451 . . 3 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)} = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
3635inteqd 4975 . 2 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → {𝑥 ∈ On ∣ (( +no “ ({𝐴} × 𝐵)) ⊆ 𝑥 ∧ ( +no “ (𝐴 × {𝐵})) ⊆ 𝑥)} = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
371, 36eqtrd 2780 1 ((𝐴 ∈ On ∧ 𝐵 ∈ On) → (𝐴 +no 𝐵) = {𝑥 ∈ On ∣ (∀𝑦𝐵 (𝐴 +no 𝑦) ∈ 𝑥 ∧ ∀𝑧𝐴 (𝑧 +no 𝐵) ∈ 𝑥)})
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 206  wa 395   = wceq 1537  wcel 2108  wral 3067  {crab 3443  wss 3976  {csn 4648   cint 4970   × cxp 5698  dom cdm 5700  cima 5703  Oncon0 6397  Fun wfun 6569   Fn wfn 6570  (class class class)co 7450   +no cnadd 8723
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 1967  ax-7 2007  ax-8 2110  ax-9 2118  ax-10 2141  ax-11 2158  ax-12 2178  ax-ext 2711  ax-rep 5303  ax-sep 5317  ax-nul 5324  ax-pow 5383  ax-pr 5447  ax-un 7772
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 847  df-3or 1088  df-3an 1089  df-tru 1540  df-fal 1550  df-ex 1778  df-nf 1782  df-sb 2065  df-mo 2543  df-eu 2572  df-clab 2718  df-cleq 2732  df-clel 2819  df-nfc 2895  df-ne 2947  df-ral 3068  df-rex 3077  df-reu 3389  df-rab 3444  df-v 3490  df-sbc 3805  df-csb 3922  df-dif 3979  df-un 3981  df-in 3983  df-ss 3993  df-pss 3996  df-nul 4353  df-if 4549  df-pw 4624  df-sn 4649  df-pr 4651  df-op 4655  df-uni 4932  df-int 4971  df-iun 5017  df-br 5167  df-opab 5229  df-mpt 5250  df-tr 5284  df-id 5593  df-eprel 5599  df-po 5607  df-so 5608  df-fr 5652  df-se 5653  df-we 5654  df-xp 5706  df-rel 5707  df-cnv 5708  df-co 5709  df-dm 5710  df-rn 5711  df-res 5712  df-ima 5713  df-pred 6334  df-ord 6400  df-on 6401  df-suc 6403  df-iota 6527  df-fun 6577  df-fn 6578  df-f 6579  df-f1 6580  df-fo 6581  df-f1o 6582  df-fv 6583  df-ov 7453  df-oprab 7454  df-mpo 7455  df-1st 8032  df-2nd 8033  df-frecs 8324  df-nadd 8724
This theorem is referenced by:  naddcom  8740  naddrid  8741  naddssim  8743  naddelim  8744  naddsuc2  8759  naddov4  43347  nadd1suc  43356
  Copyright terms: Public domain W3C validator