SlideShare ist ein Scribd-Unternehmen logo
1 von 10
SUBTOPIC 5               :       MATHEMATICAL INDUCTION



        Mathematical induction can be used to prove statements that assert that ∀ n ∈         , P (n) is
true. But, it is important to note that mathematical induction can be used only to prove results
obtained in some other way. It is not a tool for discovering formula or theorem.

        Principle of Induction. To prove that P (n) is true for all positive integers n, where P (n)
is a propositional function. A proof by mathematical induction has two parts:

        Basic step: We verify that P (1) is true.
        Inductive step: We show that the conditional proposition ∀ k ∈           , P (k) ⇒ P (k + 1) is
        true.

    In the induction step, the assumption that P (n) holds is called the Induction Hypothesis
(IH). In more formal notation, this proof technique can be stated as



                              [P (0) ˄∀ k (P (k) ⇒ P (k + 1)      ∀n P (n)

        You can think of the proof by (mathematical) induction as a kind of recursive proof:
Instead of attacking the problem directly, we only explain how to get a proof for P(n + 1) out of a
proof for P(n).


How would you prove that the proof by induction indeed works??


Proof (by contradiction) Assume that for some values of n, P(n) is false. Let         be the least such
n that P_n0_ is false.       Cannot be 0, because P(0) is true. Thus,      must be in the form      =1
+ . Since         <   then by P (       is true. Therefore, by inductive hypothesis P (   + 1) must be
true. It follows then that P (      is true.




                                                                                                     33
The base case can start with any nonnegative number. If that number is          then you would prove
that assertion P(n) holds for all n ≥    .


                            [P (   ) ˄∀ k ≥   (P (k) ⇒ P (k + 1)     ∀n P (n)

The induction step not necessarily should start with n. You can change the step from n -1 to n,
where n > 0. Sometimes this yields slightly shorter expressions. However, you cannot make a
step from n - 1 to n + 1.


Example:


Prove for ≥ 1
                1 x 1! + 2 x 2! + 3 x 3! + ... + n x n! = (n + 1)! - 1
This could be also written by using ∑ notation




If you take 15-355 (http://www.andrew.cmu.edu/course/15-355/) you will learn a more general
approach for deriving and proving combinatorial identities.


Proof
Base case: n _ 1
The left hand side is 1x1! The right hand side is 2! - 1. They are equal.
Inductive hypothesis: Suppose this holds




We need to prove



                                                                                                 34
Consider the left hand side




(n+1)! – 1 + (n+1) x (n+1) =


(n+1)! (1+n+1) -1 = (n+2)! -1


Suppose we have a sequence of propositions which we would like to prove:
P (0), P (1), P (2), P (3)… P (n)


We can picture each proposition as a domino:

                                                 P (k)




A sequence of propositions is visualized as a sequence of dominos.




          P (0)           P (1)          P (2)                            P (k)        P
                                                                 …..                  (k+1)




When the domino falls (to right), the corresponding proposition is considered true:


                                                                                              35
P (k)
                                                true




Suppose that the dominos satisfy two constraints.
   1. Well positioned: if any domino falls to right, the next domino to right must fall also.



                                 P (k)            P
                                 true          (k+1)
                                               true




   2. First domino has fallen to right.




                                  P (0) true




Than can conclude that all the domino fall.


         P (0)           P (1)            P (2)                           P (k)             P
                                                                  …..                     (k+1)




         P (0)           P (1)            P (2)                           P (k)             P
                                                                  …..                     (k+1)
          true



                                                                                                  36
P (1)        P (2)                   P (k)    P
                                              …..           (k+1)
P (0) true     true

  true




                            P (2)                   P (k)    P
                                              …..           (k+1)
P (0) true   P (1) true     True




                                       true         P (k)    P
                                              …..           (k+1)
P (0) true   P (1) true   P (2) true




                                                    P (k)    P
                                              …..           (k+1)
P (0) true   P (1) true   P (2) true   true         true




                                                                    37
P (0) true       P (1) true      P (2) true      true      ….. P (k) true   P (k+1) true




Principle of Mathematical Induction.
If:
      1. Basis P(1) is true
      2. Induction ∀ n P(k)        P(k+1) is true




          P (0) true       P (1) true      P (2) true      true      ….. P (k) true   P (k+1) true




Then, ∀ n P (n) is true.


Use induction to prove that the sum of the first n odd integers is
                                                                             Yeah!
Base case (n=1): the sum of the first 1 odd integer is
Assume p (k): the sum of the first k odd integers is                           =1

Where,
         1 + 3 + … + (2k+1) =
Prove that
         1 + 3 + … + + (2k-1) + (2k+1) =
         1 + 3 + … + + (2k-1) + (2k+1) =
                                            =



                                                                                                38
Prove that:                 1 x 1! + 2 x 2! + … + n x n! = (n+1)! -1, ∀ n
Base case (n=1):                                  1 x 1! = (1 x 1)! -1?      1 x 1! = 1
Assume P (k):               1 x 1! + 2 x 2! + … + k x k! = (k+1)! -1
                                                                             2! – 1 = 1
Prove that: 1 x 1! + 2 x 2! + … + k x k! + (k+1) (k+1)! = (k+2)! -1
              1 x 1! + 2 x 2! + … + k x k! + (k+1) (k+1)! = (k+1)! -1+ (k+1) (k+1)
                                                         = (1 + (k+1)) (k+1)! – 1
                                                         = (k+2) (k+1)! -1
                                                         = (k+2)! - 1




                                                                                          39
EXERCISE:



  1. For every n ≥ 4, n! >


  2. Proof that,


     We have seen that for any natural number n ,
                             1 + 2 + ... + n = n( n + 1 )/2
     and
                             12 + 22 + ... + n2 = n( n + 1 )( 2n + 1 )/6
     hold.




                                                                           40
ANSWER:


  1. Proof:
     In this problem          .
     Basis Step: If n = 4, then LHS = 4! = 24, and RHS =               .
     Hence LHS > RHS .


     Induction: Assume that n! >          for an arbitrary n ≥ 4 . -- Induction Hypothesis


     To prove that this inequality holds for n+1, first try to express LHS for n+1 in terms of
     LHS for n and try to use the induction hypothesis.
     Note here (n + 1)! = (n + 1) n!
     Thus using the induction hypothesis, we get (n + 1)! = (n + 1)n! > (n + 1)       .


     Since n ≥ 4 , (n+1) > 2.


     Hence, (n + 1)      >            .


     Hence, (n + 1)! >            .


  2. One might then wonder what 13 + 23 + ... + n3 would be equal to.


     One way to find that out is to make a conjecture (i.e. educated guess) and prove the
     conjecture.


     Let us first take a guess.
     By looking at the sums 1 + 2 + ... + n = n( n + 1 )/2 --- a function of n2
     and 12 + 22 + ... + n2 = n( n + 1 )( 2n + 1 )/6 --- a function of n3 ,
     one can guess that 13 + 23 + ... + n3 is equal to some function of n4, that is
     13 + 23 + ... + n3 = an4 + bn3 + cn2 + dn + e ---- (1) for some constants a, b, c, d and e.



                                                                                                   41
Now to determine the value of a, b, c, d and e, we compare the value of the both sides of
the equation (1) for five values of n.
For n = 0, LHS = 0, and RHS = e. Hence we get e = 0.
Similarly for n = 1, 1 = a + b + c + d,
for n = 2, 9 = 16a + 8b + 4c + 2d,
for n = 3, 36 = 81a + 27b + 9c + 3d , and
for n = 4, 100 = 256a + 64b + 16c + 4d .


Solving this system of equations we obtain
a = c = 1/4, b = 1/2, and d = 0.
Hence our conjecture is
13 + 23 + ... + n3 = 1/4 n2 ( n2 + 2n + 1 ) = ( 1/2 n ( n + 1 ) )2 .


What we do next is to try to prove it by mathematical induction.


Proof by Mathematical Induction:
Basis Step: For n = 0, LHS = 03 = 0 , and
RHS = ( 1/2* 0 ( 0 + 1 ) )2 = 0 .
Hence LHS = RHS.
Induction: Assume that 13 + 23 + ... + n3 = ( 1/2 n ( n + 1 ) )2 for an arbitrary n. ---------
Induction Hypothesis
Then for n + 1, LHS = 13 + 23 + ... + n3 + ( n + 1 )3
  = (13 + 23 + ... + n3) + ( n + 1 )3
  = ( 1/2 n ( n + 1 ) )2 + ( n + 1 )3 by the induction hypothesis.
  = ( 1/4 ( n + 1 )2( n2 + 4*( n + 1 ) )
  = ( 1/2 ( n + 1 )( n + 2 ) )2 ,
which is equal to RHS.
End of Proof


Thus we now know for sure that
13 + 23 + ... + n3 = ( 1/2 n ( n + 1 ) )2 .

                                                                                            42

Weitere ähnliche Inhalte

Was ist angesagt?

IJCER (www.ijceronline.com) International Journal of computational Engineerin...
IJCER (www.ijceronline.com) International Journal of computational Engineerin...IJCER (www.ijceronline.com) International Journal of computational Engineerin...
IJCER (www.ijceronline.com) International Journal of computational Engineerin...ijceronline
 
Lesson 16 The Spectral Theorem and Applications
Lesson 16  The Spectral Theorem and ApplicationsLesson 16  The Spectral Theorem and Applications
Lesson 16 The Spectral Theorem and ApplicationsMatthew Leingang
 
Brief summary of signals
Brief summary of signalsBrief summary of signals
Brief summary of signalsaroosa khan
 
Least squares support Vector Machine Classifier
Least squares support Vector Machine ClassifierLeast squares support Vector Machine Classifier
Least squares support Vector Machine ClassifierRaj Sikarwar
 
Testing for mixtures by seeking components
Testing for mixtures by seeking componentsTesting for mixtures by seeking components
Testing for mixtures by seeking componentsChristian Robert
 
Unit 1-logic
Unit 1-logicUnit 1-logic
Unit 1-logicraksharao
 
Kernel Lower Bounds
Kernel Lower BoundsKernel Lower Bounds
Kernel Lower BoundsASPAK2014
 
The Exponential Time Hypothesis
The Exponential Time HypothesisThe Exponential Time Hypothesis
The Exponential Time HypothesisASPAK2014
 
Omiros' talk on the Bernoulli factory problem
Omiros' talk on the  Bernoulli factory problemOmiros' talk on the  Bernoulli factory problem
Omiros' talk on the Bernoulli factory problemBigMC
 
Renyis entropy
Renyis entropyRenyis entropy
Renyis entropywtyru1989
 
Kolev skalna2018 article-exact_solutiontoa_parametricline
Kolev skalna2018 article-exact_solutiontoa_parametriclineKolev skalna2018 article-exact_solutiontoa_parametricline
Kolev skalna2018 article-exact_solutiontoa_parametriclineAlina Barbulescu
 
Aaex7 group2(中英夾雜)
Aaex7 group2(中英夾雜)Aaex7 group2(中英夾雜)
Aaex7 group2(中英夾雜)Shiang-Yun Yang
 
Variations on the method of Coleman-Chabauty
Variations on the method of Coleman-ChabautyVariations on the method of Coleman-Chabauty
Variations on the method of Coleman-Chabautymmasdeu
 
Lesson 32: The Fundamental Theorem Of Calculus
Lesson 32: The Fundamental Theorem Of CalculusLesson 32: The Fundamental Theorem Of Calculus
Lesson 32: The Fundamental Theorem Of CalculusMatthew Leingang
 
Coordinate sampler: A non-reversible Gibbs-like sampler
Coordinate sampler: A non-reversible Gibbs-like samplerCoordinate sampler: A non-reversible Gibbs-like sampler
Coordinate sampler: A non-reversible Gibbs-like samplerChristian Robert
 
Cs221 lecture4-fall11
Cs221 lecture4-fall11Cs221 lecture4-fall11
Cs221 lecture4-fall11darwinrlo
 

Was ist angesagt? (20)

IJCER (www.ijceronline.com) International Journal of computational Engineerin...
IJCER (www.ijceronline.com) International Journal of computational Engineerin...IJCER (www.ijceronline.com) International Journal of computational Engineerin...
IJCER (www.ijceronline.com) International Journal of computational Engineerin...
 
Lesson 16 The Spectral Theorem and Applications
Lesson 16  The Spectral Theorem and ApplicationsLesson 16  The Spectral Theorem and Applications
Lesson 16 The Spectral Theorem and Applications
 
Brief summary of signals
Brief summary of signalsBrief summary of signals
Brief summary of signals
 
Least squares support Vector Machine Classifier
Least squares support Vector Machine ClassifierLeast squares support Vector Machine Classifier
Least squares support Vector Machine Classifier
 
Testing for mixtures by seeking components
Testing for mixtures by seeking componentsTesting for mixtures by seeking components
Testing for mixtures by seeking components
 
O2
O2O2
O2
 
Unit 1-logic
Unit 1-logicUnit 1-logic
Unit 1-logic
 
Kernel Lower Bounds
Kernel Lower BoundsKernel Lower Bounds
Kernel Lower Bounds
 
Richard Everitt's slides
Richard Everitt's slidesRichard Everitt's slides
Richard Everitt's slides
 
The Exponential Time Hypothesis
The Exponential Time HypothesisThe Exponential Time Hypothesis
The Exponential Time Hypothesis
 
Omiros' talk on the Bernoulli factory problem
Omiros' talk on the  Bernoulli factory problemOmiros' talk on the  Bernoulli factory problem
Omiros' talk on the Bernoulli factory problem
 
Renyis entropy
Renyis entropyRenyis entropy
Renyis entropy
 
Kolev skalna2018 article-exact_solutiontoa_parametricline
Kolev skalna2018 article-exact_solutiontoa_parametriclineKolev skalna2018 article-exact_solutiontoa_parametricline
Kolev skalna2018 article-exact_solutiontoa_parametricline
 
Aaex7 group2(中英夾雜)
Aaex7 group2(中英夾雜)Aaex7 group2(中英夾雜)
Aaex7 group2(中英夾雜)
 
Variations on the method of Coleman-Chabauty
Variations on the method of Coleman-ChabautyVariations on the method of Coleman-Chabauty
Variations on the method of Coleman-Chabauty
 
Wg qcolorable
Wg qcolorableWg qcolorable
Wg qcolorable
 
Prml
PrmlPrml
Prml
 
Lesson 32: The Fundamental Theorem Of Calculus
Lesson 32: The Fundamental Theorem Of CalculusLesson 32: The Fundamental Theorem Of Calculus
Lesson 32: The Fundamental Theorem Of Calculus
 
Coordinate sampler: A non-reversible Gibbs-like sampler
Coordinate sampler: A non-reversible Gibbs-like samplerCoordinate sampler: A non-reversible Gibbs-like sampler
Coordinate sampler: A non-reversible Gibbs-like sampler
 
Cs221 lecture4-fall11
Cs221 lecture4-fall11Cs221 lecture4-fall11
Cs221 lecture4-fall11
 

Andere mochten auch (7)

Chapter 3
Chapter 3Chapter 3
Chapter 3
 
Dicrete structure
Dicrete structureDicrete structure
Dicrete structure
 
Chapter 4
Chapter 4Chapter 4
Chapter 4
 
Slide subtopic 4
Slide subtopic 4Slide subtopic 4
Slide subtopic 4
 
Slide subtopic 5
Slide subtopic 5Slide subtopic 5
Slide subtopic 5
 
Slide subtopic 1
Slide subtopic 1Slide subtopic 1
Slide subtopic 1
 
Slide subtopic 3
Slide subtopic 3Slide subtopic 3
Slide subtopic 3
 

Ähnlich wie Chapter 5

Chapter 4 dis 2011
Chapter 4 dis 2011Chapter 4 dis 2011
Chapter 4 dis 2011noraidawati
 
Induction.pptx
Induction.pptxInduction.pptx
Induction.pptxAppasamiG
 
Principle of mathematical induction
Principle of mathematical inductionPrinciple of mathematical induction
Principle of mathematical inductionKriti Varshney
 
17-mathematical-induction.ppt
17-mathematical-induction.ppt17-mathematical-induction.ppt
17-mathematical-induction.pptRishabhNath3
 
17-mathematical-induction.ppt
17-mathematical-induction.ppt17-mathematical-induction.ppt
17-mathematical-induction.pptSintaVeDe
 
DMA_Induction (2).pptx nnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnn
DMA_Induction (2).pptx nnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnDMA_Induction (2).pptx nnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnn
DMA_Induction (2).pptx nnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnhuong996275
 
11-Induction CIIT.pptx
11-Induction CIIT.pptx11-Induction CIIT.pptx
11-Induction CIIT.pptxjaffarbikat
 
Introduction to mathematical Induction.ppt
Introduction to mathematical Induction.pptIntroduction to mathematical Induction.ppt
Introduction to mathematical Induction.pptShaukatAliChaudhry1
 
Mathematical induction by Animesh Sarkar
Mathematical induction by Animesh SarkarMathematical induction by Animesh Sarkar
Mathematical induction by Animesh SarkarAnimesh Sarkar
 
CMSC 56 | Lecture 11: Mathematical Induction
CMSC 56 | Lecture 11: Mathematical InductionCMSC 56 | Lecture 11: Mathematical Induction
CMSC 56 | Lecture 11: Mathematical Inductionallyn joy calcaben
 
Math induction
Math inductionMath induction
Math inductionasel_d
 

Ähnlich wie Chapter 5 (20)

Chapter 4 dis 2011
Chapter 4 dis 2011Chapter 4 dis 2011
Chapter 4 dis 2011
 
Induction.pdf
Induction.pdfInduction.pdf
Induction.pdf
 
Induction.pptx
Induction.pptxInduction.pptx
Induction.pptx
 
Principle of mathematical induction
Principle of mathematical inductionPrinciple of mathematical induction
Principle of mathematical induction
 
Induction q
Induction qInduction q
Induction q
 
Induction q
Induction qInduction q
Induction q
 
6e-ch4.ppt
6e-ch4.ppt6e-ch4.ppt
6e-ch4.ppt
 
17-mathematical-induction.ppt
17-mathematical-induction.ppt17-mathematical-induction.ppt
17-mathematical-induction.ppt
 
17-mathematical-induction.ppt
17-mathematical-induction.ppt17-mathematical-induction.ppt
17-mathematical-induction.ppt
 
DMA_Induction (2).pptx nnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnn
DMA_Induction (2).pptx nnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnDMA_Induction (2).pptx nnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnn
DMA_Induction (2).pptx nnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnnn
 
11-Induction CIIT.pptx
11-Induction CIIT.pptx11-Induction CIIT.pptx
11-Induction CIIT.pptx
 
Introduction to mathematical Induction.ppt
Introduction to mathematical Induction.pptIntroduction to mathematical Induction.ppt
Introduction to mathematical Induction.ppt
 
Induction (1).ppt
Induction (1).pptInduction (1).ppt
Induction (1).ppt
 
Mathematical induction by Animesh Sarkar
Mathematical induction by Animesh SarkarMathematical induction by Animesh Sarkar
Mathematical induction by Animesh Sarkar
 
CMSC 56 | Lecture 11: Mathematical Induction
CMSC 56 | Lecture 11: Mathematical InductionCMSC 56 | Lecture 11: Mathematical Induction
CMSC 56 | Lecture 11: Mathematical Induction
 
Math induction
Math inductionMath induction
Math induction
 
Discrete Math Lecture 03: Methods of Proof
Discrete Math Lecture 03: Methods of ProofDiscrete Math Lecture 03: Methods of Proof
Discrete Math Lecture 03: Methods of Proof
 
one + 1
one + 1one + 1
one + 1
 
An engineer 1+1=2
An engineer 1+1=2An engineer 1+1=2
An engineer 1+1=2
 
Mathematical Induction DM
Mathematical Induction DMMathematical Induction DM
Mathematical Induction DM
 

Mehr von Eli Lilly and Company (14)

Slide subtopic 2
Slide subtopic 2Slide subtopic 2
Slide subtopic 2
 
Slide subtopic 2
Slide subtopic 2Slide subtopic 2
Slide subtopic 2
 
Chapter 1
Chapter 1Chapter 1
Chapter 1
 
Chapter 1
Chapter 1Chapter 1
Chapter 1
 
Akses dan ekuiti
Akses dan ekuitiAkses dan ekuiti
Akses dan ekuiti
 
Isu profesional guru dalam pengajaran matematik
Isu profesional guru dalam pengajaran matematikIsu profesional guru dalam pengajaran matematik
Isu profesional guru dalam pengajaran matematik
 
kurikulum dan kelainan upaya
kurikulum dan kelainan upayakurikulum dan kelainan upaya
kurikulum dan kelainan upaya
 
jantina dan bangsa
jantina dan bangsajantina dan bangsa
jantina dan bangsa
 
jantina dan bangsa
jantina dan bangsajantina dan bangsa
jantina dan bangsa
 
Jantina dan bangsa
Jantina dan bangsaJantina dan bangsa
Jantina dan bangsa
 
ISU JANTINA
ISU JANTINAISU JANTINA
ISU JANTINA
 
Qayyum
QayyumQayyum
Qayyum
 
Trend kurikulum
Trend kurikulumTrend kurikulum
Trend kurikulum
 
Isu profesional guru dalam pengajaran matematik
Isu profesional guru dalam pengajaran matematikIsu profesional guru dalam pengajaran matematik
Isu profesional guru dalam pengajaran matematik
 

Kürzlich hochgeladen

4.11.24 Mass Incarceration and the New Jim Crow.pptx
4.11.24 Mass Incarceration and the New Jim Crow.pptx4.11.24 Mass Incarceration and the New Jim Crow.pptx
4.11.24 Mass Incarceration and the New Jim Crow.pptxmary850239
 
Mythology Quiz-4th April 2024, Quiz Club NITW
Mythology Quiz-4th April 2024, Quiz Club NITWMythology Quiz-4th April 2024, Quiz Club NITW
Mythology Quiz-4th April 2024, Quiz Club NITWQuiz Club NITW
 
How to Make a Duplicate of Your Odoo 17 Database
How to Make a Duplicate of Your Odoo 17 DatabaseHow to Make a Duplicate of Your Odoo 17 Database
How to Make a Duplicate of Your Odoo 17 DatabaseCeline George
 
Daily Lesson Plan in Mathematics Quarter 4
Daily Lesson Plan in Mathematics Quarter 4Daily Lesson Plan in Mathematics Quarter 4
Daily Lesson Plan in Mathematics Quarter 4JOYLYNSAMANIEGO
 
ARTERIAL BLOOD GAS ANALYSIS........pptx
ARTERIAL BLOOD  GAS ANALYSIS........pptxARTERIAL BLOOD  GAS ANALYSIS........pptx
ARTERIAL BLOOD GAS ANALYSIS........pptxAneriPatwari
 
Expanded definition: technical and operational
Expanded definition: technical and operationalExpanded definition: technical and operational
Expanded definition: technical and operationalssuser3e220a
 
Decoding the Tweet _ Practical Criticism in the Age of Hashtag.pptx
Decoding the Tweet _ Practical Criticism in the Age of Hashtag.pptxDecoding the Tweet _ Practical Criticism in the Age of Hashtag.pptx
Decoding the Tweet _ Practical Criticism in the Age of Hashtag.pptxDhatriParmar
 
Reading and Writing Skills 11 quarter 4 melc 1
Reading and Writing Skills 11 quarter 4 melc 1Reading and Writing Skills 11 quarter 4 melc 1
Reading and Writing Skills 11 quarter 4 melc 1GloryAnnCastre1
 
Using Grammatical Signals Suitable to Patterns of Idea Development
Using Grammatical Signals Suitable to Patterns of Idea DevelopmentUsing Grammatical Signals Suitable to Patterns of Idea Development
Using Grammatical Signals Suitable to Patterns of Idea Developmentchesterberbo7
 
MS4 level being good citizen -imperative- (1) (1).pdf
MS4 level   being good citizen -imperative- (1) (1).pdfMS4 level   being good citizen -imperative- (1) (1).pdf
MS4 level being good citizen -imperative- (1) (1).pdfMr Bounab Samir
 
Team Lead Succeed – Helping you and your team achieve high-performance teamwo...
Team Lead Succeed – Helping you and your team achieve high-performance teamwo...Team Lead Succeed – Helping you and your team achieve high-performance teamwo...
Team Lead Succeed – Helping you and your team achieve high-performance teamwo...Association for Project Management
 
Grade Three -ELLNA-REVIEWER-ENGLISH.pptx
Grade Three -ELLNA-REVIEWER-ENGLISH.pptxGrade Three -ELLNA-REVIEWER-ENGLISH.pptx
Grade Three -ELLNA-REVIEWER-ENGLISH.pptxkarenfajardo43
 
Sulphonamides, mechanisms and their uses
Sulphonamides, mechanisms and their usesSulphonamides, mechanisms and their uses
Sulphonamides, mechanisms and their usesVijayaLaxmi84
 
DIFFERENT BASKETRY IN THE PHILIPPINES PPT.pptx
DIFFERENT BASKETRY IN THE PHILIPPINES PPT.pptxDIFFERENT BASKETRY IN THE PHILIPPINES PPT.pptx
DIFFERENT BASKETRY IN THE PHILIPPINES PPT.pptxMichelleTuguinay1
 
Q4-PPT-Music9_Lesson-1-Romantic-Opera.pptx
Q4-PPT-Music9_Lesson-1-Romantic-Opera.pptxQ4-PPT-Music9_Lesson-1-Romantic-Opera.pptx
Q4-PPT-Music9_Lesson-1-Romantic-Opera.pptxlancelewisportillo
 
How to Manage Buy 3 Get 1 Free in Odoo 17
How to Manage Buy 3 Get 1 Free in Odoo 17How to Manage Buy 3 Get 1 Free in Odoo 17
How to Manage Buy 3 Get 1 Free in Odoo 17Celine George
 
Grade 9 Quarter 4 Dll Grade 9 Quarter 4 DLL.pdf
Grade 9 Quarter 4 Dll Grade 9 Quarter 4 DLL.pdfGrade 9 Quarter 4 Dll Grade 9 Quarter 4 DLL.pdf
Grade 9 Quarter 4 Dll Grade 9 Quarter 4 DLL.pdfJemuel Francisco
 
Blowin' in the Wind of Caste_ Bob Dylan's Song as a Catalyst for Social Justi...
Blowin' in the Wind of Caste_ Bob Dylan's Song as a Catalyst for Social Justi...Blowin' in the Wind of Caste_ Bob Dylan's Song as a Catalyst for Social Justi...
Blowin' in the Wind of Caste_ Bob Dylan's Song as a Catalyst for Social Justi...DhatriParmar
 

Kürzlich hochgeladen (20)

4.11.24 Mass Incarceration and the New Jim Crow.pptx
4.11.24 Mass Incarceration and the New Jim Crow.pptx4.11.24 Mass Incarceration and the New Jim Crow.pptx
4.11.24 Mass Incarceration and the New Jim Crow.pptx
 
Mythology Quiz-4th April 2024, Quiz Club NITW
Mythology Quiz-4th April 2024, Quiz Club NITWMythology Quiz-4th April 2024, Quiz Club NITW
Mythology Quiz-4th April 2024, Quiz Club NITW
 
Paradigm shift in nursing research by RS MEHTA
Paradigm shift in nursing research by RS MEHTAParadigm shift in nursing research by RS MEHTA
Paradigm shift in nursing research by RS MEHTA
 
How to Make a Duplicate of Your Odoo 17 Database
How to Make a Duplicate of Your Odoo 17 DatabaseHow to Make a Duplicate of Your Odoo 17 Database
How to Make a Duplicate of Your Odoo 17 Database
 
Daily Lesson Plan in Mathematics Quarter 4
Daily Lesson Plan in Mathematics Quarter 4Daily Lesson Plan in Mathematics Quarter 4
Daily Lesson Plan in Mathematics Quarter 4
 
ARTERIAL BLOOD GAS ANALYSIS........pptx
ARTERIAL BLOOD  GAS ANALYSIS........pptxARTERIAL BLOOD  GAS ANALYSIS........pptx
ARTERIAL BLOOD GAS ANALYSIS........pptx
 
INCLUSIVE EDUCATION PRACTICES FOR TEACHERS AND TRAINERS.pptx
INCLUSIVE EDUCATION PRACTICES FOR TEACHERS AND TRAINERS.pptxINCLUSIVE EDUCATION PRACTICES FOR TEACHERS AND TRAINERS.pptx
INCLUSIVE EDUCATION PRACTICES FOR TEACHERS AND TRAINERS.pptx
 
Expanded definition: technical and operational
Expanded definition: technical and operationalExpanded definition: technical and operational
Expanded definition: technical and operational
 
Decoding the Tweet _ Practical Criticism in the Age of Hashtag.pptx
Decoding the Tweet _ Practical Criticism in the Age of Hashtag.pptxDecoding the Tweet _ Practical Criticism in the Age of Hashtag.pptx
Decoding the Tweet _ Practical Criticism in the Age of Hashtag.pptx
 
Reading and Writing Skills 11 quarter 4 melc 1
Reading and Writing Skills 11 quarter 4 melc 1Reading and Writing Skills 11 quarter 4 melc 1
Reading and Writing Skills 11 quarter 4 melc 1
 
Using Grammatical Signals Suitable to Patterns of Idea Development
Using Grammatical Signals Suitable to Patterns of Idea DevelopmentUsing Grammatical Signals Suitable to Patterns of Idea Development
Using Grammatical Signals Suitable to Patterns of Idea Development
 
MS4 level being good citizen -imperative- (1) (1).pdf
MS4 level   being good citizen -imperative- (1) (1).pdfMS4 level   being good citizen -imperative- (1) (1).pdf
MS4 level being good citizen -imperative- (1) (1).pdf
 
Team Lead Succeed – Helping you and your team achieve high-performance teamwo...
Team Lead Succeed – Helping you and your team achieve high-performance teamwo...Team Lead Succeed – Helping you and your team achieve high-performance teamwo...
Team Lead Succeed – Helping you and your team achieve high-performance teamwo...
 
Grade Three -ELLNA-REVIEWER-ENGLISH.pptx
Grade Three -ELLNA-REVIEWER-ENGLISH.pptxGrade Three -ELLNA-REVIEWER-ENGLISH.pptx
Grade Three -ELLNA-REVIEWER-ENGLISH.pptx
 
Sulphonamides, mechanisms and their uses
Sulphonamides, mechanisms and their usesSulphonamides, mechanisms and their uses
Sulphonamides, mechanisms and their uses
 
DIFFERENT BASKETRY IN THE PHILIPPINES PPT.pptx
DIFFERENT BASKETRY IN THE PHILIPPINES PPT.pptxDIFFERENT BASKETRY IN THE PHILIPPINES PPT.pptx
DIFFERENT BASKETRY IN THE PHILIPPINES PPT.pptx
 
Q4-PPT-Music9_Lesson-1-Romantic-Opera.pptx
Q4-PPT-Music9_Lesson-1-Romantic-Opera.pptxQ4-PPT-Music9_Lesson-1-Romantic-Opera.pptx
Q4-PPT-Music9_Lesson-1-Romantic-Opera.pptx
 
How to Manage Buy 3 Get 1 Free in Odoo 17
How to Manage Buy 3 Get 1 Free in Odoo 17How to Manage Buy 3 Get 1 Free in Odoo 17
How to Manage Buy 3 Get 1 Free in Odoo 17
 
Grade 9 Quarter 4 Dll Grade 9 Quarter 4 DLL.pdf
Grade 9 Quarter 4 Dll Grade 9 Quarter 4 DLL.pdfGrade 9 Quarter 4 Dll Grade 9 Quarter 4 DLL.pdf
Grade 9 Quarter 4 Dll Grade 9 Quarter 4 DLL.pdf
 
Blowin' in the Wind of Caste_ Bob Dylan's Song as a Catalyst for Social Justi...
Blowin' in the Wind of Caste_ Bob Dylan's Song as a Catalyst for Social Justi...Blowin' in the Wind of Caste_ Bob Dylan's Song as a Catalyst for Social Justi...
Blowin' in the Wind of Caste_ Bob Dylan's Song as a Catalyst for Social Justi...
 

Chapter 5

  • 1. SUBTOPIC 5 : MATHEMATICAL INDUCTION Mathematical induction can be used to prove statements that assert that ∀ n ∈ , P (n) is true. But, it is important to note that mathematical induction can be used only to prove results obtained in some other way. It is not a tool for discovering formula or theorem. Principle of Induction. To prove that P (n) is true for all positive integers n, where P (n) is a propositional function. A proof by mathematical induction has two parts: Basic step: We verify that P (1) is true. Inductive step: We show that the conditional proposition ∀ k ∈ , P (k) ⇒ P (k + 1) is true. In the induction step, the assumption that P (n) holds is called the Induction Hypothesis (IH). In more formal notation, this proof technique can be stated as [P (0) ˄∀ k (P (k) ⇒ P (k + 1) ∀n P (n) You can think of the proof by (mathematical) induction as a kind of recursive proof: Instead of attacking the problem directly, we only explain how to get a proof for P(n + 1) out of a proof for P(n). How would you prove that the proof by induction indeed works?? Proof (by contradiction) Assume that for some values of n, P(n) is false. Let be the least such n that P_n0_ is false. Cannot be 0, because P(0) is true. Thus, must be in the form =1 + . Since < then by P ( is true. Therefore, by inductive hypothesis P ( + 1) must be true. It follows then that P ( is true. 33
  • 2. The base case can start with any nonnegative number. If that number is then you would prove that assertion P(n) holds for all n ≥ . [P ( ) ˄∀ k ≥ (P (k) ⇒ P (k + 1) ∀n P (n) The induction step not necessarily should start with n. You can change the step from n -1 to n, where n > 0. Sometimes this yields slightly shorter expressions. However, you cannot make a step from n - 1 to n + 1. Example: Prove for ≥ 1 1 x 1! + 2 x 2! + 3 x 3! + ... + n x n! = (n + 1)! - 1 This could be also written by using ∑ notation If you take 15-355 (http://www.andrew.cmu.edu/course/15-355/) you will learn a more general approach for deriving and proving combinatorial identities. Proof Base case: n _ 1 The left hand side is 1x1! The right hand side is 2! - 1. They are equal. Inductive hypothesis: Suppose this holds We need to prove 34
  • 3. Consider the left hand side (n+1)! – 1 + (n+1) x (n+1) = (n+1)! (1+n+1) -1 = (n+2)! -1 Suppose we have a sequence of propositions which we would like to prove: P (0), P (1), P (2), P (3)… P (n) We can picture each proposition as a domino: P (k) A sequence of propositions is visualized as a sequence of dominos. P (0) P (1) P (2) P (k) P ….. (k+1) When the domino falls (to right), the corresponding proposition is considered true: 35
  • 4. P (k) true Suppose that the dominos satisfy two constraints. 1. Well positioned: if any domino falls to right, the next domino to right must fall also. P (k) P true (k+1) true 2. First domino has fallen to right. P (0) true Than can conclude that all the domino fall. P (0) P (1) P (2) P (k) P ….. (k+1) P (0) P (1) P (2) P (k) P ….. (k+1) true 36
  • 5. P (1) P (2) P (k) P ….. (k+1) P (0) true true true P (2) P (k) P ….. (k+1) P (0) true P (1) true True true P (k) P ….. (k+1) P (0) true P (1) true P (2) true P (k) P ….. (k+1) P (0) true P (1) true P (2) true true true 37
  • 6. P (0) true P (1) true P (2) true true ….. P (k) true P (k+1) true Principle of Mathematical Induction. If: 1. Basis P(1) is true 2. Induction ∀ n P(k) P(k+1) is true P (0) true P (1) true P (2) true true ….. P (k) true P (k+1) true Then, ∀ n P (n) is true. Use induction to prove that the sum of the first n odd integers is Yeah! Base case (n=1): the sum of the first 1 odd integer is Assume p (k): the sum of the first k odd integers is =1 Where, 1 + 3 + … + (2k+1) = Prove that 1 + 3 + … + + (2k-1) + (2k+1) = 1 + 3 + … + + (2k-1) + (2k+1) = = 38
  • 7. Prove that: 1 x 1! + 2 x 2! + … + n x n! = (n+1)! -1, ∀ n Base case (n=1): 1 x 1! = (1 x 1)! -1? 1 x 1! = 1 Assume P (k): 1 x 1! + 2 x 2! + … + k x k! = (k+1)! -1 2! – 1 = 1 Prove that: 1 x 1! + 2 x 2! + … + k x k! + (k+1) (k+1)! = (k+2)! -1 1 x 1! + 2 x 2! + … + k x k! + (k+1) (k+1)! = (k+1)! -1+ (k+1) (k+1) = (1 + (k+1)) (k+1)! – 1 = (k+2) (k+1)! -1 = (k+2)! - 1 39
  • 8. EXERCISE: 1. For every n ≥ 4, n! > 2. Proof that, We have seen that for any natural number n , 1 + 2 + ... + n = n( n + 1 )/2 and 12 + 22 + ... + n2 = n( n + 1 )( 2n + 1 )/6 hold. 40
  • 9. ANSWER: 1. Proof: In this problem . Basis Step: If n = 4, then LHS = 4! = 24, and RHS = . Hence LHS > RHS . Induction: Assume that n! > for an arbitrary n ≥ 4 . -- Induction Hypothesis To prove that this inequality holds for n+1, first try to express LHS for n+1 in terms of LHS for n and try to use the induction hypothesis. Note here (n + 1)! = (n + 1) n! Thus using the induction hypothesis, we get (n + 1)! = (n + 1)n! > (n + 1) . Since n ≥ 4 , (n+1) > 2. Hence, (n + 1) > . Hence, (n + 1)! > . 2. One might then wonder what 13 + 23 + ... + n3 would be equal to. One way to find that out is to make a conjecture (i.e. educated guess) and prove the conjecture. Let us first take a guess. By looking at the sums 1 + 2 + ... + n = n( n + 1 )/2 --- a function of n2 and 12 + 22 + ... + n2 = n( n + 1 )( 2n + 1 )/6 --- a function of n3 , one can guess that 13 + 23 + ... + n3 is equal to some function of n4, that is 13 + 23 + ... + n3 = an4 + bn3 + cn2 + dn + e ---- (1) for some constants a, b, c, d and e. 41
  • 10. Now to determine the value of a, b, c, d and e, we compare the value of the both sides of the equation (1) for five values of n. For n = 0, LHS = 0, and RHS = e. Hence we get e = 0. Similarly for n = 1, 1 = a + b + c + d, for n = 2, 9 = 16a + 8b + 4c + 2d, for n = 3, 36 = 81a + 27b + 9c + 3d , and for n = 4, 100 = 256a + 64b + 16c + 4d . Solving this system of equations we obtain a = c = 1/4, b = 1/2, and d = 0. Hence our conjecture is 13 + 23 + ... + n3 = 1/4 n2 ( n2 + 2n + 1 ) = ( 1/2 n ( n + 1 ) )2 . What we do next is to try to prove it by mathematical induction. Proof by Mathematical Induction: Basis Step: For n = 0, LHS = 03 = 0 , and RHS = ( 1/2* 0 ( 0 + 1 ) )2 = 0 . Hence LHS = RHS. Induction: Assume that 13 + 23 + ... + n3 = ( 1/2 n ( n + 1 ) )2 for an arbitrary n. --------- Induction Hypothesis Then for n + 1, LHS = 13 + 23 + ... + n3 + ( n + 1 )3 = (13 + 23 + ... + n3) + ( n + 1 )3 = ( 1/2 n ( n + 1 ) )2 + ( n + 1 )3 by the induction hypothesis. = ( 1/4 ( n + 1 )2( n2 + 4*( n + 1 ) ) = ( 1/2 ( n + 1 )( n + 2 ) )2 , which is equal to RHS. End of Proof Thus we now know for sure that 13 + 23 + ... + n3 = ( 1/2 n ( n + 1 ) )2 . 42