Advanced Calculus: MATH 410 Riemann Integrals and Integrability
Advanced Calculus: MATH 410 Riemann Integrals and Integrability
                        1. Definite Integrals
  In this section we revisit the definite integral that you were intro-
duced to when you first studied calculus. You undoubtedly learned that
given a positive function f over an interval [a, b] the definite integral
                              Z b
                                  f (x) dx ,
                                 a
provided it was defined, was a number equal to the area under the
graph of f over [a, b]. You also likely learned that the definite integral
was defined as a limit of Riemann sums. The Riemann sums you most
likely used involved partitioning [a, b] into n uniform subintervals of
length (b  a)/n and evaluating f at either the right-hand endpoint,
the left-hand endpoint, or the midpoint of each subinterval. At the
time your understanding of the notion of limit was likely more intu-
itive than rigorous. In this section we present the Riemann Integral,
a rigorous development of the definite integral built upon the rigorous
understanding of limit that you have studied earlier in this course.
                                                                                       
4
splits the task of evaluating a definite integrals into two steps. The
first step is by far the easier. It is a rare integrand f for which one can
find a sequence of Darboux or Riemann sums that allows one of the
limits (17) or (18) to be evaluated directly.
Proof. If f is Riemann integrable over [a, b] then one can use character-
ization (2) of the Riemann-Darboux Theorem to construct a sequence
of partitions that satisfies (16), and is thereby Archimedean for f . Con-
versely, given a sequence of partitions of [a, b] that is Archimedean for
f , then the fact that f is integrable over [a, b] follows directly from
characterization (2) of the Riemann-Darboux Theorem. The details of
these arguments are left as an exercise.
   We now establish the limits (17) and (18). Let {P n }  n=1 be a sequence
of partitions of [a, b] that is Archimedean for f and let {Qn }    n=1 be a
sequence of associated quadrature points. The bounds on Riemann
sums given by (15) yield the inequalities
                  L(f, P n )  R(f, P n , Qn )  U (f, P n ) ,
while, because f is Riemann integrable, we also have the inequalities
                               Z b
                          n
                    L(f, P )      f  U (f, P n ) .
                                      a
It follows from these inequalities that
                                           Z       b
           n            n             n
    L(f, P )  U (f, P )  L(f, P )          f
                                               a
                                               Z b
                                     n   n
                             R(f, P , Q )        f
                                                a
                                          Z b
                                     n
                             U (f, P )      f  U (f, P n )  L(f, P n ) ,
                                               a
which implies that
                              Z b 
                                    
                L(f, P n )      f    U (f, P n )  L(f, P n ) ,
                                    
                                a
                              Z b 
                                    
            R(f, P n , Qn )     f    U (f, P n )  L(f, P n ) ,
                                    
                                a
                              Z b 
                                    
                U (f, P n )     f   U (f, P n )  L(f, P n ) .
                
                                  a
Proof. Let  > 0. There exist partitions PL and PU of [a, b] such that
                                                                     
       0  L(f )  L(f, PL ) < ,          0  U (f, PU )  U (f ) < .
                                   2                                  2
Let P = PL  PU . Let n be the number of subintervals in P  . Pick
                           
                                        + L(f, P  )  L(f, P ) ,
                                                                 
(20)
             0  U (f, P )  U (f ) = U (f, P  )  U (f )
                                                            
                                        + U (f, P )  U (f, P  ) .
                                                                 
We will prove the theorem by showing that each of the four terms in
parentheses on the right-hand sides above is less than /2.
  Because P  is a refinement of P  , which is a refinement of both PL
and PU , the Refinement Lemma implies that
              0  L(f )  L(f, P  )  L(f )  L(f, P  )
                                                                 
                                       L(f )  L(f, PL ) <       ,
                                                                 2
             0  U (f, P  )  U (f )  U (f, P  )  U (f )
                                                              
                                       U (f, PU )  U (f ) <  .
                                                              2
