Successor Set
Definition 6.1. A set X⊆R is said to be a successor set
(i) if 1∈X,
(ii) if n∈X, then n+1∈X.
실수 집합 R은 그 자체로 successor set이기 때문에,(A9, A1) 위와 같이 정의한 successor set은 적어도 하나는 존재한다고 말할 수 있다.
Lemma 6.2
Lemma 6.2. If A is any nonempty collection of successor sets, then ∩A is a successor set.
Proof. Since 1 is in every succerssor set, 1∈∩A. Let n∈∩A. Then n∈A,∀A∈A. Then n+1 is also in any A in A by definition 6.1. Thus ∩A is a successor set. ◼
Positive Integer
Definition 6.3. The set P of positive integers is the intersection of the family of all successor sets.
위 lemma에 의해 P는 successor set이고, intersection의 정의상 집합 간의 포함 관계에 대하여 successor set들 중smallest set임이 분명하다.
Mathematical Induction
Theorem 6.4. Suppose that for each positive integer n, we have a statement S(n). Suppose also that
(i) S(1) is true.
(ii) If S(n) is true, then S(n+1) is true. Then S(n) is true for every positive integer n.
Proof. Let T={n∈P|S(n) is true}. Then by the assumption, T is a successor set. Then P⊂T and clearly T⊂P. Thus T=P. ◼
Theorem 6.5
Theorem 6.5. If n is a positive integer, then n≥1.
Proof. We will use mathematical induction. Let S(n) be the statement which is n≥1. Note that S(1) is clearly true. If S(k) is true, then k≥1. Note that k−1∈P or k=1 by definition 4.1. If k=1, then k∈P by theorem 4.2. If k−1∈P, (k−1)+1=k∈P. Thus k∈P, and k=k+1−1∈P⟹k+1>1⟹k+1≥1. Thus S(n) is true for all positive integer n. ◼
Theorem 6.6
Theorem 6.6. If m,n∈P, then m+n∈P.
Proof. Let S(n) be the statement which is m+n∈P. Since m∈P, clearly m+1∈P by the definition 6.1, so S(1) is true. If S(n) is true, that is, m+n∈P, then m+n+1∈P by the definition 6.1, so S(n+1) is true. Then by mathematical induction, S(n) is true for all positive integers. ◼
Lemma 6.7
Lemma 6.7. If n∈P, then either n−1=0 or n−1∈P.
Proof. Let G={n∈P|n−1=0 or n−1∈P}. We will show that G=P. Clearly G⊂P. Note that 1∈G. If n∈G, then (n+1)−1=n≠0 and n∈P. Thus n+1∈G, so G is a successor set. Since P is the smallest successor set, P⊂G, so G=P. ◼
Lemma 6.8
Lemma 6.8. If m,n∈P and m<n, then n‒m∈P.
Proof. Let S(m) be the statement which is n−m∈P. By the assumption, 1<n. Then by Lemma 6.7, either n−1=0 or n−1∈P. Since 1<n, n−1 cannot equal to 0, so n−1∈P, which means that S(1) is true.
Suppose that S(m) is true, i.e., n−m∈P for the positive integers n,m such that n>m. If m+1<n, then n−1∈P because n−1 cannot equal to 0, so n−1∈P by Lemma 6.7. Since m<n−1 and S(m) is true, n−1−m=n−(m+1)∈P. Thus S(m+1) is also true. By mathematical induction, S(m) is true for all positive integers. ◼
Lemma 6.9
Lemma 6.9. Let n be a positive integer. No positive integer m satisfies the inequality n<m<n+1.
Proof. Suppose that ∃m∈P such that n<m<n+1. Then m−n∈P by Lemma 6.8. But m<n+1, so m−n<1 which is a contradiction by Theorem 6.5. Thus there is no positive integer m such that n<m<n+1. ◼
Well-Ordering Theorem
Theorem 6.10. If X is a nonempty subset of the positive integers, then X contains a least element; that is, there exists a∈X such that a≤x for all x∈X.
Proof. Let S(n) be the statement: "If n∈X, then X contains a least element."
If 1∈X, then 1 is the least element of X by Theorem 6.5.
Suppose that S(n) is true and n+1∈X. Since n∈X∪{n}, X∪{n} has the least element l. If l∈X, then l≤x and ≤n<n+1 for all x∈X, so l is the least element of X. If l∉X, then n=l because l∈X∪{n}. Then n≤x and n<n+1 \for all x∈X, so n is the least element of X. Thus, X always has the least element by mathematical induction. ◼
Theorem 6.11
Theorem 6.11. The set of positive integers is not bounded above.
Proof. Suppose that P is bounded above. Then P has the least upper bound a by A13. Then a−1 is not an upper bound for P, so ∃n∈P such that a−1<n. But a<n+1, which is a contradiction. Thus P is not bounded above. ◼
Corollary 6.12
Corollary 6.12. The set of real numbers is Archimedean ordered;
(1) If a and b are positive real numbers, there exists a positive integer n such that a<nb.
(2) If ε is a positive real number, there exists a positive integer N such that 1N<ε.
Proof. (1) Suppose that there does not exist a positive integer n such that a<nb. Then ∀n∈P,a≥nb. Then n≤an,∀n∈P, which means that P is bounded above, but it is a contradiction by Theorem 6.11. Thus there exists a positive integer n such that a<nb.
(2) In (1), take a=1 and b=ε. Then ∃N∈P such that 1<Nε⟺1N<ε. ◼