Numerical Analysis – Lecture 31 2 Orthogonal Polynomials

Numerical Analysis – Lecture 31 2 Orthogonal Polynomials

Mathematical Tripos Part IB: Lent 2010 Numerical Analysis – Lecture 31 2 Orthogonal polynomials 2.1 Orthogonality in general linear spaces n Rn We have already seen the scalar product x, y = i=1 xiyi, acting on x, y . Likewise, given h i n ∈ arbitrary weights w1, w2,...,w > 0, we may defineP x, y = w x y . In general, a scalar (or n h i i=1 i i i inner) product is any function V V R, where V is a vectorP space over the reals, subject to the following three axioms: × → Symmetry: x, y = y, x x, y V; Nonnegativity:h ix, xh 0i ∀x V∈ and x, x =0 iff x = 0; and Linearity: ax +hby, zi ≥= a∀x,∈z + b y,hz xi , y, z V, a, b R. Given a scalarh product,i we mayh definei horthogonality:i ∀ ∈x, y V∈are orthogonal if x, y = 0. V V ∈ b h i Let = C[a, b], w be a fixed positive function and define f, g := a w(x)f(x)g(x) dx for all f, g V. It is easy∈ to verify all three axioms of the scalar product.h i R ∈ 2.2 Orthogonal polynomials – definition, existence, uniqueness Given a scalar product in V = P [x], we say that p P [x] is the nth orthogonal polynomial n n ∈ n if pn,p = 0 for all p Pn−1[x]. [Note: different inner products lead to different orthogonal h i ∈ n polynomials.] A polynomial in Pn[x] is monic if the coefficient of x therein equals one. Theorem For every n 0 there exists a unique monic orthogonal polynomial of degree n. More- ≥ over, any p P [x] can be expanded as a linear combination of p0,p1,...,p , ∈ n n Proof. We let p0(x) 1 and prove the theorem by induction on n. Thus, suppose that ≡ p0,p1,...,pn have been already derived consistently with both assertions of the theorem and let n+1 q(x) := x P +1[x]. Motivated by the Gram–Schmidt algorithm, we choose ∈ n n q,pk pn+1(x) = q(x) h i pk(x), x R. (2.1) − pk,pk ∈ kX=0 h i Clearly, pn+1 Pn+1[x] and it is monic (since all the terms in the sum are of degree n). Let m 0, 1,...,n∈ . It follows from (2.1) and the induction hypothesis that ≤ ∈ { } n q,pk q,pm pn+1,pm = q,pm h i pk,pm = q,pm h i pm,pm = 0. h i h i − pk,pk h i h i − pm,pm h i kX=0 h i h i Hence, pn+1 is orthogonal to p0,...,pn. Consequently, according to the second inductive assertion, it is orthogonal to all p P [x]. ∈ n To prove uniqueness, we suppose the existence of two monic orthogonal polynomials p +1, p˜ +1 n n ∈ P +1[x]. Let p := p +1 p˜ +1 P [x], hence p +1,p = p˜ +1,p = 0, and this implies n n − n ∈ n h n i h n i 0 = p +1,p p˜ +1,p = p +1 p˜ +1,p = p,p , h n i − h n i h n − n i h i 1Corrections and suggestions to these notes should be emailed to [email protected]. All handouts are available on the WWW at the URL http://www.damtp.cam.ac.uk/user/na/PartIB/. 1 and we deduce p 0. ≡ Finally, in order to prove that each p Pn+1[x] is a linear combination of p0,...,pn+1, we note ∈ n+1 that we can always write it in the form p = cpn+1 + q, where c is the coefficient of x in p and where q P [x]. According to the induction hypothesis, q can be expanded as a linear combination ∈ n of p0,p1,...,pn, hence our assertion is true. 2 Well-known examples of orthogonal polynomials include Name Notation Interval Weight function Legendre Pn [ 1, 1] w(x) 1 − ≡ 2 −1/2 Chebyshev Tn [ 1, 1] w(x) = (1 x ) − − −x Laguerre Ln [0, ) w(x) = e ∞ 2 Hermite H ( , ) w(x) = e−x n −∞ ∞ 2.3 The three-term recurrence relation How to construct orthogonal polynomials? (2.1) might help, but it suffers from loss of accuracy due to imprecisions in the calculation of scalar products. A considerably better procedure follows from our next theorem. Theorem Monic orthogonal polynomials are given by the formula p−1(x) 0, p0(x) 1, ≡ ≡ p +1(x) = (x α )p (x) β p −1(x), n = 0, 1,..., (2.2) n − n n − n n where pn,xpn pn,pn αn := h i, βn = h i > 0. p ,p p −1,p −1 h n ni h n n i Proof. Pick n 0 and let ψ(x) := p +1(x) (x α )p (x) + β p −1(x). Since p and p +1 are ≥ n − − n n n n n n monic, it follows that ψ P [x]. Moreover, because of orthogonality of p −1,p ,p +1, ∈ n n n n ψ,p = p +1,p p , (x α )p + β p −1,p = 0, ℓ = 0, 1,...,n 2. h ℓi h n ℓi − h n − n ℓi nh n ℓi − Because of monicity, xp −1 = p + q, where q P −1[x]. Thus, from the definition of α , β , n n ∈ n n n ψ,p −1 = p ,xp −1 + β p −1,p −1 = p ,p + β p −1,p −1 = 0, h n i −h n n i nh n n i −h n ni nh n n i ψ,p = xp ,p + α p ,p = 0. h ni −h n ni nh n ni Every p Pn[x] that obeys p,pℓ = 0, ℓ = 0, 1,...,n, must necessarily be the zero polynomial. ∈ h i s For suppose that it is not so and let x be the highest power of x in p. Then p,ps = 0, which is impossible. We deduce that ψ 0, hence (2.2) is true. h i 6 2 ≡ Example Chebyshev polynomials We choose the scalar product 1 dx f, g := f(x)g(x) 2 , f, g C[ 1, 1] h i Z−1 √1 x ∈ − − and define Tn Pn[x] by the relation Tn(cos θ) = cos(nθ). Hence T0(x) 1, T1(x) = x, T2(x) = 2x2 1 etc. Changing∈ the integration variable, ≡ − 1 π π dx 1 Tn,Tm = Tn(x)Tm(x) 2 = cos nθ cos mθ dθ = 2 [cos(n+m)θ + cos(n m)θ] dθ = 0 h i Z−1 √1 x Z0 Z0 − − whenever n = m. The recurrence relation for Chebyshev polynomials is particularly simple, 6 T +1(x) = 2xT (x) T −1(x), as can be verified at once from the identity cos[(n + 1)θ] + cos[(n n n − n − 1)θ] = 2 cos(θ) cos(nθ). Note that the Tns aren’t monic, hence the inconsistency with (2.2). To obtain monic polynomials take T (x)/2n−1, n 1. n ≥ 2.

View Full Text

Details

  • File Type
    pdf
  • Upload Time
    -
  • Content Languages
    English
  • Upload User
    Anonymous/Not logged-in
  • File Pages
    2 Page
  • File Size
    -

Download

Channel Download Status
Express Download Enable

Copyright

We respect the copyrights and intellectual property rights of all users. All uploaded documents are either original works of the uploader or authorized works of the rightful owners.

  • Not to be reproduced or distributed without explicit permission.
  • Not used for commercial purposes outside of approved use cases.
  • Not used to infringe on the rights of the original creators.
  • If you believe any content infringes your copyright, please contact us immediately.

Support

For help with questions, suggestions, or problems, please contact us