Exercise 1.4.1

Prove all the displayed formulas in this section and visualize them using Venn diagrams.

Answers

For commutivity, Venn diagrams are not very useful.

Proof. For all x , we have that

x A B x A x B x B x A x B A ,

which shows that A B = B A . Similarly, we have that

x A B x A x B x B x A x B A ,

which proves that A B = B A . □

Venn diagrams also provide no insight for associativity.

Proof. Again, for any x , we have that

( A B ) C x A B x C ( x A x B ) x C x A x B x C x A ( x B x C ) x A x B C x A ( B C ) ,

showing that ( A B ) C = A ( B C ) . Likewise, we have

( A B ) C x A B x C ( x A x B ) x C x A x B x C x A ( x B x C ) x A x B C x A ( B C ) ,

and hence ( A B ) C = A ( B C ) . □

For distributivity, Venn diagrams do provide insight. The Venn diagram for the distributive identity A ( B C ) = ( A B ) ( A C ) is shown below:

A proof of this follows directly from the distributivity of logical conjunction.

Proof. For all x , we have

x A ( B C ) x A ( x B x C ) ( x A x B ) ( x A x C ) x A B x A C x ( A B ) ( A C ) ,

which proves the result. □

Likewise, the Venn diagram for A ( B C ) = ( A B ) ( A C ) is shown below:

This time, the proof follows directly from the distributivity of logical disjunction.

Proof. For every x , we have that

x A ( B C ) x A ( x B x C ) ( x A x B ) ( x A x C ) x A B x A C x ( A B ) ( A C ) ,

proving the desired result. □

Regarding the two DeMorgan laws, proofs of these rely on the DeMorgan and distributive laws of logic. First, we have C ( A B ) = ( C A ) ( C B ) :

Proof. For all x ,

x C ( A B ) x C x A B x C ¬ ( x A B ) x C ¬ ( x A x B ) x C ( x A x B ) ( x C x A ) ( x C x B ) x C A x C B x ( C A ) ( C B ) ,

of course showing the result. □

The other DeMorgan law is of course C ( A B ) = ( C A ) ( C B ) :

Proof. Again, for all x , we have

x C ( A B ) x C x A B x C ¬ ( x A B ) x C ¬ ( x A x B ) x C ( x A x B ) ( x C x A ) ( x C x B ) x C A x C B x ( C A ) ( C B ) ,

which proves the result. □

Next, we have the property A ( B C ) = ( A B ) C , which is visualized below:

The proof of this follows from the associativity of logical conjunction.

Proof. For all x , we have

x A ( B C ) x A x B C x A ( x B x C ) ( x A x B ) x C x A B x C x ( A B ) C ,

showing the result. □

The next claim is that A B = if and only if A B , for which a Venn diagram is not useful.

Proof. (→) First suppose that A B = and consider any x A . Suppose that x B . Then we would have x A but x B so that x A B , contradicting the fact that A B = . Hence, it has to be that x B so that A B since x was arbitrary.

(←) Now suppose that A B but that A B so that there is an x A B . Therefore, x A but x B . However, since A B it must also be that x B since x A , a contradiction! So it in fact has to be that A B = as desired. □

To prove the next property, it is first useful to establish the following lemma.

Lemma 1. For any set A , A A = .

Proof. This is very nearly self-evident, but suppose A A so that there is an x A A . Then it would both be true that x A and x A . As this is a clear contradiction, it has to be that in fact A A = as claimed. □

The next property is then that A A = , for which again a Venn diagram provides no insight and in fact does not really even make sense.

Proof. By definition and the above lemma,

A A = ( A A ) ( A A ) = = .

Clearly = since, were there an x , we would have x or x , the same impossibility in either case. □

The penultimate property asserted in this section is that A B = B A .

Proof. This follows trivially from the commutativity of the union operation, proven above. By definition, we simply have

A B = ( A B ) ( B A ) = ( B A ) ( A B ) = B A .

The final property is ( A B ) C = A ( B C ) , i.e. that the symmetric difference operation is associative. This set is visualized below:

In order to prove this while avoiding great tedium, we introduce the logical “exclusive or” operation, also called XOR. The reader may already have some familiarity with this operation, but for propositions P and Q , we denote the XOR of P and Q as P Q . The XOR operation is defined by the following truth table:

P Q P Q
F F F
F T T
T F T
T T F

Lemma 2. We claim the logical identity P Q ( P ¬ Q ) ( Q ¬ P )

Proof. To prove this, we work out the truth table for the right-hand side, in which we set R = ( P ¬ Q ) ( Q ¬ P ) for brevity:

P Q ¬ P ¬ Q P ¬ Q Q ¬ P R
F F T T F F F
F T T F F T T
T F F T T F T
T T F F F F F

Since the truth table for R is identical to that for P Q above, this proves the identity. □

Lemma 3. The logical XOR operation is associative, that is that ( P Q ) R P ( Q R ) .

Proof. This is again most easily proved via exhaustive truth tables:

P Q R P Q ( P Q ) R
F F F F F
F F T F T
F T F T T
F T T T F
T F F T T
T F T T F
T T F F F
T T T F T

P Q R Q R P ( Q R )
F F F F F
F F T T T
F T F T T
F T T F F
T F F F T
T F T T F
T T F T F
T T T F T

Since the final column of both tables are identical, this shows the desired result. □

Lemma 4. For sets A and B and any x , x A B if and only if x A x B .

Proof. For any x , define the proposition P as x A and Q as x B . Then we have that

x A B x ( A B ) ( B A ) Definition of  x A B x B A Definition of union ( x A x B ) ( x B x A ) Definition of set difference ( P ¬ Q ) ( Q ¬ P ) Definitions of  P  and  Q P Q Lemma  2 x A x B , Definitions of  P  and  Q

which of course proves the result. □

Finally, we are ready to prove the original assertion that the symmetric difference is associative.

Proof. For any x , define the proposition P as x A , Q as x B and R as x C . We then have that

x ( A B ) C ( x A x B ) x C Lemma  4 ( P Q ) R Definitions of  P Q , and  R P ( Q R ) Lemma  3 x A ( x B x C ) Definitions of  P Q , and  R x A ( B C ) . Lemma  4

This of course suffices to show that ( A B ) C = A ( B C ) . □

User profile picture
2024-07-15 11:42
Comments