Quiz 1
Quiz 1
Quiz 1
Duration: 45 minutes (12 marks)
1. (2 × 2 = 4 points) Translate the following sentences into a predicate formula. The domain of discourse
should be the set of students in the class; in addition, the only predicates that you may use are (1)
Equality, (2) E(x, y) meaning that “x has sent e-mail to y.”
Note: I have used the predicate Student(x) for clarity, but its not really necessary.
(a) There is a student who has e-mailed at most n other people in the class, besides possibly himself.
Let S denote the set of students, the we can say
k k
∃s ∈ S, ∀k > n, ( ⋀ (xi ∈ S)) Ô⇒ ¬ ( ⋀ E(s, xi ))
i=1 i=1
(b) There is a student who has emailed at least n other people in the class, besides possibly himself.
Let S denote the set of students, the we can say
k k k
∃s ∈ S, ∃k ≥ n, ( ⋀ (xi ∈ S) ∧ ⋀ ¬(xp = xq )) ∧ ( ⋀ E(s, xi ))
i=1 p≠q=1 i=1
However many of you have used an extra cardinality predicate to express this, and we have given
marks for these as well.
2. (4 points) Use the Well Ordering Principle to prove that any integer greater than or equal to 8 can
be represented as the sum of nonnegative integer multiples of 3 and 5.
Proof. For the sake of contradiction assume that the set of counterexamples C is nonempty, i.e.,
By WOP C contains a least element m. Now note that if m can’t be represented as a sum of non-
negative integer multiples of 3 and 5, then neither can m − 3. Therefore m − 3 cannot be greater than
10, as if m ≥ 11 then m − 3 ≥ 8, and thus m − 3 would be in C, which is a contradiction since m is the
least element of C. The only remaining cases are n = 8, 9, 10, which are clearly not in C.
.
Note that from the stronger hypothesis, when m = 0, we recover our simpler hypothesis! Let us proceed
to prove the stronger hypothesis by induction:
√ √
• Base case: ∀m ∈ N ∪ {0}, m + 1 < m + 2 is clearly true.
• Inductive case: Assume as your induction hypothesis,
√ √ √ √
∀n ∈ N, ∀m ∈ N ∪ {0}, (m + 1) (m + 2) (m + 3) . . . (m + n − 1) < (m + 2)
as required. Note that the last inequality follows by squaring the equation on both sides (this is
ok since they are both positive quantities).