Thus, the first terms on the right-hand sides of (20) are less than /2.
  Because P  is a refinement of P , for each i = 1,    , n we let Pi de-
note the partition of [xi1 , xi ] induced by P  . The Refinement Lemma
10
then yields
                                     n
                                     X
       0  L(f, P  )  L(f, P ) =         L(f, Pi )  mi (xi  xi1 ) ,
                                                                      
                                     i=1
                                     n
                                     X
       0  U (f, P )  U (f, P  ) =    mi (xi  xi1 )  U (f, Pi ) .
                                                                    
                                     i=1
                            
Because P has at most n  1 partition points that are not partition
points of P , there are at most n 1 indices i for which [xi1 , xi ] contains
at least one partition point of Pi within (xi1 , xi ). For all other indices
the terms in the above sums are zero. Each of the nonzero terms in
the above sums satisfy the bounds
        0  mi (xi  xi1 )  U (f, Pi )  2M (xi  xi1 ) < 2M  ,
        0  L(f, Pi )  mi (xi  xi1 )  2M (xi  xi1 ) < 2M  .
Because there are at most n  1 such terms, we obtain the bounds
                                                        
                 0  U (f, P )  U (f, P  ) < n 2M  < ,
                                                        2
                                                      
                 0  L(f, P )  L(f, P ) < n 2M  < .
                                                        2
This shows the second terms on the right-hand sides of (20) are each
less than /2, thereby completing the proof of the lemma.         
  An immediate consequence of the Partitions Lemma is the following
characterization of Riemann integrable functions.
Theorem 1.3. (Darboux) Let f : [a, b]  R be bounded. Then f
Riemann integrable over [a, b] if and only if for every  > 0 there exists
a  > 0 such that for every partition P of [a, b] one has
               |P | <    =      0  U (f, P )  L(f, P ) <  .
Proof. The direction (=) follows from the Riemann-Darboux The-
orem. The direction (=) follows from the definition of the Riemann
integral and the Partitions Lemma. The details of the proof are left as
an exercise.                                                         
  An immediate consequence of the Darboux Theorem is that there a
simple criterion for a sequence of partitions to be Archimedean for any
Riemann integrable function.
Theorem 1.4. (Archimedean Sequence) Every sequence {P n }            n=1
of partitions of [a, b] such that |P n |  0 as n   is Archimedean for
every function f : [a, b]  R that is Riemann integrable over [a, b].
                                                                            11
Proof. Exercise.                                                            
Remark. The condition that |P n |  0 as n   is not necessary for a
sequence {P n }
               n=1 of partitions to be Archimedean. For example, every
sequence of partitions is Archimedean for every constant function.
  The Partitions Lemma also leads to a useful characterization of Rie-
mann integrable functions in terms of limits of Riemann sums. The
key step towards this characterization is taken by the following lemma.
Lemma 1.5. Let f : [a, b]  R be bounded. Let {P n }         n=1 be any
sequence of partitions of [a, b] such that |P n |  0 as n  . Then
(21)      lim L(f, P n ) = L(f ) ,           lim U (f, P n ) = U (f ) .
          n                               n
Proof. The proof of (21) follows from the Partitions Lemma. To prove
(22), it follows from (5) that for each partition P n there exist sets of
associated quadrature points QnL and QnU such that
                                                        1
                   0  R(f, P n , QnL )  L(f, P n ) < n ,
                                                       2
                                                        1
                   0  U (f, P n )  R(f, P n , QnU ) < n .
                                                       2
The details of the proof are left as an exercise.                      
  An immediate consequence of the previous lemma is the following
characterization of Riemann integrable functions in terms of limits of
Riemann sums.
Theorem 1.5. Let f : [a, b]  R be bounded. Let {P n }     n=1 be any
                                             n
sequence of partitions of [a, b] such that |P |  0 as n  . Suppose
that there exists a unique A  R such that for every sequence {Q n }
                                                                    n=1
of associated quadrature points one has
(23)                     lim R(f, P n , Qn ) = A .
                         n
