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

Theorem partfun 6707
Description: Rewrite a function defined by parts, using a mapping and an if construct, into a union of functions on disjoint domains. (Contributed by Thierry Arnoux, 30-Mar-2017.)
Assertion
Ref Expression
partfun (𝑥𝐴 ↦ if(𝑥𝐵, 𝐶, 𝐷)) = ((𝑥 ∈ (𝐴𝐵) ↦ 𝐶) ∪ (𝑥 ∈ (𝐴𝐵) ↦ 𝐷))

Proof of Theorem partfun
StepHypRef Expression
1 mptun 6706 . 2 (𝑥 ∈ ((𝐴𝐵) ∪ (𝐴𝐵)) ↦ if(𝑥𝐵, 𝐶, 𝐷)) = ((𝑥 ∈ (𝐴𝐵) ↦ if(𝑥𝐵, 𝐶, 𝐷)) ∪ (𝑥 ∈ (𝐴𝐵) ↦ if(𝑥𝐵, 𝐶, 𝐷)))
2 inundif 4482 . . 3 ((𝐴𝐵) ∪ (𝐴𝐵)) = 𝐴
3 eqid 2728 . . 3 if(𝑥𝐵, 𝐶, 𝐷) = if(𝑥𝐵, 𝐶, 𝐷)
42, 3mpteq12i 5258 . 2 (𝑥 ∈ ((𝐴𝐵) ∪ (𝐴𝐵)) ↦ if(𝑥𝐵, 𝐶, 𝐷)) = (𝑥𝐴 ↦ if(𝑥𝐵, 𝐶, 𝐷))
5 elinel2 4198 . . . . 5 (𝑥 ∈ (𝐴𝐵) → 𝑥𝐵)
65iftrued 4540 . . . 4 (𝑥 ∈ (𝐴𝐵) → if(𝑥𝐵, 𝐶, 𝐷) = 𝐶)
76mpteq2ia 5255 . . 3 (𝑥 ∈ (𝐴𝐵) ↦ if(𝑥𝐵, 𝐶, 𝐷)) = (𝑥 ∈ (𝐴𝐵) ↦ 𝐶)
8 eldifn 4128 . . . . 5 (𝑥 ∈ (𝐴𝐵) → ¬ 𝑥𝐵)
98iffalsed 4543 . . . 4 (𝑥 ∈ (𝐴𝐵) → if(𝑥𝐵, 𝐶, 𝐷) = 𝐷)
109mpteq2ia 5255 . . 3 (𝑥 ∈ (𝐴𝐵) ↦ if(𝑥𝐵, 𝐶, 𝐷)) = (𝑥 ∈ (𝐴𝐵) ↦ 𝐷)
117, 10uneq12i 4162 . 2 ((𝑥 ∈ (𝐴𝐵) ↦ if(𝑥𝐵, 𝐶, 𝐷)) ∪ (𝑥 ∈ (𝐴𝐵) ↦ if(𝑥𝐵, 𝐶, 𝐷))) = ((𝑥 ∈ (𝐴𝐵) ↦ 𝐶) ∪ (𝑥 ∈ (𝐴𝐵) ↦ 𝐷))
121, 4, 113eqtr3i 2764 1 (𝑥𝐴 ↦ if(𝑥𝐵, 𝐶, 𝐷)) = ((𝑥 ∈ (𝐴𝐵) ↦ 𝐶) ∪ (𝑥 ∈ (𝐴𝐵) ↦ 𝐷))
Colors of variables: wff setvar class
Syntax hints:   = wceq 1533  wcel 2098  cdif 3946  cun 3947  cin 3948  ifcif 4532  cmpt 5235
This theorem was proved from axioms:  ax-mp 5  ax-1 6  ax-2 7  ax-3 8  ax-gen 1789  ax-4 1803  ax-5 1905  ax-6 1963  ax-7 2003  ax-8 2100  ax-9 2108  ax-ext 2699
This theorem depends on definitions:  df-bi 206  df-an 395  df-or 846  df-tru 1536  df-ex 1774  df-sb 2060  df-clab 2706  df-cleq 2720  df-clel 2806  df-v 3475  df-dif 3952  df-un 3954  df-in 3956  df-if 4533  df-opab 5215  df-mpt 5236
This theorem is referenced by:  mptiffisupp  32494  mptprop  32499  cycpm2tr  32861  fsuppssindlem2  41856
  Copyright terms: Public domain W3C validator