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

Theorem cbvopab1g 5140
Description: Change first bound variable in an ordered-pair class abstraction, using explicit substitution. Usage of this theorem is discouraged because it depends on ax-13 2390. See cbvopab1 5139 for a version with more disjoint variable conditions, but not requiring ax-13 2390. (Contributed by NM, 6-Oct-2004.) (Revised by Mario Carneiro, 14-Oct-2016.) (New usage is discouraged.)
Hypotheses
Ref Expression
cbvopab1g.1 𝑧𝜑
cbvopab1g.2 𝑥𝜓
cbvopab1g.3 (𝑥 = 𝑧 → (𝜑𝜓))
Assertion
Ref Expression
cbvopab1g {⟨𝑥, 𝑦⟩ ∣ 𝜑} = {⟨𝑧, 𝑦⟩ ∣ 𝜓}
Distinct variable groups:   𝑥,𝑦   𝑦,𝑧
Allowed substitution hints:   𝜑(𝑥,𝑦,𝑧)   𝜓(𝑥,𝑦,𝑧)

Proof of Theorem cbvopab1g
Dummy variables 𝑤 𝑣 are mutually distinct and distinct from all other variables.
StepHypRef Expression
1 nfv 1915 . . . . 5 𝑣𝑦(𝑤 = ⟨𝑥, 𝑦⟩ ∧ 𝜑)
2 nfv 1915 . . . . . . 7 𝑥 𝑤 = ⟨𝑣, 𝑦
3 nfs1v 2160 . . . . . . 7 𝑥[𝑣 / 𝑥]𝜑
42, 3nfan 1900 . . . . . 6 𝑥(𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑)
54nfex 2343 . . . . 5 𝑥𝑦(𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑)
6 opeq1 4803 . . . . . . . 8 (𝑥 = 𝑣 → ⟨𝑥, 𝑦⟩ = ⟨𝑣, 𝑦⟩)
76eqeq2d 2832 . . . . . . 7 (𝑥 = 𝑣 → (𝑤 = ⟨𝑥, 𝑦⟩ ↔ 𝑤 = ⟨𝑣, 𝑦⟩))
8 sbequ12 2253 . . . . . . 7 (𝑥 = 𝑣 → (𝜑 ↔ [𝑣 / 𝑥]𝜑))
97, 8anbi12d 632 . . . . . 6 (𝑥 = 𝑣 → ((𝑤 = ⟨𝑥, 𝑦⟩ ∧ 𝜑) ↔ (𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑)))
109exbidv 1922 . . . . 5 (𝑥 = 𝑣 → (∃𝑦(𝑤 = ⟨𝑥, 𝑦⟩ ∧ 𝜑) ↔ ∃𝑦(𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑)))
111, 5, 10cbvexv1 2362 . . . 4 (∃𝑥𝑦(𝑤 = ⟨𝑥, 𝑦⟩ ∧ 𝜑) ↔ ∃𝑣𝑦(𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑))
12 nfv 1915 . . . . . . 7 𝑧 𝑤 = ⟨𝑣, 𝑦
13 cbvopab1g.1 . . . . . . . 8 𝑧𝜑
1413nfsb 2565 . . . . . . 7 𝑧[𝑣 / 𝑥]𝜑
1512, 14nfan 1900 . . . . . 6 𝑧(𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑)
1615nfex 2343 . . . . 5 𝑧𝑦(𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑)
17 nfv 1915 . . . . 5 𝑣𝑦(𝑤 = ⟨𝑧, 𝑦⟩ ∧ 𝜓)
18 opeq1 4803 . . . . . . . 8 (𝑣 = 𝑧 → ⟨𝑣, 𝑦⟩ = ⟨𝑧, 𝑦⟩)
1918eqeq2d 2832 . . . . . . 7 (𝑣 = 𝑧 → (𝑤 = ⟨𝑣, 𝑦⟩ ↔ 𝑤 = ⟨𝑧, 𝑦⟩))
20 sbequ 2090 . . . . . . . 8 (𝑣 = 𝑧 → ([𝑣 / 𝑥]𝜑 ↔ [𝑧 / 𝑥]𝜑))
21 cbvopab1g.2 . . . . . . . . 9 𝑥𝜓
22 cbvopab1g.3 . . . . . . . . 9 (𝑥 = 𝑧 → (𝜑𝜓))
2321, 22sbie 2544 . . . . . . . 8 ([𝑧 / 𝑥]𝜑𝜓)
2420, 23syl6bb 289 . . . . . . 7 (𝑣 = 𝑧 → ([𝑣 / 𝑥]𝜑𝜓))
2519, 24anbi12d 632 . . . . . 6 (𝑣 = 𝑧 → ((𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑) ↔ (𝑤 = ⟨𝑧, 𝑦⟩ ∧ 𝜓)))
2625exbidv 1922 . . . . 5 (𝑣 = 𝑧 → (∃𝑦(𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑) ↔ ∃𝑦(𝑤 = ⟨𝑧, 𝑦⟩ ∧ 𝜓)))
2716, 17, 26cbvexv1 2362 . . . 4 (∃𝑣𝑦(𝑤 = ⟨𝑣, 𝑦⟩ ∧ [𝑣 / 𝑥]𝜑) ↔ ∃𝑧𝑦(𝑤 = ⟨𝑧, 𝑦⟩ ∧ 𝜓))
2811, 27bitri 277 . . 3 (∃𝑥𝑦(𝑤 = ⟨𝑥, 𝑦⟩ ∧ 𝜑) ↔ ∃𝑧𝑦(𝑤 = ⟨𝑧, 𝑦⟩ ∧ 𝜓))
2928abbii 2886 . 2 {𝑤 ∣ ∃𝑥𝑦(𝑤 = ⟨𝑥, 𝑦⟩ ∧ 𝜑)} = {𝑤 ∣ ∃𝑧𝑦(𝑤 = ⟨𝑧, 𝑦⟩ ∧ 𝜓)}
30 df-opab 5129 . 2 {⟨𝑥, 𝑦⟩ ∣ 𝜑} = {𝑤 ∣ ∃𝑥𝑦(𝑤 = ⟨𝑥, 𝑦⟩ ∧ 𝜑)}
31 df-opab 5129 . 2 {⟨𝑧, 𝑦⟩ ∣ 𝜓} = {𝑤 ∣ ∃𝑧𝑦(𝑤 = ⟨𝑧, 𝑦⟩ ∧ 𝜓)}
3229, 30, 313eqtr4i 2854 1 {⟨𝑥, 𝑦⟩ ∣ 𝜑} = {⟨𝑧, 𝑦⟩ ∣ 𝜓}
Colors of variables: wff setvar class
Syntax hints:  wi 4  wb 208  wa 398   = wceq 1537  wex 1780  wnf 1784  [wsb 2069  {cab 2799  cop 4573  {copab 5128
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1796  ax-4 1810  ax-5 1911  ax-6 1970  ax-7 2015  ax-8 2116  ax-9 2124  ax-10 2145  ax-11 2161  ax-12 2177  ax-13 2390  ax-ext 2793
This theorem depends on definitions:  df-bi 209  df-an 399  df-or 844  df-3an 1085  df-tru 1540  df-ex 1781  df-nf 1785  df-sb 2070  df-clab 2800  df-cleq 2814  df-clel 2893  df-nfc 2963  df-rab 3147  df-v 3496  df-dif 3939  df-un 3941  df-in 3943  df-ss 3952  df-nul 4292  df-if 4468  df-sn 4568  df-pr 4570  df-op 4574  df-opab 5129
This theorem is referenced by:  cbvmptfg  5166
  Copyright terms: Public domain W3C validator