Predicate Logic and Quantifiers

(述語論理、全称限量子、存在限量子)

Discrete Mathematics I

7th lecture, November 6, 2020

https://www.sw.it.aoyama.ac.jp/2020/Math1/lecture7.html

Martin J. Dürst

AGU

© 2005-20 Martin J. Dürst Aoyama Gakuin University

Today's Schedule

 

Leftovers of Last Lecture

Limits of sets

Summary of Last Lecture

 

Homework Due November 5, Problem 1

Prove/check the following laws using truth tables (important: always add a sentence stating the conclusion):

  1. Reductio ad absurdum: A→¬A = ¬A

    [solution removed]

  2. Contraposition: AB = ¬B→¬A

    [solution removed]

  3. The associative law for conjunction: (AB) ∧ C = A ∧  (BC)

    [solution removed]

  4. One of De Morgan's laws: ¬(AB) = ¬A ∨ ¬B

    [solution removed]

 

Homework Due November 5, Problem 2

Prove transitivity of implication (((AB) ∧ (BC)) ⇒ (AC)) by formula manipulation.

For each simplification step, indicate which law you used.

Hint: Show that ((AB) ∧ (BC)) → (AC) is a tautology by simplifying it to T.

[solution removed]

 

Homework Comment

This homework is a good example of a general strategy to simplify formulæ:

 

Homework Due October 29

[solution removed]

 

Types of Symbolic Logic

 

Limitations of Propositions

With propositions, related statements have to be made separately

Examples:
2 is even. 5 is even.
Today it is sunny. Tomorrow it is sunny. The day after tomorrow, it is sunny.

We can express "If today is sunny, then tomorrow will also be sunny." or "If 2 is even, then 3 is not even".

But we cannot express "If it's sunny on a given day, it's also sunny on the next day." or "If x is even, then x+2 is also even.".

⇒ This problem can be solved using predicates

 

Examples of Predicates

 

Predicate Overview

 

How to Write Predicates

There are two ways to write predicates:

  1. Functional notation:
  2. Operator notation:

 

Formulas Containing Predicates

Using predicates, we can express new things:

Similar to propositions, predicates can be true or false.

But predicates can also be unknown/undefined, for example if they contain variables.

Even if a predicate is undefined (e.g. even( x)),
a formula containing this predicate can have a defined value (true or false)
(e.g. even(y) → even(y+2), or odd(z) → even(z+24))

 

First Order Predicate Logic

 

Universal Quantifier

Example: ∀n∈ℕ: even(n) → even(n+2)

Readings:

General form: ∀x: P (x)

∀ is the A of "for All", inverted.

Readings in Japanese:

 

Examples of Universal Quantifiers

n∈ℕ: n > -1

n∈ℕ: ∀m∈ℕ: n+m = m+n

a∈ℚ: ∀b∈ℕ: a+b = b+a

a∈{T, F}: ∀b∈{T, F}: ab = ba

Let S be the set of all students, B the set of all books, and let read(s, b) denote the fact that student s reads book b.

Then ∀sS: ∀bB: read(s, b) means that all students read all books.

Remark: ∀sS: ∀bB: read(s, b) is interpreted as ∀sS: (∀bB: read(s, b))

 

Knowledge about Field of Application

 

Existential Quantifier

Example: ∃n∈ℕ: odd (n)

Readings:

General form: ∃y: P (y)

∃ is the mirrored form of the E in "there Exists".

Readings in Japanese:

 

Structure of Quantifier Expressions

Example: m, n∈ℕ: m > nm2n2

 

More Quantifier Examples

n∈ℕ: n + n + n = 3n

n∈ℕ: n2 = n3

n∈ℝ: n2 < 50n < n3

m, n∈ℕ: 7m + 2n = 2n + 7m

 

Applied Quantifier Examples

S: Set of students

F: Set of foods

like(p, f): Person p likes food f

  1. All students like all foods:
  2. Some students like all foods:
  3. There is a food that all students like:
  4. There is no food that all students like:
  5. Each student dislikes a food:

 

Peano Axioms in Predicate Logic

Peano Axioms (Guiseppe Peano, 1858-1932)

  1. 1∈ℕ
  2. a∈ℕ: s(a)∈ℕ
  3. ¬∃x∈ℕ: s(x) = 1
  4. a, b∈ℕ: abs(a) ≠ s(b)
  5. P(1) ∧ (∀k∈ℕ: (P(k)→P(s(k)))) ⇒ ∀a∈ℕ: P(a)

 

The Use of Variables with Quantifiers

