Induction
Induction
Principles
Patricia H ILL
School of Computing
University of Leeds, United Kingdom
Roberto B AGNARA
Department of Mathematics
University of Parma, Italy
Copyright c 2004–2013 Patricia Hill. Distributed under the terms of the GNU Free Documentation License 1.2 1
M ATHEMATICAL I NDUCTION
Let P (n) be a property of natural numbers n = 0, 1, 2, . . . The
principle of mathematical induction says that to show P (n) holds for
all natural numbers, it is sufficient to show:
• The step case: If P (m) holds then so does P (m + 1), for any
natural number m.
M ATHEMATICAL I NDUCTION 2
M ATHEMATICAL I NDUCTION : E XAMPLE 1
Let us show that P (n) ≡ 0 + 2 + 4 + · · · + 2n = n(n + 1) :
Pm
• Inductive hypothesis: P (m) ≡ i=0 2i = m(m + 1) .
• Base case, m = 0: P (0) ≡ 0 = 0(0 + 1) .
so that P (m + 1) holds.
1 + 3 + 5 + · · · + (2n + 1) = (n + 1)2 ;
1 1 1 1 n+1
+ + + ···+ = ;
1·2 2·3 3·4 (n + 1)(n + 2) n+2
2 1 − r n+1
n
1 + r + r + ···+ r = .
1−r
E XERCISES 4
M ATHEMATICAL I NDUCTION : E XAMPLE 2
Let Q(n) be the property that, for all symbols a, b, s1 , . . . , sn , we have
(as1 · · · sn = s1 · · · sn b) =⇒ a = b. We show that ∀n ∈ N : Q(n).
• Inductive hypothesis:
Q(m) ≡ (as1 · · · sm = s1 · · · sm b) =⇒ a = b .
• Base case, m = 0: Q(0) ≡ (a = b =⇒ a = b).
• Step case, m ≥ 0: Suppose
as1 · · · sm = s1 · · · sm sm+1 = s1 · · · sm b.
S TRUCTURAL I NDUCTION 7
S TRUCTURAL I NDUCTION : E XERCISE
Definition:
a0 ⊐ a1 ⊐ a2 ⊐ · · ·
a0 ≻ a1 ≻ · · · ≻ ai ≻ · · ·
∀S ⊆ A : (S 6= ∅ =⇒ ∃m ∈ S . ∀s ∈ S : s ⊀ m)
a b ⇐⇒ a = b ∨ a ≺ b
(a1 R a2 ∧ a2 R a3 ) =⇒ a1 R a3 ;
(a1 R a2 ∧ a2 R a1 ) =⇒ a1 = a2 .
PARTIAL O RDERING 12
W ELL -F OUNDED R ELATIONS AND PARTIAL O RDERINGS
Exercise: Let ‘≺’ a well-founded relation over a set A.
D EFINITIONS BY I NDUCTION 16