Proof. Exercise.                                                            
12
We thereby obtain
                                                n
                                                X
          0  U (f, P )  L(f, P ) =                  (mi  mi ) (xi  xi1 )
                                                i=1
                     n
                     X                                n
                                                      X                    
             |P |         (mi  mi ) = |P |            f (xi )  f (xi1 ) ,
                     i=1                              i=1
2.3.1. Linearity. One basic fact about Riemann integrals is that they
depend linearly on the integrand. This fact is not completely trivial
because we defined the Riemann integral through Darboux sums, which
do not depend linearly on the integrand.
with
                                    n
                                                   !       n
                        Z       b   X                      X          Z       b
                                          k f k       =         k               fk .
                            a       k=1                    k=1            a
16
Proof. Exercise.
Proof. Exercise.
2.3.4. Bounds. The basic bounds on definite integrals now follows from
Proposition 2.3.
Moreover,
                       Z b 
                             
                       
                          f   M (b  a) ,
                         a
                                 	
where M = sup |f (x)| : x  [a, b] .
Proof. Exercise.                                                       
                                                                                  17
  We now show that the sum over the bad set I is small because
the partition P is refined enough to make the set I sufficiently small.
Indeed, because   mi  mi for every i  I , we have
           X                 X
             (xi  xi1 )     (mi  mi )(xi  xi1 )
            iI               iI
                                                            
                              U (f, P )  L(f, P ) <             ,
                                                        2(m  m )
whereby the set I is small in the sense that
                   X                        
                       (xi  xi1 ) <           .
                   iI
                                      2(m  m )
                         
         0  U (G(f ), P )  L(G(f ), P )
             X                             X
           =    (mi  mi )(xi  xi1 ) +   (mi  mi )(xi  xi1 )
             iI<                          iI
                
         < + = .
            2 2
Because  was arbitrary, G(f ) is Riemann integrable by characteriza-
tion (2) of the Riemann-Darboux Theorem.                           
  An important consequence of the Composition Theorem is that the
product of Riemann integrable functions is also Riemann integrable.
Proposition 2.5. (Product) Let f : [a, b]  R and g : [a, b]  R
be Riemann integrable over [a, b]. Then the product f g : [a, b]  R is
Riemann integrable over [a, b].
Remark. Taken together the Linearity and Product Propositions show
that the class of Riemann integrable functions is an algebra.
Proof. The proof is based on the algebraic identity
                     f g = 14 (f + g)2  (f  g)2 .
                                                 
                                                                       19
or the identity
                              1
                                  f 2 + g 2  (f  g)2 .
                                                      
                     fg =     2
   One can use Riemann sums to establish (29). This part of the proof
is left as an exercise.                                            
  The restriction a < b < c in the interval additivity formula (28) can
be dropped provided one adopts the following convention.
Definition 2.2. Let f : [a, b]  R be Riemann integrable over [a, b].
Define                    Z a       Z b
                               f =     f.
                              b             a
Proof. Let  > 0. Let Range(f)  [m, m]. Let  > 0 such that
                                                     ba
                  (m  m) <          and        <       .
                               3                       2
Because the restriction of f to [a + , b  ] is Riemann integrable, there
exists a partition P of [a + , b  ] such that
                                                    
                      0  U (f, P )  L(f, P ) < .
                                                    3
Let P  be the extension of P to [a, b] obtained by adding a and b as
partition points. Then
     0  U (f, P  )  L(f, P  )
       = U (f, [a, a + ])  L(f, [a, a + ]) + U (f, P )  L(f, P )
                                                                         
                         
        (m  m) + + (m  m) <  .
                         3
Hence, the extension f is Riemann integrable over [a, b] by characteri-
zation (2) of the Riemann-Darboux Theorem.
  Now let f1 and f2 be two extensions of f to [a, b]. Let {P n }        n=1 be