Bound variable:
Variable quantified by a quantifier
Example: the x in: ∀x: (P(x)∧Q(y))
Free variable:
Variable not quantified by a quantifier
Example: the y in: ∀x: (P(x)∧Q(y))
Closed formula:
A formula without free variables.
Scope:
The part of a formula where a bound variable (or a quantifier) is active.
All occurrences of a bound variable within its scope can be exchanged by another variable.
Example: ∀sS: (age(s)≤30 ∧ college(s)=CSE) ⇔ ∀uS: (age(u)≤30 ∧ college(u)=CSE)
Using a bound variable outside its scope is an error.
Example: (∀x: P(x))∧Q(x)

  

Manipulation of Bound Variables

(∀sS: age(s)≤30) ∧ (∀tS: college(t)=CSE) = ∀uS: (age(u)≤30∧college(u)=CSE)

is the same as

(∀sS: age(s)≤30) ∧ (∀sS: college(s)=CSE) = ∀sS: (age(s)≤30∧college(s)=CSE)

There are three different variables s in the last statement.

Advice:

 

Important Points for Quantifiers

 

Laws for Quantifiers

  1. ¬∀x: P(x) = ∃x: ¬P(x)
  2. ¬∃x: P(x) = ∀x: ¬P(x)
  3. (X≠{}∧∀xX: P(x)) → (∃x: P(x))
  4. (∀x: P(x)) ∧ Q(y) = ∀x: P(x)∧Q(y)
  5. (∃x: P(x)) ∧ Q(y) = ∃x: P(x)∧Q(y)
  6. (∀x: P(x)) ∨ Q(y) = ∀x: P(x)∨Q(y)
  7. (∃x: P(x)) ∨ Q(y) = ∃x: P(x)∨Q(y)
  8. (∀x: P(x)) ∧ (∀x: R(x)) = ∀x: P(x)∧R(x)
  9. (∀x: P(x)) ∨ (∀x: R(x)) ⇒ ∀x: P(x)∨R(x)
  10. (∃x: P(x)) ∨ (∃x: R(x)) = ∃x: P(x)∨R(x)
  11. (∃x: P(x)) ∧ (∃x: R(x)) ⇐ ∃x: P(x)∧R(x)
  12. (∃y: ∀x: P(x, y)) ⇒ (∀x: ∃y: P(x, y))
  13. P(x) is a tautology ⇔∀x: P(x) is a tautology

 

Combination of Quantifiers

(∃y: ∀x: P(x, y)) ⇒ (∀x: ∃y: P(x, y))

(∀x: ∃y: P(x, y)) ⇏ (∃y: ∀x: P(x, y))

The number of prime numbers is infinite.

(This means that whatever big number x we choose, there will always be a bigger prime number y.)

x: ∃y: (y > x ∧ prime(y))

Reversing the order of the quantifiers changes the meaning:

y: ∀x: (y > x ∧ prime(y))

(There is a prime number y that is bigger than any (natural number) x. This statement is obviously false.)

 

Proof that the Number of Primes is Infinite

This proves that there is no largest prime number, and therefore, the number of primes is infinite.

This is a proof by contradiction.

  

Summary

 

This Week's Homework

Deadline: Thursday November 12, 2020, 22:00.

Problems: See handout

If you have a printer, print out and fill in the handout.

If you do not have a printer, use a page of white A4 paper, and number the solutions carefully.

Format: A4 scanned PDF (more than one page is okay, but single file; NO cover page), easily readable handwriting (NO printouts), name (kanji and kana) and student number at the top right

Where to submit: Moodle assignment

 

Glossary

Mathematical induction
数学的帰納法
Pascal's triangle
パスカルの三角形
predicate logic
述語論理
quantifier
限量子
evaluate
評価する
evaluation
評価
array
配列
tautology
恒真 (式)、トートロジー
contradiction
恒偽 (式)
symbolic logic
記号論理
multi-valued logic
多値論理
fuzzy logic
ファジィ論理
ambiguity
曖昧さ
first-order predicate logic
一階述語論理
temporal logic
時相論理
binary logic
二値論理
generalization
一般化
argument
引数
undefined
未定
higher-order logic
高階述語論理
universal quantifier
全称限量子 (全称記号)
existential quantifier
存在限量子 (存在記号)
inference
推論
College of Science and Engineering
理工学部
native of ...
...出身
bound variable
束縛変数
free variable
自由変数
local variable
局所変数
closed formula
閉論理式
scope
作用領域、スコープ
prime (number)
素数