Lecture-08
Lecture-08
Topics:
1. Set Operations
2. Set Identities
3. De Morgan’s Law for Set Operations
2.2 Set Operations
Definition 1: Let A and B be sets. The union of the sets A and B, denoted
by A ∪ B, is the set that contains those elements that are either in A or in
B, or in both. An element x belongs to the union of the sets A and B if and
only if x belongs to A or x belongs to B.
This tells us that A ∪ B = {x ∣ x ∈ A ∨ x ∈ B}.
EXAMPLE 1: The union of the sets {1, 3, 5} and {1, 2, 3} is the set {1,
2, 3, 5}; that is, {1, 3, 5}∪{1, 2, 3} = {1, 2, 3, 5}
EXAMPLE 3: The intersection of the sets {1, 3, 5} and {1, 2, 3} is the
set {1, 3}; that is, {1, 3, 5}∩{1, 2, 3}={1, 3}.
Venn Diagram
U U
A B A B
A ∪ B is shaded. A ∩ B is shaded.
Disjoint Set
that is, {1, 3, 5} − {1, 2, 3} = {5}. This is different from the difference of {1, 2, 3} and
{1, 3, 5}, which is the set {2}
Complement of a set
Definition 5: Let U be the universal set. The complement of the set A, denoted
by Ac, is the complement of A with respect to U.
Therefore, the complement of the set A is U − A.
Remark: The definition of the complement of A depends on a particular universal
set U. This definition makes sense for any superset U of A. If we want to identify
the universal set U, we would write “the complement of A with respect to the set
U.” An element belongs to Ac if and only if x ∉ A.
This tells us that Ac = {x ∈ U ∣ x ∉ A}.
Venn Diagram
U U
A
A B
Venn diagram for the difference of A Venn diagram for the complement of
and B the set A.
2.2.2 Set Identities
Identity Name
A ∪ (B ∪ C) = (A ∪ B) ∪ C Associative laws
A ∩ (B ∩ C) = (A ∩ B) ∩ C
A ∪ (B ∩ C) = (A ∪ B) ∩ (A ∪ C) Distributive laws
A ∩ (B ∪ C) = (A ∩ B) ∪ (A ∩ C)
A ∪ (A ∩ B) = A Absorption laws
A ∩ (A ∪ B) = A
= {x ∣ ¬(x ∈ A) ∨ ¬(x ∈ B)} by the first De Morgan law for logical equivalences
U
U
A B A B
C C
1 1 1 1 1 1 1 1
1 1 0 1 1 1 0 1
1 0 1 1 1 0 1 1
1 0 0 0 0 0 0 0
0 1 1 1 0 0 0 0
0 1 0 1 0 0 0 0
0 0 1 1 0 0 0 0
0 0 0 0 0 0 0 0
EXAMPLE 14 : Let A, B, and C be sets. Let A, B, and C be sets.
Show that (A ∪ (B ∩ C)) c = (C c ∪ B c) ∩ Ac.
Solution: We have (A ∪ (B ∩ C)) c
= Ac ∩ (B ∩ C) c by the first De Morgan law
= Ac ∩ (B c ∪ C c) by the second De Morgan law
= (B c ∪ C c) ∩ Ac by the commutative law for intersections
= (C c ∪ B c) ∩ Ac by the commutative law for unions.
Union and intersection of a collection of sets
Definition 6 The union of a collection of sets is the set that contains those elements that
are members of at least one set in the collection.
Definition 7 The intersection of a collection of sets is the set that contains those elements
that are members of all the sets in the collection.