• Aucun résultat trouvé

January19 ,2021 PROOFSBYINDUCTION ConceptsinAbstractMathematics

N/A
N/A
Protected

Academic year: 2022

Partager "January19 ,2021 PROOFSBYINDUCTION ConceptsinAbstractMathematics"

Copied!
13
0
0

Texte intégral

(1)

MAT246H1-S – LEC0201/9201

Concepts in Abstract Mathematics

PROOFS BY INDUCTION

January 19th, 2021

(2)

Proof by induction: the formal statement

Theorem

Let𝒫(𝑛)be a statement depending on𝑛 ∈ ℕ.

If𝒫(0)is true and if𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)is true for all𝑛 ∈ ℕ, then𝒫(𝑛)is true for all𝑛 ∈ ℕ. Formally,

{ 𝒫(0)

∀𝑛 ∈ ℕ, (𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)) ⟹ ∀𝑛 ∈ ℕ, 𝒫(𝑛) Proof. We define the set𝐴 = {𝑛 ∈ ℕ ∶ 𝒫(𝑛)is true}. Then:

• 𝐴 ⊂ ℕby definition of𝐴.

• 0 ∈ ℕsince𝒫(0)is true.

• 𝑠(𝐴) ⊂ 𝐴

Indeed, let𝑛 ∈ 𝑠(𝐴). Then𝑛 = 𝑠(𝑚) = 𝑚 + 1for some𝑚 ∈ 𝐴.

By definition of𝐴,𝒫(𝑚)is true. But by assumption𝒫(𝑚) ⟹ 𝒫(𝑚 + 1)is also true. Hence𝒫(𝑚 + 1)is true, meaning that𝑛 = 𝑚 + 1 ∈ 𝐴.

By theinduction principlewe get𝐴 = ℕ. Hence, for every𝑛 ∈ ℕ, we have that𝒫(𝑛)is true. ■

(3)

Proof by induction: the formal statement

Theorem

Let𝒫(𝑛)be a statement depending on𝑛 ∈ ℕ.

If𝒫(0)is true and if𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)is true for all𝑛 ∈ ℕ, then𝒫(𝑛)is true for all𝑛 ∈ ℕ. Formally,

{ 𝒫(0)

∀𝑛 ∈ ℕ, (𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)) ⟹ ∀𝑛 ∈ ℕ, 𝒫(𝑛)

Proof. We define the set𝐴 = {𝑛 ∈ ℕ ∶ 𝒫(𝑛)is true}. Then:

• 𝐴 ⊂ ℕby definition of𝐴.

• 0 ∈ ℕsince𝒫(0)is true.

• 𝑠(𝐴) ⊂ 𝐴

Indeed, let𝑛 ∈ 𝑠(𝐴). Then𝑛 = 𝑠(𝑚) = 𝑚 + 1for some𝑚 ∈ 𝐴.

By definition of𝐴,𝒫(𝑚)is true. But by assumption𝒫(𝑚) ⟹ 𝒫(𝑚 + 1)is also true. Hence𝒫(𝑚 + 1)is true, meaning that𝑛 = 𝑚 + 1 ∈ 𝐴.

By theinduction principlewe get𝐴 = ℕ. Hence, for every𝑛 ∈ ℕ, we have that𝒫(𝑛)is true. ■

(4)

Proof by induction: the formal statement

Theorem

Let𝒫(𝑛)be a statement depending on𝑛 ∈ ℕ.

If𝒫(0)is true and if𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)is true for all𝑛 ∈ ℕ, then𝒫(𝑛)is true for all𝑛 ∈ ℕ. Formally,

{ 𝒫(0)

∀𝑛 ∈ ℕ, (𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)) ⟹ ∀𝑛 ∈ ℕ, 𝒫(𝑛) Proof. We define the set𝐴 = {𝑛 ∈ ℕ ∶ 𝒫(𝑛)is true}. Then:

• 𝐴 ⊂ ℕby definition of𝐴.

• 0 ∈ ℕsince𝒫(0)is true.

• 𝑠(𝐴) ⊂ 𝐴

