Math 3450 - Homework # 2
Set Theory
1. Let A = {1, 5, −12, 100, 1/3, π}, B = {5, 1, −12, 18, −1/3}, C = {10, −1, 0},
D = {1, 2}, and E = {1, −1}. Calculate the following:
(a) A ∪ B
Solution: {1, 5, −12, 100, 1/3, π, 18, −1/3}
(b) A ∩ B
Solution: {1, 5, −12}
(c) A ∩ C
Solution: ∅
(d) A ∩ ∅
Solution: ∅
(e) B ∪ ∅
Solution: B
(f) D × E
Solution: {(1, 1), (1, −1), (2, 1), (2, −1)}
(g) (D ∩ A) × (E ∪ D)
Solution: D ∩ A = {1}, E ∪ D = {1, 2, −1}, (D ∩ A) × (E ∪ D) =
{(1, 1), (1, 2), (1, −1)}
(h) C × D
Solution: {(10, 1), (−1, 1), (0, 1), (10, 2), (−1, 2), (0, 2)}
(i) A − B
Solution: {100, 1/3, π}
(j) C − A
Solution: C
(k) A − ∅
Solution: A
2. Let A = {2k | k ∈ Z} and B = {3n | n ∈ Z}. Prove that A ∩ B =
{6m | m ∈ Z}.
Proof. (⊆)
First we show that A ∩ B ⊆ {6m | m ∈ Z}.
Suppose that x ∈ A ∩ B.
Then x ∈ A and x ∈ B.
Then x = 2k and x = 3n where k, n ∈ Z.
Thus 2k = 3n.
Therefore, 3n is even.
Since an odd integer multiplied by and odd integer is odd, we cannot
have that n is odd.
Therefore n is even.
So n = 2l where l ∈ Z.
Thus x = 3n = 3(2l) = 6l ∈ {6m | m ∈ Z}.
So A ∩ B ⊆ {6m | m ∈ Z}.
(⊇)
Now we show that {6m | m ∈ Z} ⊆ A ∩ B.
Let x ∈ {6m | m ∈ Z}.
Then x = 6m where m ∈ Z.
Note that x = 6m = 2(3m) = 3(2m).
Hence x ∈ A and x ∈ B.
Thus x ∈ A ∩ B.
So {6m | m ∈ Z} ⊆ A ∩ B.
Therefore by (⊆) and (⊇) we get that A ∩ B = {6m | m ∈ Z}.
3. Let A, B, and C be sets. Prove that if A ⊆ B, then A − C ⊆ B − C.
Proof. Let x ∈ A − C.
We will show that x ∈ B − C.
We know that x ∈ A and x ∈
/ C, because x ∈ A − C.
Since x ∈ A and A ⊆ B we have that x ∈ B.
Since x ∈ B and x ∈
/ C it follows that x ∈ B − C.
Therefore A − C ⊆ B − C.
4. Let A and B be sets. Prove that A ⊆ B if and only if A − B = ∅.
Proof 1 - by contraposition. In this version of the proof we will use
contraposition. Recall that P iff Q is equivalent to ¬P iff ¬Q. Thus
“A ⊆ B if and only if A − B = ∅” is equivalent to “A 6⊆ B if and only
if A − B 6= ∅”. We instead prove this second statement.
(⇒) Suppose that A 6⊆ B.
This means that there exists an x ∈ A with x 6∈ B.
Thus there exists x with x ∈ A − B.
So A − B 6= ∅.
(⇐) Suppose that A − B 6= ∅.
Then there exists x ∈ A − B.
So x ∈ A and x 6∈ B.
Thus A 6⊆ B.
Proof 2 - by contradiction. (⇒)
First, we will show that if A ⊆ B, then A − B = ∅.
We will prove this by contradiction.
Suppose that A ⊆ B, but A − B 6= ∅.
Then there exists x ∈ A − B.
So x ∈ A and x ∈
/ B.
But A ⊆ B, so x ∈ A implies that x ∈ B.
Contradiction.
Therefore A − B = ∅.
(⇐)
Next, we will show that if A − B = ∅, then A ⊆ B.
Suppose x ∈ A. We will show that x ∈ B.
Suppose to the contrary that x ∈
/ B.
Then x ∈ A − B, since x ∈ A and x 6∈ B.
But A − B = ∅.
Contradiction.
Therefore x ∈ B.
Therefore A ⊆ B.
5. Let A, B, and C be sets. Prove that if A ⊆ B, then A ∪ C ⊆ B ∪ C.
Proof. Suppose x ∈ A ∪ C.
We will show that x ∈ B ∪ C.
We know that x ∈ A or x ∈ C.
Case 1: Suppose that x ∈ A.
Since A ⊆ B we have that x ∈ B.
Thus x ∈ B and x ∈ C.
So x ∈ B ∪ C.
Case 2: Suppose that x ∈ C.
Then x ∈ B ∪ C.
In either case above, we get that x ∈ B ∪ C.
So A ∪ C ⊆ B ∪ C.
6. Let A, B, and C be sets. Prove that A × (B ∩ C) = (A × B) ∩ (A × C).
Proof. (⊆)
First, we will show that A × (B ∩ C) ⊆ (A × B) ∩ (A × C).
Suppose that (x, y) ∈ A × (B ∩ C).
Then x ∈ A and y ∈ B ∩ C.
Since y ∈ B ∩ C, we have that y ∈ B and y ∈ C.
Since x ∈ A and y ∈ B, we have that (x, y) ∈ A × B.
Since x ∈ A and y ∈ C, we have that (x, y) ∈ A × C.
So (x, y) ∈ (A × B) ∩ (A × C).
Therefore A × (B ∩ C) ⊆ (A × B) ∩ (A × C).
(⊇)
Next, we will show that (A × B) ∩ (A × C) ⊆ A × (B ∩ C).
Suppose that (x, y) ∈ (A × B) ∩ (A × C).
Then (x, y) ∈ A × B and (x, y) ∈ A × C.
Since (x, y) ∈ A × B we get that x ∈ A and y ∈ B.
Since (x, y) ∈ A × C we get that x ∈ A and y ∈ C.
So y ∈ B ∩ C, because y ∈ B and y ∈ C.
Thus (x, y) ∈ A × (B ∩ C), because x ∈ A and y ∈ B ∩ C.
Ergo, (A × B) ∩ (A × C) ⊆ A × (B ∩ C).
Therefore by (⊆) and (⊇) we get that A × (B ∩ C) = (A × B) ∩ (A ×
C).
7. Let A, B, and C be sets. Prove or disprove: If A∩B 6= ∅ and B ∩C 6= ∅,
then A ∩ C 6= ∅.
Solution:
False. Here’s a counterexample: A = {1}, B = {1, 2}, C = {2}.
8. Let An = {x ∈ Z | − n ≤ x ≤ n}. List the elements
T∞ in the sets
S∞A1 , A2 ,
A3 , and A4 . Then calculate the following sets i=2 An and i=5 An .
Solution:
A1 = {−1, 0, 1}, A2 = {−2, −1, 0, 1, 2}, A3 = {−3, −2, −1, 0, 1, 2, 3},
A4 = {−4, −3, −2, −1, 0, 1, 2, 3, 4}
T∞
i=2 An = {−2, −1, 0, 1, 2}
S∞
i=5 An = Z
9. Calculate the following intersections and unions.
(a) Calculate ∞
S T∞
n=1 An and n=1 An where An = (−n, n).
Solution:
S∞
An = R
Tn=1
∞
n=1 An = (−1, 1)
(b) Calculate ∞
S T∞
n=2 An and n=2 An where An = (1/n, 1).
Solution:
S∞
An = (0, 1)
Tn=2
∞
n=2 An = (1/2, 1)
(c) Calculate ∞
S T∞
n=3 An and n=3 An where An = (2 + 1/n, n).
Solution:
S∞
An = (2, ∞)
Tn=3
∞
n=3 An = (2 + 1/3, 3) = (7/3, 3)
10. Let A, B, and C be sets. Prove that A ∩ (B ∩ C) = (A ∩ B) ∩ C.
Proof. (⊆) First, we will show that A ∩ (B ∩ C) ⊆ (A ∩ B) ∩ C.
Suppose x ∈ A ∩ (B ∩ C).
Then x ∈ A and x ∈ B ∩ C.
So x ∈ A and x ∈ B and x ∈ C.
Since x ∈ A and x ∈ B we have that x ∈ A ∩ B.
So x ∈ (A ∩ B) ∩ C, because x ∈ A ∩ B and x ∈ C.
Therefore, A ∩ (B ∩ C) ⊆ (A ∩ B) ∩ C.
(⊇) Now we will show that (A ∩ B) ∩ C ⊆ A ∩ (B ∩ C).
Let x ∈ (A ∩ B) ∩ C.
Then x ∈ (A ∩ B) and x ∈ C.
Thus x ∈ A and x ∈ B and x ∈ C.
Since x ∈ B and x ∈ C we have that x ∈ B ∩ C.
Hence x ∈ A ∩ (B ∩ C) since x ∈ A and x ∈ B ∩ C.
Therefore, by (⊆) and (⊇) we get that A ∩ (B ∩ C) = (A ∩ B) ∩ C.
11. Let A, B, and C be sets. Prove that A ∪ (B ∩ C) = (A ∪ B) ∩ (A ∪ C).
Proof. (⊆) First, we will show that A ∪ (B ∩ C) ⊆ (A ∪ B) ∩ (A ∪ C).
Let x ∈ A ∪ (B ∩ C).
We know x ∈ A or x ∈ B ∩ C.
Case 1: Suppose that x ∈ A.
Then x ∈ A ∪ B, since x ∈ A.
Also, x ∈ A ∪ C, since x ∈ A.
Thus x ∈ A ∪ B and x ∈ A ∪ C.
So, x ∈ (A ∪ B) ∩ (A ∪ C).
Case 2: Suppose that x ∈ B ∩ C.
Then x ∈ B and x ∈ C.
So x ∈ A ∪ B, because x ∈ B.
Also x ∈ A ∪ C, because x ∈ C.
Thus x ∈ A ∪ B and x ∈ A ∪ C.
So x ∈ (A ∪ B) ∩ (A ∪ C).
In either case, we have x ∈ (A ∪ B) ∩ (A ∪ C).
So A ∪ (B ∩ C) ⊆ (A ∪ B) ∩ (A ∪ C).
(⊇) Next, we will show that (A ∪ B) ∩ (A ∪ C) ⊆ A ∪ (B ∩ C).
Suppose that x ∈ (A ∪ B) ∩ (A ∪ C).
Then x ∈ (A ∪ B) and x ∈ (A ∪ C).
So x ∈ A or x ∈ B, because x ∈ (A ∪ B).
Case 1: Suppose that x ∈ A.
Then x ∈ A ∪ (B ∩ C), because x ∈ A.
Case 2: Suppose that x ∈ B.
We know that x ∈ A or x ∈ C, because x ∈ (A ∪ C) (from above before
case 1).
We break case 2 into two sub-cases.
Case 2i: Suppose that x ∈ A.
Then x ∈ A ∪ (B ∩ C), because x ∈ A.
Case 2ii: Suppose that x ∈ C.
Then x ∈ B ∩ C, because x ∈ B and x ∈ C.
So x ∈ A ∪ (B ∩ C), because x ∈ B ∩ C.
In every case, we have x ∈ A ∪ (B ∩ C).
Therefore (A ∪ B) ∩ (A ∪ C) ⊆ A ∪ (B ∩ C).
Therefore, by (⊆) and (⊇) we get that A ∪ (B ∩ C) = (A ∪ B) ∩ (A ∪
C)
12. Let A, B, and C be sets. Prove that if A ⊆ B then A ⊆ B ∪ C.
Solution: Suppose that A ⊆ B.
We use this to show that A ⊆ B ∪ C.
Let x ∈ A.
Since A ⊆ B and x ∈ A, we know that x ∈ B.
Since x ∈ B, we know that x ∈ B ∪ C.
Therefore, if x ∈ A, then x ∈ B ∪ C is true.
So A ⊆ B ∪ C.
13. Let A = {1, x, 5}. List the elements of the power set P(A).
Solution:
∅, {1}, {x}, {5}, {1, x}, {1, 5}, {x, 5}, A
14. Let A and B be sets.
(a) Prove that P(A ∩ B) = P(A) ∩ P(B).
Proof. (⊆) First, we will show that P(A ∩ B) ⊆ P(A) ∩ P(B).
Suppose that S ∈ P(A ∩ B). We will show that S ∈ P(A) ∩ P(B).
We know that S ⊆ A ∩ B, because S ∈ P(A ∩ B).
So every element of S is in A ∩ B.
So every element of S is in both A and B.
So S ⊆ A and S ⊆ B.
So S ∈ P(A) and P(B).
So S ∈ P(A) ∩ P(B).
Therefore P(A ∩ B) ⊆ P(A) ∩ P(B).
(⊇) Next, we will show that P(A) ∩ P(B) ⊆ P(A ∩ B).
Suppose that S ∈ P(A) ∩ P(B). We will show that S ∈ P(A ∩ B).
We know that S ∈ P(A) and P(B), because S ∈ P(A) ∩ P(B).
So S ⊆ A and S ⊆ B.
So every element of S is in both A and B.
So every element of S is in A ∩ B.
So S ⊆ A ∩ B.
So S ∈ P(A ∩ B).
Therefore P(A) ∩ P(B) ⊆ P(A ∩ B).
Therefore, by (⊆) and (⊇) we get that P(A ∩ B) = P(A) ∩ P(B).
(b) Prove that P(A) ∪ P(B) ⊆ P(A ∪ B).
Proof. Suppose that S ∈ P(A) ∪ P(B).
Then S ∈ P(A) or S ∈ P(B).
Case 1: Suppose that S ∈ P(A).
Then S ⊆ A.
So S ⊆ A ∪ B, by problem 12 above.
Case 2: S ∈ P(B)
Then S ⊆ B.
So S ⊆ A ∪ B, by problem 12 above.
In either case, we have S ⊆ A ∪ B.
So S ∈ P(A ∪ B).
Thus, if S ∈ P(A) ∪ P(B), then S ∈ P(A ∪ B).
Therefore P(A) ∪ P(B) ⊆ P(A ∪ B).
(c) Give an example where P(A) ∪ P(B) 6= P(A ∪ B).
Solution:
A = {1}, B = {2}
P(A) = {∅, {1}}
P(B) = {∅, {2}}
P(A) ∪ P(B) = {∅, {1}, {2}}
A ∪ B = {1, 2}
P(A ∪ B) = {∅, {1}, {2}, {1, 2}}
15. Let A and B be sets. Prove that A − B and B are disjoint.
Proof. We will show that (A − B) ∩ B = ∅.
We do this by contradiction.
Suppose that (A − B) ∩ B 6= ∅.
Then there exists x ∈ (A − B) ∩ B.
So x ∈ A − B and x ∈ B.
But x ∈ A − B implies that x ∈ A and x ∈
/ B.
Thus we have that x ∈ B and x 6∈ B.
Contradiction. (We cannot have both x ∈ B and x 6∈ B.)
Therefore (A − B) ∩ B = ∅.
Therefore A − B and B are disjoint.
16. Let A, B, C, and D be sets. Prove that (A × B) ∩ (C × D) = (A ∩
C) × (B ∩ D).
Proof. (⊆) First, we will show that (A × B) ∩ (C × D) ⊆ (A ∩ C) ×
(B ∩ D).
Suppose (x, y) ∈ (A × B) ∩ (C × D).
Then (x, y) ∈ (A × B) and (x, y) ∈ (C × D).
So x ∈ A and y ∈ B, because (x, y) ∈ (A × B).
Also, x ∈ C and y ∈ D, because (x, y) ∈ (C × D).
So x ∈ A ∩ C, because x ∈ A and x ∈ C.
Also y ∈ B ∩ D, because y ∈ B and y ∈ D.
So (x, y) ∈ (A ∩ C) × (B ∩ D), because x ∈ A ∩ C and y ∈ B ∩ D.
Therefore (A × B) ∩ (C × D) ⊆ (A ∩ C) × (B ∩ D).
(⊇) Next, we will show that (A ∩ C) × (B ∩ D) ⊆ (A × B) ∩ (C × D).
Suppose that (x, y) ∈ (A ∩ C) × (B ∩ D).
Then x ∈ A ∩ C and y ∈ B ∩ D.
So x ∈ A and x ∈ C, because x ∈ A ∩ C.
Also y ∈ B and y ∈ D, because y ∈ B ∩ D.
So (x, y) ∈ A × B, because x ∈ A and y ∈ B.
Also, (x, y) ∈ C × D, because x ∈ C and y ∈ D.
Therefore (x, y) ∈ (A × B) ∩ (C × D), because (x, y) ∈ A × B and
(x, y) ∈ C × D .
So (A ∩ C) × (B ∩ D) ⊆ (A × B) ∩ (C × D).
Therefore, by (⊆) and (⊇) we get that(A × B) ∩ (C × D) = (A ∩ C) ×
(B ∩ D).