2

This is Velleman's exercise 3.6.8.b (And of course not a duplicate of Uniqueness proof for $\forall A\in\mathcal{P}(U)\ \exists!B\in\mathcal{P}(U)\ \forall C\in\mathcal{P}(U)\ (C\setminus A=C\cap B)$):

Prove that $∀A ∈ \mathscr P(U)∃!B ∈ \mathscr P(U) ∀C ∈ \mathscr P(U) (C ∩ A = C \setminus B)$.

$\mathscr P$ is used to denote the power set.

$∃!B$ means that "there exists a unique set B such that..."

And here's my proof of it:

Proof.

Existence. Let $B = (U\setminus A) ∈ \mathscr P(U)$. Then clearly for all $A ∈ \mathscr P(U)$ and $C ∈ \mathscr P(U)$, $C\setminus B = C\setminus (U\setminus A) = C ∩ A$.

Uniqueness. To see that $B$ is unique, we choose some $B'$ in $\mathscr P(U)$ such that for all $A ∈ \mathscr P(U)$ and $C ∈ \mathscr P(U)$, $C ∩ A = C \setminus B')$. Then in particular, taking $C = U$, we can conclude that $U ∩ A = U \setminus B'$ which is equivalent to $A = U \setminus B'$ and thus $B' = U\setminus A = B$.

Here is my question:

Is my proof valid? Particularly "$C\setminus (U\setminus A) = C ∩ A$" and "$A = U \setminus B'$ and thus $B' = U\setminus A = B$" parts. In other words, do the mentioned parts need more explanation\justification?

Thanks.

Heptapod
  • 1,171

3 Answers3

2

I dont's think that the passages that you mentioned need further details. However, there is a small errer in your proof. That's when you write “Uniqueness. To see that $B$ is unique, we choose some $B'$ in $\mathscr P(U)$ such that for all $A ∈ \mathscr P(U)$…”. The quantifier $\forall A\in\mathscr{A}$ comes first. Therefore, your proof should start with: “Uniqueness. Let $A\in\mathscr P(U)$. To see that $B$ is unique, we choose some $B'$ in $\mathscr P(U)$ for all $C\in\mathscr P(U)$…”

2

I agree with José Carlos Santos and I noticed a similar error in the proof of existence when you write "Then clearly for all $A ∈\mathscr{P}(U)$ and...": again, the quantifier "for all $A \in \mathscr{P}(U)$" should come at the beginning of your proof. Indeed, you have already fixed an $A \in \mathscr{P}(U)$ just to define $B$, so saying "for all $A \in \mathscr{P}(U)$" after the definition of $B$ is an abstract nonsense. Therefore, you should write "Existence. Let $A \in \mathscr{P}(U)$ and $B=(U∖A)∈ \mathscr{P}(U)$. Then clearly for all $C∈\mathscr{P}(U)$...".

  • I would start the proof with "Let $A$ be an arbitrary subset of $U$." Then I would split the proof into "Existence" and "Uniqueness" parts, with $A$ fixed in both parts of the proof. – Dan Velleman Jun 02 '24 at 13:57
0

I working on the exact same problem in the How to Prove it by Velleman and have a bit of difficult time proving that B is unique. I don't think it is at all. The user on top of the page uses B = U\A as the desired set which satisfied the given property of C intersect A = C\B... However I picked B = C/A and that set also satisfies the given property. Clearly U\A and C\A are two different sets that satisfy the same property...?

  • The order of the quantifiers indicates that $B$ can't depend on $C$: you need the same set $B$ to work for every choice of $C$. So $B = C \setminus A$ is not an acceptable choice for $B$. – Dan Velleman Jun 02 '24 at 13:53