Indeed, let𝑛 ∈ 𝑠(𝐴). Then𝑛 = 𝑠(𝑚) = 𝑚 + 1for some𝑚 ∈ 𝐴.

By definition of𝐴,𝒫(𝑚)is true. But by assumption𝒫(𝑚) ⟹ 𝒫(𝑚 + 1)is also true.

Hence𝒫(𝑚 + 1)is true, meaning that𝑛 = 𝑚 + 1 ∈ 𝐴.

By theinduction principlewe get𝐴 = ℕ. Hence, for every𝑛 ∈ ℕ, we have that𝒫(𝑛)is true. ■

(5)

Proof by induction: in practice

When writing a proof by induction, there are several steps that you should make appear clearly.

• What statement are you proving? What is your𝒫(𝑛)?

Particularly, on which parameter are you doing the induction?

You should make everything clear for the reader!

Base case: prove that𝒫(0)is true.

Induction step: prove that if𝒫(𝑛)is true for some𝑛 ∈ ℕthen𝒫(𝑛 + 1)is also true.

It is important to clearly write the induction hypothesis and what you want to prove in this step (the reader shouldn’t have to guess).

Make sure that you used the induction hypothesis somewhere, otherwise there is something suspicious with your proof.

(6)

Proof by induction: an example

Proposition

∀𝑛 ∈ ℕ, 0 + 1 + 2 + 3 + ⋯ + 𝑛 = 𝑛(𝑛 + 1) 2

Proof.We are proving the above statement by induction on𝑛.

Base case at𝑛 = 0. Then the sum in the left hand side is equal to 0. And 𝑛(𝑛+1)

2 = 0⋅12 = 0. So the equality holds.

Induction step. Assume that0 + 1 + 2 + 3 + ⋯ + 𝑛 = 𝑛(𝑛+1)2 for some𝑛 ∈ ℕthen

0 + 1 + 2 + 3 + ⋯ + 𝑛 + (𝑛 + 1) = 𝑛(𝑛 + 1)

2 + (𝑛 + 1) by the induction hypothesis

= 𝑛(𝑛 + 1) + 2(𝑛 + 1)

2 = (𝑛 + 1)(𝑛 + 2) 2

Which proves the induction step. ■

(7)

Proof by induction: an example

Proposition

∀𝑛 ∈ ℕ, 0 + 1 + 2 + 3 + ⋯ + 𝑛 = 𝑛(𝑛 + 1) 2

Proof.We are proving the above statement by induction on𝑛.

Base case at𝑛 = 0. Then the sum in the left hand side is equal to 0. And 𝑛(𝑛+1)

2 = 0⋅12 = 0.

So the equality holds.

Induction step. Assume that0 + 1 + 2 + 3 + ⋯ + 𝑛 = 𝑛(𝑛+1)2 for some𝑛 ∈ ℕthen

0 + 1 + 2 + 3 + ⋯ + 𝑛 + (𝑛 + 1) = 𝑛(𝑛 + 1)

2 + (𝑛 + 1) by the induction hypothesis

= 𝑛(𝑛 + 1) + 2(𝑛 + 1)

2 = (𝑛 + 1)(𝑛 + 2) 2

Which proves the induction step. ■

(8)

Proof by induction: base case at 𝑛

0

– 1

Theorem

Let𝑛0∈ ℕ. Let𝒫(𝑛)be a statement depending on a natural number𝑛 ≥ 𝑛0.

If𝒫(𝑛0)is true and if𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)is true for every natural number𝑛 ≥ 𝑛0, then𝒫(𝑛)is true for every natural number𝑛 ≥ 𝑛0. Formally,

{ 𝒫(𝑛0)

∀𝑛 ∈ ℕ≥𝑛0, (𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)) ⟹ ∀𝑛 ∈ ℕ≥𝑛0, 𝒫(𝑛)

Proof.For𝑛 ∈ ℕ, we defineℛ(𝑛)by

ℛ(𝑛)is true⇔ 𝒫(𝑛 + 𝑛0)is true

Thenℛ(0)is true since𝒫(𝑛0)is. And, for all𝑛 ∈ ℕ,ℛ(𝑛) ⟹ ℛ(𝑛 + 1)is true. By the usual inductionℛ(𝑛)is true for any𝑛 ∈ ℕ, i.e.𝒫(𝑛)is true for any𝑛 ∈ ℕ≥𝑛0.

