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

Theorem csbopg 4915
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 4605 . . 3 𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅) = if([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V), 𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}}, 𝐴 / 𝑥∅)
2 sbcan 3857 . . . . 5 ([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V) ↔ ([𝐴 / 𝑥]𝐶 ∈ V ∧ [𝐴 / 𝑥]𝐷 ∈ V))
3 sbcel1g 4439 . . . . . 6 (𝐴𝑉 → ([𝐴 / 𝑥]𝐶 ∈ V ↔ 𝐴 / 𝑥𝐶 ∈ V))
4 sbcel1g 4439 . . . . . 6 (𝐴𝑉 → ([𝐴 / 𝑥]𝐷 ∈ V ↔ 𝐴 / 𝑥𝐷 ∈ V))
53, 4anbi12d 631 . . . . 5 (𝐴𝑉 → (([𝐴 / 𝑥]𝐶 ∈ V ∧ [𝐴 / 𝑥]𝐷 ∈ V) ↔ (𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V)))
62, 5bitrid 283 . . . 4 (𝐴𝑉 → ([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V) ↔ (𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V)))
7 csbprg 4734 . . . . 5 (𝐴𝑉𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}} = {𝐴 / 𝑥{𝐶}, 𝐴 / 𝑥{𝐶, 𝐷}})
8 csbsng 4733 . . . . . 6 (𝐴𝑉𝐴 / 𝑥{𝐶} = {𝐴 / 𝑥𝐶})
9 csbprg 4734 . . . . . 6 (𝐴𝑉𝐴 / 𝑥{𝐶, 𝐷} = {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷})
108, 9preq12d 4766 . . . . 5 (𝐴𝑉 → {𝐴 / 𝑥{𝐶}, 𝐴 / 𝑥{𝐶, 𝐷}} = {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}})
117, 10eqtrd 2780 . . . 4 (𝐴𝑉𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}} = {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}})
12 csbconstg 3940 . . . 4 (𝐴𝑉𝐴 / 𝑥∅ = ∅)
136, 11, 12ifbieq12d 4576 . . 3 (𝐴𝑉 → if([𝐴 / 𝑥](𝐶 ∈ V ∧ 𝐷 ∈ V), 𝐴 / 𝑥{{𝐶}, {𝐶, 𝐷}}, 𝐴 / 𝑥∅) = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅))
141, 13eqtrid 2792 . 2 (𝐴𝑉𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅) = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅))
15 dfopif 4894 . . 3 𝐶, 𝐷⟩ = if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅)
1615csbeq2i 3929 . 2 𝐴 / 𝑥𝐶, 𝐷⟩ = 𝐴 / 𝑥if((𝐶 ∈ V ∧ 𝐷 ∈ V), {{𝐶}, {𝐶, 𝐷}}, ∅)
17 dfopif 4894 . 2 𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷⟩ = if((𝐴 / 𝑥𝐶 ∈ V ∧ 𝐴 / 𝑥𝐷 ∈ V), {{𝐴 / 𝑥𝐶}, {𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷}}, ∅)
1814, 16, 173eqtr4g 2805 1 (𝐴𝑉𝐴 / 𝑥𝐶, 𝐷⟩ = ⟨𝐴 / 𝑥𝐶, 𝐴 / 𝑥𝐷⟩)
Colors of variables: wff setvar class
Syntax hints:  wi 4  wa 395   = wceq 1537  wcel 2108  Vcvv 3488  [wsbc 3804  csb 3921  c0 4352  ifcif 4548  {csn 4648  {cpr 4650  cop 4654
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
This theorem depends on definitions:  df-bi 207  df-an 396  df-or 847  df-3an 1089  df-tru 1540  df-fal 1550  df-ex 1778  df-nf 1782  df-sb 2065  df-clab 2718  df-cleq 2732  df-clel 2819  df-nfc 2895  df-rab 3444  df-v 3490  df-sbc 3805  df-csb 3922  df-dif 3979  df-un 3981  df-ss 3993  df-nul 4353  df-if 4549  df-sn 4649  df-pr 4651  df-op 4655
This theorem is referenced by:  sbcop  5509  opsbc2ie  32504  esum2dlem  34056  csbfinxpg  37354
  Copyright terms: Public domain W3C validator