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

Theorem csbopg 4896
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 4588 . . 3 𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅) = if([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V), 𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}}, 𝐴 / 𝑥∅)
2 sbcan 3844 . . . . 5 ([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V) ↔ ([𝐴 / 𝑥]𝐶 ∈ V ∧ [𝐴 / 𝑥]𝐷 ∈ V))
3 sbcel1g 4422 . . . . . 6 (𝐴𝑉 → ([𝐴 / 𝑥]𝐶 ∈ V ↔ 𝐴 / 𝑥𝐶 ∈ V))
4 sbcel1g 4422 . . . . . 6 (𝐴𝑉 → ([𝐴 / 𝑥]𝐷 ∈ V ↔ 𝐴 / 𝑥𝐷 ∈ V))
53, 4anbi12d 632 . . . . 5 (𝐴𝑉 → (([𝐴 / 𝑥]𝐶 ∈ V ∧ [𝐴 / 𝑥]𝐷 ∈ V) ↔ (𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V)))
62, 5bitrid 283 . . . 4 (𝐴𝑉 → ([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V) ↔ (𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V)))
7 csbprg 4714 . . . . 5 (𝐴𝑉𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}} = {𝐴 / 𝑥{𝐶}, 𝐴 / 𝑥{𝐶, 𝐷}})
8 csbsng 4713 . . . . . 6 (𝐴𝑉𝐴 / 𝑥{𝐶} = {𝐴 / 𝑥𝐶})
9 csbprg 4714 . . . . . 6 (𝐴𝑉𝐴 / 𝑥{𝐶, 𝐷} = {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷})
108, 9preq12d 4746 . . . . 5 (𝐴𝑉 → {𝐴 / 𝑥{𝐶}, 𝐴 / 𝑥{𝐶, 𝐷}} = {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}})
117, 10eqtrd 2775 . . . 4 (𝐴𝑉𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}} = {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}})
12 csbconstg 3927 . . . 4 (𝐴𝑉𝐴 / 𝑥∅ = ∅)
136, 11, 12ifbieq12d 4559 . . 3 (𝐴𝑉 → if([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V), 𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}}, 𝐴 / 𝑥∅) = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅))
141, 13eqtrid 2787 . 2 (𝐴𝑉𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅) = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅))
15 dfopif 4875 . . 3 𝐶, 𝐷⟩ = if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅)
1615csbeq2i 3916 . 2 𝐴 / 𝑥𝐶, 𝐷⟩ = 𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅)
17 dfopif 4875 . 2 𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷⟩ = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅)
1814, 16, 173eqtr4g 2800 1 (𝐴𝑉𝐴 / 𝑥𝐶, 𝐷⟩ = ⟨𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷⟩)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 395   = wceq 1537  wcel 2106  Vcvv 3478  [wsbc 3791  csb 3908  c0 4339  ifcif 4531  {csn 4631  {cpr 4633  cop 4637
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1792  ax-4 1806  ax-5 1908  ax-6 1965  ax-7 2005  ax-8 2108  ax-9 2116  ax-10 2139  ax-11 2155  ax-12 2175  ax-ext 2706
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 848  df-3an 1088  df-tru 1540  df-fal 1550  df-ex 1777  df-nf 1781  df-sb 2063  df-clab 2713  df-cleq 2727  df-clel 2814  df-nfc 2890  df-rab 3434  df-v 3480  df-sbc 3792  df-csb 3909  df-dif 3966  df-un 3968  df-ss 3980  df-nul 4340  df-if 4532  df-sn 4632  df-pr 4634  df-op 4638
This theorem is referenced by:  sbcop  5500  opsbc2ie  32504  esum2dlem  34073  csbfinxpg  37371
  Copyright terms: Public domain W3C validator