(9)

Proof by induction: base case at 𝑛

0

– 1

Theorem

Let𝑛0∈ ℕ. Let𝒫(𝑛)be a statement depending on a natural number𝑛 ≥ 𝑛0.

If𝒫(𝑛0)is true and if𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)is true for every natural number𝑛 ≥ 𝑛0, then𝒫(𝑛)is true for every natural number𝑛 ≥ 𝑛0. Formally,

{ 𝒫(𝑛0)

∀𝑛 ∈ ℕ≥𝑛0, (𝒫(𝑛) ⟹ 𝒫(𝑛 + 1)) ⟹ ∀𝑛 ∈ ℕ≥𝑛0, 𝒫(𝑛)

Proof.For𝑛 ∈ ℕ, we defineℛ(𝑛)by

ℛ(𝑛)is true⇔ 𝒫(𝑛 + 𝑛0)is true

Thenℛ(0)is true since𝒫(𝑛0)is. And, for all𝑛 ∈ ℕ,ℛ(𝑛) ⟹ ℛ(𝑛 + 1)is true.

By the usual inductionℛ(𝑛)is true for any𝑛 ∈ ℕ, i.e. 𝒫(𝑛)is true for any𝑛 ∈ ℕ≥𝑛0.

(10)

Proof by induction: base case at 𝑛

0

– 2

Proposition

For any integer𝑛 ≥ 5,2𝑛> 𝑛2.

Proof.We are going to prove that∀𝑛 ≥ 5, 2𝑛> 𝑛2by induction on𝑛.

Base case at𝑛 = 5: 25= 32 > 25 = 52.

Induction step: Assume that2𝑛> 𝑛2for some𝑛 ≥ 5and let’s prove that2𝑛+1> (𝑛 + 1)2. Note that2𝑛+1= 2 × 2𝑛≥ 2𝑛2by the induction hypothesis. Hence it is enough to prove that 2𝑛2> (𝑛 + 1)2which is equivalent to𝑛2− 2𝑛 − 1 > 0.

We study the sign of the polynomial𝑥2− 2𝑥 − 1. It is a polynomial of degree 2 with positive leading coefficient and its discriminant is(−2)2− 4 × (−1) = 8 > 0. Therefore

𝑥 𝑥2− 2𝑥 − 1

−∞ 1 − √2 1 + √2 +∞

+ 0 − 0 +

Since5 > 1 + √2, we know that𝑛2− 2𝑛 − 1 > 0for𝑛 ≥ 5. Which proves the induction step.

(11)

Proof by induction: base case at 𝑛

0

– 2

Proposition

For any integer𝑛 ≥ 5,2𝑛> 𝑛2.

Proof.We are going to prove that∀𝑛 ≥ 5, 2𝑛> 𝑛2by induction on𝑛.

Base case at𝑛 = 5: 25= 32 > 25 = 52.

Induction step: Assume that2𝑛> 𝑛2for some𝑛 ≥ 5and let’s prove that2𝑛+1> (𝑛 + 1)2. Note that2𝑛+1= 2 × 2𝑛≥ 2𝑛2by the induction hypothesis. Hence it is enough to prove that 2𝑛2> (𝑛 + 1)2which is equivalent to𝑛2− 2𝑛 − 1 > 0.

We study the sign of the polynomial𝑥2− 2𝑥 − 1. It is a polynomial of degree 2 with positive leading coefficient and its discriminant is(−2)2− 4 × (−1) = 8 > 0. Therefore

𝑥 𝑥2− 2𝑥 − 1

−∞ 1 − √2 1 + √2 +∞

+ 0 − 0 +

Since5 > 1 + √2, we know that𝑛2− 2𝑛 − 1 > 0for𝑛 ≥ 5. Which proves the induction step.

(12)

Proof by induction: strong induction

Theorem

Let𝒫(𝑛)be a statement depending on𝑛 ≥ 𝑛0.

If𝒫(𝑛0)is true and if(𝑃 (𝑛0), 𝑃 (𝑛0+ 1), … , 𝒫(𝑛)) ⟹ 𝒫(𝑛 + 1)is true for all𝑛 ≥ 𝑛0, then𝒫(𝑛)is true for all𝑛 ≥ 𝑛0. Formally,

{ 𝒫(𝑛0)

∀𝑛 ≥ 𝑛0, ((𝒫(𝑛0), 𝒫(𝑛0+ 1), … , 𝒫(𝑛)) ⟹ 𝒫(𝑛 + 1)) ⟹ ∀𝑛 ≥ 𝑛0, 𝒫(𝑛)

Proof.For𝑛 ≥ 𝑛0, we defineℛ(𝑛)by

ℛ(𝑛)is true⇔ 𝒫(𝑛0), 𝒫(𝑛0+ 1), … , 𝒫(𝑛)are true

Assume that𝒫(𝑛0)is true and that(𝑃 (𝑛0), 𝑃 (𝑛0+ 1), … , 𝒫(𝑛)) ⟹ 𝒫(𝑛 + 1)is true for all𝑛 ≥ 𝑛0. Thenℛ(0)is true since𝒫(0)is. And, for all𝑛 ≥ 𝑛0,ℛ(𝑛) ⟹ ℛ(𝑛 + 1)is true.

By the usual inductionℛ(𝑛)is true for any𝑛 ≥ 𝑛0.

Particularly,𝒫(𝑛)is true for any𝑛 ≥ 𝑛0as expected. ■

(13)

Proof by induction: strong induction

Theorem

Let𝒫(𝑛)be a statement depending on𝑛 ≥ 𝑛0.

If𝒫(𝑛0)is true and if(𝑃 (𝑛0), 𝑃 (𝑛0+ 1), … , 𝒫(𝑛)) ⟹ 𝒫(𝑛 + 1)is true for all𝑛 ≥ 𝑛0, then𝒫(𝑛)is true for all𝑛 ≥ 𝑛0. Formally,

{ 𝒫(𝑛0)

∀𝑛 ≥ 𝑛0, ((𝒫(𝑛0), 𝒫(𝑛0+ 1), … , 𝒫(𝑛)) ⟹ 𝒫(𝑛 + 1)) ⟹ ∀𝑛 ≥ 𝑛0, 𝒫(𝑛)

Proof.For𝑛 ≥ 𝑛0, we defineℛ(𝑛)by

ℛ(𝑛)is true⇔ 𝒫(𝑛0), 𝒫(𝑛0+ 1), … , 𝒫(𝑛)are true

Assume that𝒫(𝑛0)is true and that(𝑃 (𝑛0), 𝑃 (𝑛0+ 1), … , 𝒫(𝑛)) ⟹ 𝒫(𝑛 + 1)is true for all𝑛 ≥ 𝑛0. Thenℛ(0)is true since𝒫(0)is. And, for all𝑛 ≥ 𝑛0,ℛ(𝑛) ⟹ ℛ(𝑛 + 1)is true.

By the usual inductionℛ(𝑛)is true for any𝑛 ≥ 𝑛0.

Particularly,𝒫(𝑛)is true for any𝑛 ≥ 𝑛0as expected. ■

Références

Documents relatifs

A little time invested now will help you make the most of your conference and will give you the skills necessary to participate in any conference at The University of

It is important to clearly write the induction hypothesis and what you want to prove in this step (the reader shouldn’t have to guess). Make sure that you used the induction

It is important to clearly write the induction hypothesis and what you want to prove in this step (the reader shouldn’t have to guess).. Make sure that you used the induction

These requirements, in combination with the Cognitive Work Analysis (presented in the following section), informed the initial design of the User Interface (Figure

Ifthe cursor cannot find what you ask it to , it will not move. Sometimes it leaps a certain di stance, then suddenly darts back and seems stuck. We call this cursor rebound. The

Abstract—This article presents research on human interactions by using a methodology of gradually revealed images for recognitionI. The idea we measure here it to

Peut comprendre une intervention si elle est lente et soigneusement articulée et comprend de longues pauses qui permettent d’en assimiler le sens.

pastry shell in the pie plate..