any sequence of partitions of [a, b] such that |P n |  0 as n  .
This sequence is Archimedean for both f1 and f2 by Theorem 1.4. Let
{Qn }
     n=1 be any sequence of associated quadrature points such that
neither a nor b are quadrature points. Because f1 (x) = f2 (x) for every
x  (a, b), we have R(f1 , P n , Qn ) = R(f2 , P n , Qn ) for every n  Z+ .
Therefore the Archimedes-Riemann Theorem yields
      Z b                                                         Z b
          f1 = lim R(f1 , P , Q ) = lim R(f2 , P , Q ) =
                               n    n                   n    n
                                                                      f2 .
        a        n                     n                       a
                                                                              
  It is a consequence of the Extension Lemma and interval additivity
that two functions that differ at only a finite number of points are the
same when is comes to Riemann integrals.
Theorem 2.4. Let f : [a, b]  R be Riemann integrable over [a, b].
Let g : [a, b]  R such that g(x) = f (x) at all but a finite number of
points in [a, b]. Then g is Riemann integrable over [a, b] and
                              Z b    Z b
                                  g=     f.
                                  a        a
                                                                              23
Proof. Exercise.                                               
Remark. The same cannot be said of two functions that differ at a
countable number of points. Indeed, consider the function
                              (
                                1 if x  Q ,
                      g(x) =
                                0 if x / Q.
Its restriction to any closed bounded interval [a, b] is not Riemann
integrable, yet it differs from f = 0 at a countable number of points.
  We can now show that all functions that are piecewise monotonic
over [a, b] are also Riemann intergrable over [a, b]. We first recall the
definition of piecewise monotonic function.
Definition 2.3. A function f : [a, b]  R is said to be piecewise
monotonic if it is bounded and there exists a partition P = [x0 ,    , xn ]
of [a, b] such that f is monotonic over (xi1 , xi ) for every i = 1,    , n.
Theorem 2.5. Let f : [a, b]  R be piecewise monotonic. Then f is
Riemann integrable over [a, b].
Proof. This follows from Proposition 2.1, the Extension Lemma, and
the Interval Additivity Proposition. The details are left as an exercise.
   We can also show that all functions that are piecewise continuous
over [a, b] are also intergrable over [a, b]. We first recall the definition
of piecewise continuous function.
Definition 2.4. A function f : [a, b]  R is said to be piecewise
continuous if it is bounded and there exists a partition P = [x0 ,    , xn ]
of [a, b] such that f is continuous over (xi1 , xi ) for every i = 1,    , n.
We remark the class of piecewise continuous functions includes some
fairly wild functions. For example, it contains f : [1, 1]  R given by
                        
                        1 + sin(1/x)
                                         if x  (0.1] ,
                f (x) = 4                 if x = 0 ,
                        
                        1 + sin(1/x) if x  [1, 0) .
Proof. Exercise.                                                    
   Of course, one has to show that many sets do not have measure zero.
Exercise. Show that every nonempty open interval (a, b) does not
have measure zero.
Remark. When the above exercise is combined with the last assertion
of Proposition 2.8, we see that a set does not have measure zero if it
contains a nonempty open interval. There are many such sets.
   The following example shows that there are some very interesting
sets that have measure zero.
                                                                                 25
            C1 = [0, 1]  ( 31 , 23 ) = [0, 13 ]  [ 23 , 1] ,
            C2 = C1  ( 19 , 29 )  ( 97 , 98 )
                    = [0, 19 ]  [ 29 , 31 ]  [ 23 , 97 ]  [ 89 , 1] ,
                        1     2        7 8
            C3 = C2  ( 27 , 27 )  ( 27 , 27 )  ( 19 , 20 )  ( 27
                                                    27 27
                                                                  25 26
                                                                     , 27 )
                           1       2 1
                    = [0, 27 ]  [ 27 , 9 ]  [ 29 , 27
                                                      7        8 1
                                                        ]  [ 27 , 3]
                         [ 23 , 27
                                 19       20 7
                                    ]  [ 27 , 9 ]  [ 98 , 25
                                                            27
                                                               ]  [ 26
                                                                     27
                                                                        , 1] ,
               ..
                .
In general one has
                                             [
                    Cn = Cn1                     ( 2k1
                                                      3n
                                                          , 32kn ) for n > 3 .
                                           2k<3n
One can show by induction that each Cn is the union of 2n closed inter-
vals each of which have length 1/3n . Each Cn is therefore sequentially
compact. Moreover, these sets are nested as
                        C1  C2      Cn  Cn+1     .
The Cantor set C is then defined to be the intersection of these sets:
                                 \
                            C=       Cn .
                                                    n=1
Proof. The key step is to show that there exists a p  (c, d) such that
f (p) > 0 and f is continuous at p. Indeed, consider the sets
              Y = {x  (c, d) : f (x) = 0} ,
               Z = {x  (c, d) : f is not continous at x} .
The set Y has measure zero by hypothesis. The set Z has measure
zero by the Lebesgue Theorem. The set Y  Z therefore has measure
zero by the first assertion of Proposition 2.8. But then Y  Z cannot
contain (c, d) because otherwise the last assertion of Proposition 2.8
would imply (c, d) has measure zero, which it does not. Hence, the set
(c, d)  Y  Z is nonempty. The rest of the proof is left as an exercise.
Proposition 2.10. (Strict Order) Let f : [a, b]  R and g : [a, b] 
R be Riemann integrable. Suppose that f  g and that f (x) < g(x)
almost everywhere over a nonempty (c, d)  [a, b]. Then
                           Z b    Z b
                               f<     g.
                               a       a
Proof. Exercise.                                                       
                                                                            27
where
                                             n
                                             X
                                   p
                                 S (n) =             ip .
                                              i=1
28
                                b
                                                       br+1 p       bp+1
                        Z
(31)                                xp dx = lim             S (n) =      .
                            0                      n np+1         p+1
Once this is done then for every [a, b] (0, ) one has
                   b                          b                      a
                                                                                   bp+1  ap+1
           Z                          Z                      Z
                        p                          p
                       x dx =                     x dx                  xp dx =               ,
               a                          0                      0                    p+1
                                                       1                    1
(32)                                  lim                  S p (n) =           .
                                      n         np+1                     p+1
The details of proving (32) are presented in the book for the cases
p = 0, 1, 2 with b = 1. Most calculus books prove this limit for cases no
higher than p = 3. They usually proceed by first establishing formulas
for S p (n) like
                                                                                     n(n + 1)
          S 0 (n) = n ,                                                    S 1 (n) =           ,
                                                                                         2
                            n(n + 1)(2n + 1)                                         n2 (n + 1)2
          S 2 (n) =                          ,                             S 3 (n) =             .
                                   6                                                      4
The first of these formulas is trivial. The others are typically verified by
an induction argument on n. Given such an explicit formula for S p (n),
establishing (32) is easy. However, this approach does not give any
insight into how to obtain these formulas, which grow in complexity as
p increases.
   Here we will take a different approach that allows us to prove (32)
for every p  N. We will first find a relation that expresses S p (n) in
terms of all the S j (n) with j = 0,    , p  1. Then, instead of using
this relation to generate complicated explicit formulas for S p (n), we
will use it to prove (32) via an induction argument on p.
Proof. Clearly S 0 (n) = n, so that limit (32) holds for p = 0. Now
assume that for some q  1 limit (32) holds for every p < q. By a
telescoping sum, the binomial formula, and the definition of S p (n), one
                                                                                     29
Upon solving for S q (n) and dividing by nq+1 , we obtain the relation
                              "
           1     q         1    (n + 1)q+1      1
               S   (n) =                     q+1
         n q+1           q+1       n q+1      n
(33)                               q1
                                                                   #
                                   X      (q + 1)!      1
                                                       q+1
                                                            S p (n) .
                                   p=0
                                       p!(q  p + 1)! n
Because we know
                   (n + 1)q+1                 1
                 lim          = 1 ,     lim      = 0,
              n     nq+1             n nq+1
This can be used to generate explicit formulas for S p (n) for any p  1.
To get an idea of how complicated these explict formulas become, start
with the fact S 0 (n) = n and use the above relation to generate explicit
formulas for S 1 (n), S 2 (n), S 3 (n), and S 4 (n).
30
  Given the above explicit formula for R(xp , P n , Qn ), one only needs
to show that
                                 rn  1        1
(34)                       lim (p+1)       =        .
                          n r
                                n    1      p+1
Then
                                                 rn  1    bp+1  ap+1
   lim R(xp , P n , Qn ) = bp+1  ap+1 lim (p+1)
                                        
                                                         =             ,
  n                                     n r
                                                n     1      p+1
which yields (30) for the case p 6= 1. The case p = 1 is left as an
exercise.                                                                
Exercise. Prove (34).
Exercise. Prove (30) for the case p = 1.
                                                                    31
The function F (x) = |x| is a primitive of f over [1, 1], yet is not
differentiable at x = 0. Similarly, consider the function
                          (
                            1 for x  [1, 0)  (0, 1] ,
                  f (x) =
                            0 for x = 0 ,
                                                                                  33
Corollary 3.1. Let f : [a, b]  R have a primitive over [a, b]. Let
xo  [a, b] and yo  R. Then f has a unique primitive F such that
F (xo ) = yo .
Proof. Exercise.                                                                  
Exercise. Let f : [0, 3]  R be defined by
                            
                            x
                                  for 0  x < 1 ,
                    f (x) = x for 1  x < 2 ,
                            
                            1     for 2  x  3 .
Find F , the primitive of f over [0, 3] specified by F (0) = 1.
  We are now ready to for the big theorem.
34
The change of variable formula (38) immediately follows from the last
two equations.                                                         
Remark. The assumption that G is increasing over [a, b] could have
been replaced by the assumption that G is decreasing over [a, b]. In
that case the interval [G(b), G(a)] replaces the interval [G(a), G(b)] in
the hypotheses regarding f and F , but the change of variable formula
(38) remains unchanged.
Exercise. The assumption that G is increasing over [a, b] in Proposi-
tion 3.1 can be weakened to the assumption that G is nondecreasing
over [a, b]. Prove this slightly strengthend lemma. The proof can be
very similar to the one given above, however you will have to work a
bit harder to show that F (G) is a primitive of f (G)g over [a, b].
   It is natural to ask whether one needs a hypothesis like G is mono-
tonic over [a, b] in order to establish the change of variable formula
(38). Indeed, one does not. However, without it one must take care
to insure the compositions f (G) and F (G) are defined over [a, b], to
insure that F (G) is a primitive of f (G)g over [a, b], and to insure that
f (G)g is Riemann integrable over [a, b]. Here we do this by assuming
that f is continuous over an interval containing Range(G).
Proposition 3.2. (Nonmonotonic Substitution) Let g : [a, b]  R
be Riemann integrable and have a primitive G over [a, b]. Suppose that
Range(G)  [m, m] and let f : [m, m]  R be continuous over [m, m].
Then the change of variable formula (38) holds.
everywhere over [a, b]. Then there exists a point p  (a, b) such that
                          Z b             Z b
(39)                          f g = f (p)     g
                              a            a
In other words, when both f and g are continuous the Integral Mean-
Value Theorem is just the Cauchy Mean-Value Theorem for differen-
tiable functions applied to primitives of f g and g.
Remark. The only way to bound the Taylor remainder using the
Lagrange form (41) is to use uniform bounds on f (n+1) (p) over all p
that lie between c and x. While this approach is sufficient for some
tasks (like showing that the formal Taylor series of ex , cos(x), and
sin(x) converge to those functions for every x  R), it fails for other
tasks. However, if you are able to obtain suitable pointwise bounds on
its intrgrand then the Cauchy form (42) can sometimes yield bounds on
the Taylor remainder that are sufficient for those tasks. This remark
is illustrated by the following example.
Example. Let f (x) = log(1 + x) for every x > 1. Then
                            (k  1)!
      f (k) (x) = (1)k1              for every x > 1 and k  Z+ .
                            (1 + x)k
The formal Taylor aeries of f about 0 is therefore
                               
                               X (1)k1
                                            xk .
                               k=1
                                       k
The Absolute Ratio Test shows that this series converges absolutely for
|x| < 1 and diverges for |x| > 1. For x = 1 the series is the negative of
the harmonic series, and therefore diverges. For x = 1 the Alternating
Series Test shows the series converges. We therefore conclude that the
series converges if and only if x  (1, 1]. These arguments do not
show however that the sum of the series is f (x). This requires showing
that for every x  (1, 1] the Taylor remainder f (x)  T0n f (x) vanishes
as n  .
   First let us approach this problem using the Lagrange form of the
remainder (41): there exists a p between 0 and x such that
                                                             n+1
                                        xn+1     (1)n
                                                       
                 n          (n+1)                        x
       f (x)  T0 f (x) = f       (p)          =                   .
                                      (n + 1)!   n+1 1+p
If x  (0, 1] then p  (0, x) and we obtain the bound
                      f (x)  T0n f (x) < 1 xn+1 .
                                       
                                           n+1
This bound clearly vanishes as n   for every x  (0, 1]. On the
other hand, if x  (1, 0) then p  (|x|, 0) and we obtain the bound
                                                    n+1
                 f (x)  T n f (x) < 1       |x|
                                  
                            0                             .
                                       n + 1 1  |x|
This bound will only vanish as n   for x  [ 21 , 0). This approach
leaves the question open for x  (1,  21 ).
                                                                          45
  Now let us approach this problem using the Cauchy form of the
remainder (42):
                      Z x
                                      (x  t)n
            n
   f (x)  T0 f (x) =     f (n+1) (t)          dt
                       0                 n!
                             Z x                    Z x     n
                           n        (x  t)n             tx     dt
                    = (1)                n+1
                                               dt =                 .
                               0 (1 + t)             0   1+t    1+t
Let us only consider the case x  (1, 0). Consider the substitution
       tx          1+x                      1+x                1+x
  s=         =1            ,      t+1=             ,   dt =            ds .
       1+t           1+t                      1s              (1  s)2
Notice that s decreases from x (= |x|) to 0 as t goes from 0 to x.
Hence, because
              1          1           1
                  <            =           for every s  (0, |x|) ,
           1s       1  |x|     1+x
we obtain the bound
                                Z |x| n
                          
         f (x)  T0n f (x) =          s
                                              ds
                                 0     1s
                                        Z |x|
                                   1                   1 |x|n+1
                              <               sn ds =               .
                                1+x 0                 1+x n+1
This bound clearly vanishes as n   for every x  (1, 0).
  Collecting all of our results, we have shown that
                          
                         X    (1)k1 k
         log(1 + x) =                   x for every x  (1, 1] ,
                         k=1
                                 k
and that the series diverges for all other values of x.
Exercise. When q  N the binomial expansion yields
             n                     q
         q
            X        q!      k
                                  X   q(q  1)    (q  k + 1) k
  (1 + x) =                 x =1+                               x .
            k=0
                k!(q   k)!       k=1
                                                  k!
Now let q  R  N. Let f (x) = (1 + x)q for every x > 1. Then
f (k) (x) = q(q1)    (qk+1)(1+x)qk for every x > 1 and k  Z+ .
The formal Taylor series of f about 0 is therefore
                      
                     X    q(q  1)    (q  k + 1) k
                 1+                                 x .
                     k=1
                                      k!
Show that this series converges absolutely to (1 + x)q when |x| < 1
and diverges when |x| > 1. (This formula is Newtons extension of the
binomial expansion to powers q that are real.)