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

Theorem csbopg 4822
Description: Distribution of class substitution over ordered pairs. (Contributed by Drahflow, 25-Sep-2015.) (Revised by Mario Carneiro, 29-Oct-2015.) (Revised by ML, 25-Oct-2020.)
Assertion
Ref Expression
csbopg (𝐴𝑉𝐴 / 𝑥𝐶, 𝐷⟩ = ⟨𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷⟩)

Proof of Theorem csbopg
StepHypRef Expression
1 csbif 4516 . . 3 𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅) = if([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V), 𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}}, 𝐴 / 𝑥∅)
2 sbcan 3768 . . . . 5 ([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V) ↔ ([𝐴 / 𝑥]𝐶 ∈ V ∧ [𝐴 / 𝑥]𝐷 ∈ V))
3 sbcel1g 4347 . . . . . 6 (𝐴𝑉 → ([𝐴 / 𝑥]𝐶 ∈ V ↔ 𝐴 / 𝑥𝐶 ∈ V))
4 sbcel1g 4347 . . . . . 6 (𝐴𝑉 → ([𝐴 / 𝑥]𝐷 ∈ V ↔ 𝐴 / 𝑥𝐷 ∈ V))
53, 4anbi12d 631 . . . . 5 (𝐴𝑉 → (([𝐴 / 𝑥]𝐶 ∈ V ∧ [𝐴 / 𝑥]𝐷 ∈ V) ↔ (𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V)))
62, 5bitrid 282 . . . 4 (𝐴𝑉 → ([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V) ↔ (𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V)))
7 csbprg 4645 . . . . 5 (𝐴𝑉𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}} = {𝐴 / 𝑥{𝐶}, 𝐴 / 𝑥{𝐶, 𝐷}})
8 csbsng 4644 . . . . . 6 (𝐴𝑉𝐴 / 𝑥{𝐶} = {𝐴 / 𝑥𝐶})
9 csbprg 4645 . . . . . 6 (𝐴𝑉𝐴 / 𝑥{𝐶, 𝐷} = {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷})
108, 9preq12d 4677 . . . . 5 (𝐴𝑉 → {𝐴 / 𝑥{𝐶}, 𝐴 / 𝑥{𝐶, 𝐷}} = {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}})
117, 10eqtrd 2778 . . . 4 (𝐴𝑉𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}} = {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}})
12 csbconstg 3851 . . . 4 (𝐴𝑉𝐴 / 𝑥∅ = ∅)
136, 11, 12ifbieq12d 4487 . . 3 (𝐴𝑉 → if([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V), 𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}}, 𝐴 / 𝑥∅) = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅))
141, 13eqtrid 2790 . 2 (𝐴𝑉𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅) = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅))
15 dfopif 4800 . . 3 𝐶, 𝐷⟩ = if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅)
1615csbeq2i 3840 . 2 𝐴 / 𝑥𝐶, 𝐷⟩ = 𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅)
17 dfopif 4800 . 2 𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷⟩ = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅)
1814, 16, 173eqtr4g 2803 1 (𝐴𝑉𝐴 / 𝑥𝐶, 𝐷⟩ = ⟨𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷⟩)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 396   = wceq 1539  wcel 2106  Vcvv 3432  [wsbc 3716  csb 3832  c0 4256  ifcif 4459  {csn 4561  {cpr 4563  cop 4567
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1798  ax-4 1812  ax-5 1913  ax-6 1971  ax-7 2011  ax-8 2108  ax-9 2116  ax-10 2137  ax-11 2154  ax-12 2171  ax-ext 2709
This theorem depends on definitions:  df-bi 206  df-an 397  df-or 845  df-3an 1088  df-tru 1542  df-fal 1552  df-ex 1783  df-nf 1787  df-sb 2068  df-clab 2716  df-cleq 2730  df-clel 2816  df-nfc 2889  df-rab 3073  df-v 3434  df-sbc 3717  df-csb 3833  df-dif 3890  df-un 3892  df-nul 4257  df-if 4460  df-sn 4562  df-pr 4564  df-op 4568
This theorem is referenced by:  sbcop  5403  opsbc2ie  30824  esum2dlem  32060  csbfinxpg  35559
  Copyright terms: Public domain W3C validator