Users' Mathboxes Mathbox for ML < Previous   Next >
Nearby theorems
Mirrors  >  Home  >  MPE Home  >  Th. List  >   Mathboxes  >  finxpreclem3 Structured version   Visualization version   GIF version

Theorem finxpreclem3 37388
Description: Lemma for ↑↑ recursion theorems. (Contributed by ML, 20-Oct-2020.)
Hypothesis
Ref Expression
finxpreclem3.1 𝐹 = (𝑛 ∈ ω, 𝑥 ∈ V ↦ if((𝑛 = 1o𝑥𝑈), ∅, if(𝑥 ∈ (V × 𝑈), ⟨ 𝑛, (1st𝑥)⟩, ⟨𝑛, 𝑥⟩)))
Assertion
Ref Expression
finxpreclem3 (((𝑁 ∈ ω ∧ 2o𝑁) ∧ 𝑋 ∈ (V × 𝑈)) → ⟨ 𝑁, (1st𝑋)⟩ = (𝐹‘⟨𝑁, 𝑋⟩))
Distinct variable groups:   𝑛,𝑁,𝑥   𝑈,𝑛,𝑥   𝑛,𝑋,𝑥
Allowed substitution hints:   𝐹(𝑥,𝑛)

Proof of Theorem finxpreclem3
StepHypRef Expression
1 finxpreclem3.1 . . . 4 𝐹 = (𝑛 ∈ ω, 𝑥 ∈ V ↦ if((𝑛 = 1o𝑥𝑈), ∅, if(𝑥 ∈ (V × 𝑈), ⟨ 𝑛, (1st𝑥)⟩, ⟨𝑛, 𝑥⟩)))
21a1i 11 . . 3 (((𝑁 ∈ ω ∧ 2o𝑁) ∧ 𝑋 ∈ (V × 𝑈)) → 𝐹 = (𝑛 ∈ ω, 𝑥 ∈ V ↦ if((𝑛 = 1o𝑥𝑈), ∅, if(𝑥 ∈ (V × 𝑈), ⟨ 𝑛, (1st𝑥)⟩, ⟨𝑛, 𝑥⟩))))
3 eqeq1 2734 . . . . . . 7 (𝑛 = 𝑁 → (𝑛 = 1o𝑁 = 1o))
4 eleq1 2817 . . . . . . 7 (𝑥 = 𝑋 → (𝑥𝑈𝑋𝑈))
53, 4bi2anan9 638 . . . . . 6 ((𝑛 = 𝑁𝑥 = 𝑋) → ((𝑛 = 1o𝑥𝑈) ↔ (𝑁 = 1o𝑋𝑈)))
6 eleq1 2817 . . . . . . . 8 (𝑥 = 𝑋 → (𝑥 ∈ (V × 𝑈) ↔ 𝑋 ∈ (V × 𝑈)))
76adantl 481 . . . . . . 7 ((𝑛 = 𝑁𝑥 = 𝑋) → (𝑥 ∈ (V × 𝑈) ↔ 𝑋 ∈ (V × 𝑈)))
8 unieq 4885 . . . . . . . . 9 (𝑛 = 𝑁 𝑛 = 𝑁)
98adantr 480 . . . . . . . 8 ((𝑛 = 𝑁𝑥 = 𝑋) → 𝑛 = 𝑁)
10 fveq2 6861 . . . . . . . . 9 (𝑥 = 𝑋 → (1st𝑥) = (1st𝑋))
1110adantl 481 . . . . . . . 8 ((𝑛 = 𝑁𝑥 = 𝑋) → (1st𝑥) = (1st𝑋))
129, 11opeq12d 4848 . . . . . . 7 ((𝑛 = 𝑁𝑥 = 𝑋) → ⟨ 𝑛, (1st𝑥)⟩ = ⟨ 𝑁, (1st𝑋)⟩)
13 opeq12 4842 . . . . . . 7 ((𝑛 = 𝑁𝑥 = 𝑋) → ⟨𝑛, 𝑥⟩ = ⟨𝑁, 𝑋⟩)
147, 12, 13ifbieq12d 4520 . . . . . 6 ((𝑛 = 𝑁𝑥 = 𝑋) → if(𝑥 ∈ (V × 𝑈), ⟨ 𝑛, (1st𝑥)⟩, ⟨𝑛, 𝑥⟩) = if(𝑋 ∈ (V × 𝑈), ⟨ 𝑁, (1st𝑋)⟩, ⟨𝑁, 𝑋⟩))
155, 14ifbieq2d 4518 . . . . 5 ((𝑛 = 𝑁𝑥 = 𝑋) → if((𝑛 = 1o𝑥𝑈), ∅, if(𝑥 ∈ (V × 𝑈), ⟨ 𝑛, (1st𝑥)⟩, ⟨𝑛, 𝑥⟩)) = if((𝑁 = 1o𝑋𝑈), ∅, if(𝑋 ∈ (V × 𝑈), ⟨ 𝑁, (1st𝑋)⟩, ⟨𝑁, 𝑋⟩)))
16 sssucid 6417 . . . . . . . . . . . . 13 1o ⊆ suc 1o
17 df-2o 8438 . . . . . . . . . . . . 13 2o = suc 1o
1816, 17sseqtrri 3999 . . . . . . . . . . . 12 1o ⊆ 2o
19 1on 8449 . . . . . . . . . . . . . 14 1o ∈ On
2017, 19sucneqoni 37361 . . . . . . . . . . . . 13 2o ≠ 1o
2120necomi 2980 . . . . . . . . . . . 12 1o ≠ 2o
22 df-pss 3937 . . . . . . . . . . . 12 (1o ⊊ 2o ↔ (1o ⊆ 2o ∧ 1o ≠ 2o))
2318, 21, 22mpbir2an 711 . . . . . . . . . . 11 1o ⊊ 2o
24 ssnpss 4072 . . . . . . . . . . 11 (2o ⊆ 1o → ¬ 1o ⊊ 2o)
2523, 24mt2 200 . . . . . . . . . 10 ¬ 2o ⊆ 1o
26 sseq2 3976 . . . . . . . . . 10 (𝑁 = 1o → (2o𝑁 ↔ 2o ⊆ 1o))
2725, 26mtbiri 327 . . . . . . . . 9 (𝑁 = 1o → ¬ 2o𝑁)
2827con2i 139 . . . . . . . 8 (2o𝑁 → ¬ 𝑁 = 1o)
2928intnanrd 489 . . . . . . 7 (2o𝑁 → ¬ (𝑁 = 1o𝑋𝑈))
3029iffalsed 4502 . . . . . 6 (2o𝑁 → if((𝑁 = 1o𝑋𝑈), ∅, if(𝑋 ∈ (V × 𝑈), ⟨ 𝑁, (1st𝑋)⟩, ⟨𝑁, 𝑋⟩)) = if(𝑋 ∈ (V × 𝑈), ⟨ 𝑁, (1st𝑋)⟩, ⟨𝑁, 𝑋⟩))
31 iftrue 4497 . . . . . 6 (𝑋 ∈ (V × 𝑈) → if(𝑋 ∈ (V × 𝑈), ⟨ 𝑁, (1st𝑋)⟩, ⟨𝑁, 𝑋⟩) = ⟨ 𝑁, (1st𝑋)⟩)
3230, 31sylan9eq 2785 . . . . 5 ((2o𝑁𝑋 ∈ (V × 𝑈)) → if((𝑁 = 1o𝑋𝑈), ∅, if(𝑋 ∈ (V × 𝑈), ⟨ 𝑁, (1st𝑋)⟩, ⟨𝑁, 𝑋⟩)) = ⟨ 𝑁, (1st𝑋)⟩)
3315, 32sylan9eqr 2787 . . . 4 (((2o𝑁𝑋 ∈ (V × 𝑈)) ∧ (𝑛 = 𝑁𝑥 = 𝑋)) → if((𝑛 = 1o𝑥𝑈), ∅, if(𝑥 ∈ (V × 𝑈), ⟨ 𝑛, (1st𝑥)⟩, ⟨𝑛, 𝑥⟩)) = ⟨ 𝑁, (1st𝑋)⟩)
3433adantlll 718 . . 3 ((((𝑁 ∈ ω ∧ 2o𝑁) ∧ 𝑋 ∈ (V × 𝑈)) ∧ (𝑛 = 𝑁𝑥 = 𝑋)) → if((𝑛 = 1o𝑥𝑈), ∅, if(𝑥 ∈ (V × 𝑈), ⟨ 𝑛, (1st𝑥)⟩, ⟨𝑛, 𝑥⟩)) = ⟨ 𝑁, (1st𝑋)⟩)
35 simpll 766 . . 3 (((𝑁 ∈ ω ∧ 2o𝑁) ∧ 𝑋 ∈ (V × 𝑈)) → 𝑁 ∈ ω)
36 elex 3471 . . . 4 (𝑋 ∈ (V × 𝑈) → 𝑋 ∈ V)
3736adantl 481 . . 3 (((𝑁 ∈ ω ∧ 2o𝑁) ∧ 𝑋 ∈ (V × 𝑈)) → 𝑋 ∈ V)
38 opex 5427 . . . 4 𝑁, (1st𝑋)⟩ ∈ V
3938a1i 11 . . 3 (((𝑁 ∈ ω ∧ 2o𝑁) ∧ 𝑋 ∈ (V × 𝑈)) → ⟨ 𝑁, (1st𝑋)⟩ ∈ V)
402, 34, 35, 37, 39ovmpod 7544 . 2 (((𝑁 ∈ ω ∧ 2o𝑁) ∧ 𝑋 ∈ (V × 𝑈)) → (𝑁𝐹𝑋) = ⟨ 𝑁, (1st𝑋)⟩)
41 df-ov 7393 . 2 (𝑁𝐹𝑋) = (𝐹‘⟨𝑁, 𝑋⟩)
4240, 41eqtr3di 2780 1 (((𝑁 ∈ ω ∧ 2o𝑁) ∧ 𝑋 ∈ (V × 𝑈)) → ⟨ 𝑁, (1st𝑋)⟩ = (𝐹‘⟨𝑁, 𝑋⟩))
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 206  wa 395   = wceq 1540  wcel 2109  wne 2926  Vcvv 3450  wss 3917  wpss 3918  c0 4299  ifcif 4491  cop 4598   cuni 4874   × cxp 5639  suc csuc 6337  cfv 6514  (class class class)co 7390  cmpo 7392  ωcom 7845  1st c1st 7969  1oc1o 8430  2oc2o 8431
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1795  ax-4 1809  ax-5 1910  ax-6 1967  ax-7 2008  ax-8 2111  ax-9 2119  ax-10 2142  ax-11 2158  ax-12 2178  ax-ext 2702  ax-sep 5254  ax-nul 5264  ax-pr 5390  ax-un 7714
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 848  df-3or 1087  df-3an 1088  df-tru 1543  df-fal 1553  df-ex 1780  df-nf 1784  df-sb 2066  df-mo 2534  df-eu 2563  df-clab 2709  df-cleq 2722  df-clel 2804  df-nfc 2879  df-ne 2927  df-ral 3046  df-rex 3055  df-rab 3409  df-v 3452  df-sbc 3757  df-dif 3920  df-un 3922  df-in 3924  df-ss 3934  df-pss 3937  df-nul 4300  df-if 4492  df-pw 4568  df-sn 4593  df-pr 4595  df-op 4599  df-uni 4875  df-br 5111  df-opab 5173  df-tr 5218  df-id 5536  df-eprel 5541  df-po 5549  df-so 5550  df-fr 5594  df-we 5596  df-xp 5647  df-rel 5648  df-cnv 5649  df-co 5650  df-dm 5651  df-ord 6338  df-on 6339  df-suc 6341  df-iota 6467  df-fun 6516  df-fv 6522  df-ov 7393  df-oprab 7394  df-mpo 7395  df-1o 8437  df-2o 8438
This theorem is referenced by:  finxpreclem4  37389
  Copyright terms: Public domain W3C validator