Numerical Methods in Economics

Size: px
Start display at page:

Download "Numerical Methods in Economics"

Transcription

1 Numericl Methods in Economics Alexis Akir Tod November 5, 07 Polynomil interpoltion Polynomils re gret becuse we cn differentite nd integrte them very esily. Since degree n polynomil is determined by n coefficients, once we specify n points on the xy plne, there exists (t most) one polynomil tht psses through these points.. Lgrnge interpoltion The Lgrnge interpoltion gives n explicit formul. Proposition. Let x < < x n nd define the k-th Lgrnge polynomil l k L k (x) = (x x l) l k (x k x l ) for k =,..., n. Then p(x) = n y k L k (x) is the unique polynomil of degree up to n stisfying p(x k ) = y k for k =,..., n. Proof. By the definition of L k (x), we hve L k (x l ) = δ kl (Kronecker s delt ). Therefore for ll l, we hve p(x l ) = n y k L k (x l ) = n y k δ kl = y l. Clerly L k (x) is polynomil of degree n, so p(x) is polynomil of degree up to n. If we interpolte function f(x) t the points x < < x n by degree n polynomil, wht is the error? The following proposition gives n error bound if f is sufficiently smooth. tod@ucsd.edu

2 Proposition. Let f be C n nd p n be the interpolting polynomil of f t x,..., x n. Then for ny x, there exists ξ in the convex hull of {x, x,..., x n } such tht f(x) p n (x) = f (n) (ξ) n (x x k ). n! Proof. Let I = co {x, x,..., x n }. For ny t I, let R(t) = f(t) p n (t) be the error term nd define g(t) = R(t)S(x) R(x)S(t), where S(t) = n (t x k). Clerly g(x) = 0. Furthermore, since R(x k ) = S(x k ) = 0, we hve g(x k ) = 0 for k =,..., n. In generl, if g is differentible nd g() = g(b) = 0, then there exists c (, b) such tht g (c) = 0 (Rolle s theorem ). Therefore there exist n points y,..., y n between x, x,..., x n such tht g (y k ) = 0 for k =,..., n. Continuing this rgument, there exists ξ I such tht g (n) (ξ) = 0. But since S is degree n polynomil with leding coefficient, we hve S (n) = n!, so 0 = g (n) (ξ) = R (n) (ξ)s(x) R(x)n!. Since R(t) = f(t) p n (t) nd deg p n n, we obtin R (n) (ξ) = f (n) (ξ). Therefore f(x) p n (x) = R(x) = n! f (n) (ξ)s(x) = f (n) (ξ) n!. Chebyshev polynomils n (x x k ). If we wnt to interpolte function on n intervl by polynomil, how should we choose the interpoltion nodes x,..., x n? First, without loss of generlity we my ssume tht the intervl is [, ]. Since f (n) (ξ) depends on the prticulr function f but n (x x k) does not, it mkes sense to find x,..., x n so s to minimize n mx (x x x [,] k ). Chebyshev 3 hs solved this problem long time go. The degree n Chebyshev polynomil T n (x) is obtined by expnding cos nθ s degree n polynomil of cos θ nd setting x = cos θ. For instnce, cos 0θ = = T 0 (x) =, cos θ = cos θ = T (x) = x, cos θ = cos θ = T (x) = x, nd so on. In generl, dding cos(n + )θ = cos nθ cos θ sin nθ sin θ, cos(n )θ = cos nθ cos θ + sin nθ sin θ, s_theorem 3

3 nd setting x = cos nθ, we obtin Theorem 3. The solution of T n+ (x) = xt n (x) T n (x). min mx x,...,x n x [,] n (x x k ) is given by x k = cos k n π, in which cse n (x x k) = n T n (x). Proof. Let p(x) = n T n (x). By the bove recursive formul, the leding coefficient of T n (x) is n. Therefore the leding coefficient of p(x) is. Since p(cos θ) = n cos nθ, clerly sup x [,] p(x) = n. Suppose tht there exists degree n polynomil q(x) with leding coefficient such tht sup x [,] q(x) < n. Agin since p(cos θ) = n cos nθ, we hve p(x) = ( ) k n t x = y k = cos kπ/n, where k = 0,,..., n. Since q(x) < n for ll x [, ], by the intermedite vlue theorem there exits z,..., z n between y 0,..., y n such tht p(z k ) q(z k ) = 0. But since p, q re polynomils of degree n with leding coefficient, r(x) := p(x) q(x) is polynomil of degree up to n. Since r(z k ) = 0 for k =,..., n, it must be r(x) 0 or p q, which is contrdiction. Therefore n (x x k) = n T n (x), so x k = cos k n π for k =,..., n. Qudrture Mny economic problems involve mximizing the expected vlue. For exmple, typicl optiml portfolio problem looks like mx E[u(R(θ)w)], θ where w is initil welth, u is Bernoulli utility function, nd R(θ) denotes the portfolio return. Since expecttions re integrls, nd mny integrls cnnot be computed explicitly, we need methods to numericlly evlute the integrls, which re clled qudrture (or numericl integrtion). A typicl qudrture looks like f(x) dx w n f(x n ), where f is generl integrnd nd {x n } N re nodes nd {w n} N re weights of the qudrture rule. See Dvis nd Rbinowitz (984) for stndrd textbook tretment.. Newton-Cotes qudrture The simplest qudrture rule is to divide the intervl [, b] into N evenspced subintervls (so x n = + n N (b ) for n =,..., N) nd choose the weights {w n } N so tht one cn integrte ll polynomils of degree N or 3

4 less exctly. This qudrture rule is known s the N-point Newton-Cotes rule. Since we cn mp the intervl [0, ] to [, b] through the liner trnsformtion x + (b )x, without loss of generlity let us ssume = 0 nd b =. Let us consider severl cses... N = (trpezoidl rule) The -point Newton-Cotes rule is known s the trpezoidl rule. In this cse we hve x n = 0,, nd we choose w, w to integrte liner function exctly. Therefore = = 0 0 dx = w + w, x dx = w, so solving these equtions we obtin w = w =. Therefore f(x) dx b (f() + f(b)). Let us estimte the error of this pproximtion. Let p(x) be the degree interpolting polynomil of f t x =, b. Since p grees with f t, b, clerly Therefore by Proposition, we obtin p(x) dx = b (f() + f(b)). f(x) dx b (f() + f(b)) = = (f(x) p(x)) dx f (ξ(x)) (x )(x b) dx, where ξ(x) (, b). Since (x )(x b) < 0 on (, b), by the men vlue theorem for Riemn-Stieltjes integrls, there exists c (, b) such tht f (ξ(x)) (x )(x b) dx = f (c) (x )(x b) dx = f (c) (b )3. Therefore we cn estimte the error s f(x) dx b (f() + f(b)) f (b )3... N = 3 (Simpson s rule) The 3-point Newton-Cotes rule is known s Simpson s rule. In this cse we hve x n = 0, /,, nd we choose w, w, w 3 to integrte qudrtic function 4

5 exctly. Therefore = = 3 = dx = w + w + w 3, x dx = w + w 3, x dx = 4 w + w 3, so solving these equtions we obtin w = w 3 = 6 nd w = 3. Therefore Interestingly, since f(x) dx b 6 4 = 0 ( f() + 4f ( + b x 3 dx = 8 w + w 3, ) ) + f(b). Simpson s rule ctully integrtes polynomils of degree 3 exctly (even though it is not designed to do so). To estimte the error of Simpson s rule, tke ny point d (, b) nd let p(x) be degree 3 interpolting polynomil of f t x =, +b, b, d. Since Simpson s rule integrtes degree 3 polynomils exctly, by Proposition we hve f(x) dx b 6 = (f(x) p(x)) dx = ( f() + 4f ( + b ) ) + f(b) f (4) ( (ξ(x)) (x ) x + b ) (x b)(x d) dx. 4! Since d (, b) is rbitrry, we cn tke d = +b. Since ( (x ) x + b ) (x b) < 0 on (, b) lmost everywhere, s before we cn pply the men vlue theorem. Using the chnge of vrible x = +b t, we cn compute + b ( (x ) x + b ) (x b) dx ( ) 5 = (t + )t (t ) dt = 0 (b )5. Since 4! = 4 nd 4 0 = 880, the integrtion error is f(x) dx b ( ( ) + b f() + 4f + f(b)) 6 f (4) 880 (b )5. 5

6 . Compound rule Newton-Cotes rule with N 4 re lmost never used becuse beyond some order some of the weights {w n } N become negtive, which introduces rounding errors. One wy to void this problem is to divide the intervl [, b] into N evenspced subintervls nd pply the trpezoidl rule or the Simpson s rule to ech subintervl. This method is known s the compound (or composite) rule. If you use the trpezoidl rule, then there re N+ points. Letting x n = n/n for n = 0,,..., N, the formul for [0, ] is 0 f(x) dx N (f(x n ) + f(x n )) = N (f(x 0) + f(x ) + + f(x N ) + f(x N )). (Just remember tht the reltive weights re t endpoints nd in between.) Since b = /N nd there re N subintervls, the error of the (N + )-point trpezoidl rule is f N. If you use Simpson s rule, then there re 3 points on ech subintervl, of which there re N, nd N endpoints re counted twice. Therefore the totl number of points is 3N (N ) = N +. Letting x n = n/(n) for n = 0,,..., N, the formul for [0, ] is 0 f(x) dx 6N (f(x n ) + 4f(x n ) + f(x n )) = 6N (f(x 0) + 4f(x ) + f(x ) + + 4f(x N ) + f(x N )). (Just remember tht the reltive weights re t endpoints, nd they lternte like 4,, 4,,..., 4,, 4 in between.) Since b = /N nd there re N subintervls, the error of the (N + )-point Simpson s rule is f (4) 880 N 4. Since the qudrture weights re given explicitly for trpezoidl nd Simpson s rule, it is strightforwrd to write progrms tht compute numericl integrls. The tbles below show the log 0 reltive errors of integrls over the intervl [0, ] (log 0 Î/I, where I is the true integrl nd Î is the numericl one) for severl functions when we use the N-point compound trpezoidl nd Simpson s rule. As the bove error nlysis suggests, errors tend to be smller when the integrnd is smoother (hs higher order derivtives). Furthermore, Simpson s rule is more ccurte thn the trpezoidl rule. Tble. log 0 reltive errors of compound trpezoidl rule. # points x / x 3/ x 5/ x 7/ x 9/ e x

7 Tble. log 0 reltive errors of compound Simpson s rule. # points x / x 3/ x 5/ x 7/ x 9/ e x Gussin qudrture In the Newton-Cotes qudrture, we ssume tht the nodes re even-spced, but of course this is not necessry. Cn we do better by choosing the qudrture nodes optimlly? In generl, consider the integrl w(x)f(x) dx, where < b re endpoints of integrtion, w(x) > 0 is some (fixed) weighting function, nd f is generl integrnd. A typicl exmple is =, b =, nd w(x) = /σ πσ, in which cse we wnt to compute the e (x µ) expecttion E[f(X)] when X N(µ, σ ). In the discussion below, let us omit, b (so mens ) nd ssume tht w(x)x n dx exists for ll n 0. For functions f, g, let us define the inner product (f, g) by (f, g) = w(x)f(x)g(x) dx. Let p n(x) be the orthogonl polynomil of degree n corresponding to the weighting function w(x). This mens tht (p m, p n) = δ mn, where δ mn is Kronecker s delt. Orthogonl polynomils (with positive leding coefficients) uniquely exist nd cn be constructed using the Grm-Schmidt orthonormliztion. 4 In fct, we cn recursively compute the orthogonl polynomils using the three-term recurrence reltion (TTRR) s follows. Proposition 4 (TTRR). Let p (x) = 0, p 0 (x) =, nd for n 0 define p n(x) = p n (x)/(p n, p n ) /, p n+ (x) = xp n(x) (xp n, p n)p n(x) (p n, p n ) / p n (x). Then p n(x) is the n-degree orthogonl polynomil. Proof. Clerly (p n, p n) = for ll n. Therefore it suffices to show tht (p m, p n) = 0 whenever m < n. Let us prove this by induction on n 0. If n = 0, there is nothing to prove. If n =, since p (x) = xp 0(x) (xp 0, p 0)p 0(x), tking the inner product with p 0(x), we obtin (p, p 0) = (xp 0, p 0) (xp 0, p 0) =

8 Therefore by rescling p to p, we obtin (p 0, p ) = 0. Suppose the clim holds up to n. Then for n +, since p n+ (x) = xp n(x) (xp n, p n)p n(x) (p n, p n ) / p n (x), tking the inner product with p n, we obtin (p n+, p n) = (xp n, p n) (xp n, p n) = 0. Similrly, tking the inner product with p n, we obtin (p n+, p n ) = (xp n, p n ) (p n, p n ) / = (p n, xp n ) (p n, p n ) /. Let k n > 0 be the leding coefficient of p n. By the recursive definition nd the normliztion, we hve k n = k n /(p n, p n ) /. Since xp n is n n-degree polynomil with leding coefficient k n, it cn be expnded s Therefore xp n (x) = k n p k n(x) + low order polynomils. n (p n+, p n ) = k n k n (p n, p n ) / = 0. The following lemm shows tht n n-degree orthogonl polynomil hs exctly n rel roots (so they re ll simple). Lemm 5. p n(x) hs exctly n rel roots on (, b). Proof. By the fundmentl theorem of lgebr, p n(x) hs exctly n roots in C. Suppose on the contrry tht p n(x) hs less thn n rel roots on (, b). Let x,..., x k (k < n) those roots t which p n (x) chnges its sign. Let p(x) = (x x ) (x x k ). Since p n(x)p(x) > 0 (or < 0) lmost everywhere on (, b), we hve (p n, p) = w(x)p n(x)p(x) dx 0. On the other hnd, since deg p = k < n nd orthogonl polynomils re linerly independent, we cn express p s weighted sum of p m s, where m k. By the definition of the orthogonl polynomils, it follows tht (p n, p) = 0, which is contrdiction. The following theorem shows tht using the n roots of the degree n orthogonl polynomil s qudrture nodes nd choosing specific weights, we cn integrte ll polynomils of degree up to n exctly. This is known s Gussin qudrture. Theorem 6 (Gussin qudrture). Let < x < < x n < b be the n roots of p n nd define w k = w(x)l k (x) dx 8

9 for k =,..., n, where L k (x) is s in Proposition. Then n w(x)p(x) dx = w k p(x k ) for ll polynomils p(x) of degree up to n. Proof. Since deg p n nd deg p n = n, we cn write p(x) = p n(x)q(x) + r(x), where deg q, deg r n. Since q cn be expressed s liner combintion of orthogonl polynomils of degree up to n, we hve (p n, q) = 0. Hence w(x)p(x) dx = (p n, q) + w(x)r(x) dx = w(x)r(x) dx. On the other hnd, since {x k } n re roots of p n, we hve for ll k, so in prticulr p(x k ) = p n(x k )q(x k ) + r(x k ) = r(x k ) n w k p(x k ) = n w k r(x k ). Therefore it suffices to show the clim for polynomils r of degree up to n. Since by Proposition ny such polynomil cn be represented s liner combintion of L k s, it suffices to show the clim for ll L k s. But since by definition n w(x)l k (x) dx = w k = w l L k (x l ), the clim is true. In prctice, how cn we compute the nodes {x n } N nd weights {w n} N of the N-point Gussin qudrture? The solution is given by the following Golub-Welsch lgorithm. Theorem 7 (Golub-Welsch). Let k n > 0 be the leding coefficient of p n, α n = k n /k n > 0, nd β n = (xp n, p n). Define the N N symmetric mtrix J N by β 0 α 0 0. α β α... J N =. 0 α β αn 0 0 α N β N Then the Gussin qudrture nodes {x n } N re eigenvlues of J N, nd the weights {w n } N re given by l= N = p w k(x n ) > 0. n k=0 9

10 Proof. By the proof of Proposition 4, we hve (p n, p n ) / = k n /k n = α n. Therefore TTRR becomes p n+ (x) = xp n(x) β n p n(x) α n p n (x). Since p n+(x) = p n+ (x)/(p n+, p n+ ) / = p n+ (x)/α n+, TTRR becomes α n p n (x) + β n p n(x) + α n+ p n+(x) = xp n(x). In prticulr, setting x = x k (where x k is root of p N ), we obtin α n p n (x k ) + β n p n(x k ) + α n+ p n+(x k ) = xp n(x k ) for ll n nd k =,..., N. Since p = 0 by definition nd p N (x k) = 0, letting P (x) = (p 0(x),..., p N (x)) nd collecting the bove eqution into vector we obtin J N P (x k ) = x k P (x k ) for k =,..., N. Define the N N mtrix P by P = (P (x ),..., P (x N )). Since δ mn = (p m, p n) = w(x)p m(x)p n(x) dx = w k p m(x k )p n(x k ) for m, n N becuse the Gussin qudrture integrtes ll polynomils of degree up to n exctly, letting W = dig(w,..., w N ) we hve P W P = I. Therefore P, W re invertible. Solving for W nd tking the inverse, we obtin W = P P N = p w k(x n ) > 0 n for ll n. Since J N P (x n ) = x n P (x n ) for n =,..., N, collecting into mtrix we obtin J N P = XP P J N P = X, where X = dig(x,..., x N ). Therefore {x n } N re eigenvlues of J N. Below re some exmples. By googling you cn find subroutines in Mtlb or whtever lnguge tht compute the nodes nd weights of these qudrtures. Exmple. The cse (, b) = (, ), w(x) = is known s the Guss- Legendre qudrture. Exmple. The cse (, b) = (, ), w(x) = / x is known s the Guss-Chebyshev qudrture. It is useful for computing Fourier coefficients (through the chnge of vrible x = cos θ). Exmple 3. The cse (, b) = (, ), w(x) = e x is known s the Guss- Hermite qudrture, which is useful for computing the expecttion with respect to the norml distribution. Exmple 4. The cse (, b) = (0, ), w(x) = e x is known s the Guss- Lguerre qudrture, which is useful for computing the expecttion with respect to the exponentil distribution. The tble below shows the log 0 reltive errors when using the N-point Guss-Legendre qudrture. You cn see tht Gussin qudrture is overwhelmingly more ccurte thn Newton-Cotes. k=0 0

11 Tble 3. log 0 reltive errors of compound trpezoidl rule. # points x / x 3/ x 5/ x 7/ x 9/ e x Discretiztion If the gol is to solve single optimiztion problem tht involves expecttions (e.g., sttic optiml portfolio problem), highly ccurte Gussin qudrture is nturl choice. However, mny economic problems re dynmic, in which cse one needs to compute conditionl expecttions. Furthermore, to reduce the computtionl complexity of the problem, it is desirble tht the qudrture nodes re pressigned insted of being dependent on the prticulr stte of the model. Discretiztion is useful tool for solving such problems. 3. Erlier methods For concreteness, consider the Gussin AR() process x t = ρx t + ε t, ɛ t N(0, σ ). Then the conditionl distribution of x t given x t is N(ρx t, σ ). How cn we discretize (find finite-stte Mrkov chin pproximtion) of this stochstic process? A clssic method is Tuchen (986) but you should never use it becuse it is not ccurte (so I won t explin further). Similrly, the quntile method in Add nd Cooper (003) is poor. For Gussin AR() process, the Rouwenhorst (995) is good becuse the conditionl moments re exct up to order nd the method is constructive (does not involve optimiztion). It is especilly useful when ρ The Tuchen nd Hussey (99) method, which I explin now, uses the Gussin qudrture. First consider discretizing N(0, σ ). Letting {x n } N nd {w n } N be the nodes nd weights of the N-point Guss-Hermite qudrture, since for ny integrnd g we hve E[g(X)] = = g(x) πσ e x σ dx g( σy) π e y dy w n π g( σx n ), we cn use the nodes x n = σx n nd weights w n = w n / π to discretize N(0, σ ). The sme ide cn be used to discretize the Gussin AR() process. Let us fix the nodes {x n} N s constructed bove. Since for ny integrnd g, letting

12 µ = ρx m we hve E [g(x t ) x t = x m] = = g(x) πσ (x µ) e σ dx g(x)e µ xµ σ x e σ dx πσ w ne µ x n µ σ g(x n), so we cn construct the trnsition probbility mtrix P = (p mn ) by p mn w ne µ x n µ σ, where µ = ρx m nd the constnt of proportionlity is determined by N p mn =. The Tuchen-Hussey method is pretty good if ρ 0.5, lthough drwbck is tht it ssumes Gussin shocks. Furthermore, the performnce deteriortes when ρ becomes lrger. 3. Frmer-Tnk-Tod mximum entropy method Severl ppers by me nd my couthors (Tnk nd Tod, 03, 05; Frmer nd Tod, 07) provide more ccurte nd generlly pplicble discretiztion method (so it should be the first choice!). Below I briefly explin the method, but see Frmer nd Tod (07) for more detils. 3.. Discretizing probbility distributions Suppose tht we re given continuous probbility density function f : R K R, which we wnt to discretize. Let X be rndom vector with density f, nd g : R K R be ny bounded continuous function. The first step is to pick qudrture formul E[g(X)] = g(x)f(x) dx R K w n g(x n )f(x n ), () where N is the number of integrtion points, {x n } N, nd w n > 0 is the weight on the integrtion point x n. For now, we do not tke stnce on the choice of the initil qudrture formul, but tke it s given. Given the qudrture formul (), corse but vlid discrete pproximtion of the density f would be to ssign probbility q n to the point x n proportionl to w n f(x n ), so q n = w n f(x n ) N w nf(x n ). () However, this is not necessrily good pproximtion becuse the moments of the discrete distribution {q n } do not generlly mtch those of f. Tnk nd Tod (03) propose exctly mtching finite set of moments by updting the probbilities {q n } in prticulr wy. Let T : R K R L

13 be function tht defines the moments tht we wish to mtch nd let T = T (x)f(x) dx be the vector of exct moments. For exmple, if we wnt to R K mtch the first nd second moments in the one dimensionl cse (K = ), then T (x) = (x, x ). Tnk nd Tod (03) updte the probbilities {q n } by solving the optimiztion problem minimize {p n} subject to mx λ R L p n log p n q n p n T (x n ) = T, p n =, p n 0. The objective function in the priml problem (P) is the Kullbck nd Leibler (95) informtion of {p n } reltive to {q n }, which is lso known s the reltive entropy. This method mtches the given moments exctly while keeping the probbilities {p n } s close to the initil pproximtion {q n } s possible in the sense of the Kullbck-Leibler informtion. Note tht since (P) is convex minimiztion problem, the solution (if one exists) is unique. The optimiztion problem (P) is constrined minimiztion problem with lrge number (N) of unknowns ({p n }) with L + equlity constrints nd N inequlity constrints, which is in generl computtionlly intensive to solve. However, it is well-known tht entropy-like minimiztion problems re computtionlly trctble by using dulity theory (Borwein nd Lewis, 99). Tnk nd Tod (03) convert the priml problem (P) to the dul problem [ ( N )] λ T log q n e λ T (x n), (D) which is low dimensionl (L unknowns) unconstrined concve mximiztion problem nd hence computtionlly trctble. The following theorem shows how the solutions to the two problems (P) nd (D) re relted. Below, the symbols int nd co denote the interior nd the convex hull of sets. Theorem 8.. The priml problem (P) hs solution if nd only if T co T (D N ). If solution exists, it is unique.. The dul problem (D) hs solution if nd only if T int co T (D N ). If solution exists, it is unique. 3. If the dul problem (D) hs (unique) solution λ N, then the (unique) solution to the priml problem (P) is given by p n = (P) q n e λ N T (xn) N q ne = q n e λ N (T (xn) T ) λ N T (xn) N q ne λ N (T (xn) T. (3) ) Theorem 8 provides prcticl wy to implement the Tnk-Tod method. After choosing the initil discretiztion Q = {q n } nd the moment defining function T, one cn numericlly solve the unconstrined optimiztion problem (D). To this end, we cn insted solve min λ R L q n e λ (T (x n) T ) (D ) 3

14 becuse the objective function in (D ) is monotonic trnsformtion ( times the exponentil) of tht in (D). Since (D ) is n unconstrined convex minimiztion problem with (reltively) smll number (L) of unknowns (λ), solving it is computtionlly simple. Letting J N (λ) be the objective function in (D ), its grdient nd Hessin cn be nlyticlly computed s J N (λ) = J N (λ) = q n e λ (T (x n) T ) (T (x n ) T ), q n e λ (T (x n) T ) (T (x n ) T )(T (x n ) T ), (4) (4b) respectively. In prctice, we cn quickly solve (D ) numericlly using optimiztion routines by supplying the nlyticl grdient nd Hessin. 5 If solution to (D ) exists, it is unique, nd we cn compute the updted discretiztion P = {p n } by (3). If solution does not exist, it mens tht the regulrity condition T int co T (D N ) does not hold nd we cnnot mtch moments. Then one needs to select smller set of moments. Numericlly checking whether moments re mtched is strightforwrd: by (3), (D ), nd (4), the error is p n T (x n ) T = N q ne λ N (T (xn) T ) (T (x n ) T ) N q ne λ N (T (xn) T ) 3.. Discretizing generl Mrkov processes = J N (λ N ) J N (λ N ). (5) Next we show how to extend the Tnk-Tod method to the cse of timehomogeneous Mrkov processes. Consider the time-homogeneous first-order Mrkov process P (x t x x t = x) = F (x, x), where x t is the vector of stte vribles nd F (, x) is cumultive distribution function (CDF) tht determines the distribution of x t = x given x t = x. The dynmics of ny Mrkov process re completely chrcterized by its Mrkov trnsition kernel. In the cse of discrete stte spce, this trnsition kernel is simply mtrix of trnsition probbilities, where ech row corresponds to conditionl distribution. We cn discretize the continuous process x by pplying the Tnk-Tod method to ech conditionl distribution seprtely. More concretely, suppose tht we hve set of grid points D N = {x n } N nd n initil corse pproximtion Q = (q nn ), which is n N N probbility trnsition mtrix. Suppose we wnt to mtch some conditionl moments of x, represented by the moment defining function T (x). The exct conditionl moments when the current stte is x t = x n re T n = E [T (x t ) x n ] = T (x) df (x, x n ), 5 Since the dul problem (D) is concve mximiztion problem, one my lso solve it directly. However, ccording to our experience, solving (D ) is numericlly more stble. This is becuse the objective function in (D) is close to liner when λ is lrge, so the Hessin is close to singulr nd not well-behved. On the other hnd, since the objective function in (D ) is the sum of exponentil functions, it is well-behved. 4

15 where the integrl is over x, fixing x n. (If these moments do not hve explicit expressions, we cn use highly ccurte qudrture formuls to compute them.) By Theorem 8, we cn mtch these moments exctly by solving the optimiztion problem minimize {p nn } N n = subject to n = p nn log p nn q nn p nn T (x n ) = T n, n = p nn =, p nn 0 (P n ) n = for ech n =,,..., N, or equivlently the dul problem min λ R L n = q nn e λ (T (x n ) T n). (D n) (D n) hs unique solution if nd only if the regulrity condition T n int co T (D N ) (6) holds. We summrize our procedure in Algorithm below. Algorithm (Discretiztion of Mrkov processes).. Select discrete set of points D N = {x n } N nd n initil pproximtion Q = (q nn ).. Select moment defining function T (x) nd corresponding exct conditionl moments { } N Tn. If necessry, pproximte the exct conditionl moments with highly ccurte numericl integrl. 3. For ech n =,..., N, solve minimiztion problem (D n) for λ n. Check whether moments re mtched using formul (5), nd if not, select smller set of moments. Compute the conditionl probbilities corresponding to row n of P = (p nn ) using (3). The resulting discretiztion of the process is given by the trnsition probbility mtrix P = (p nn ). Since the dul problem (D n) is n unconstrined convex minimiztion problem with typiclly smll number of vribles, stndrd Newton type lgorithms cn be pplied. Furthermore, since the probbilities (3) re strictly positive by construction, the trnsition probbility mtrix P = (p nn ) is strictly positive mtrix, so the resulting Mrkov chin is sttionry nd ergodic. 4 Projection In economics we often need to solve functionl equtions. For instnce, in n income fluctution problem, we need to chrcterize the optiml consumption rule c(w, y) given welth w nd income y. The projection method ( stndrd reference is Judd, 99) pproximtes the policy function (wht you wnt to 5

16 solve for, like c(w, y)) on some compct set by polynomil. See Pohl et l. (07) for nice ppliction of the projection method. By Theorem 3 if you wnt to pproximte smooth function f on [, ] by degree N polynomil, it is optiml to interpolte f t the roots of the degree N Chebyshev polynomil. The ide of the projection method is to pproximte the policy function f by liner combintion of Chebyshev polynomils, f(x) f(x) = N n=0 n T n (x), nd determine the coefficients { n } N n=0 to mke the functionl eqution (tht you wnt to solve) true t the Chebyshev nodes. It is esier to see how things work by looking t n exmple. Suppose you wnt to solve the differentil eqution y (t) = y(t), with initil condition y(0) =. Of course the solution is y(t) = e t, but let s pretend tht we don t know the solution nd solve it numericlly. Suppose we wnt to compute numericl solution for t [0, T ]. We cn do s follows.. Mp [0, T ] to [, ] by the ffine trnsformtion t t T T.. Approximte y(t) by ŷ(t) = N n=0 nt n ( t T T ) 3. Determine { n } N n=0 by setting ŷ (t) = ŷ(t) t t corresponding to Chebyshev nodes for degree N (find t n by solving tn T T = cos ( n N π) for n =,..., N). 4. In this cse, must lso impose initil condition ŷ(0) =, so for exmple cn minimize sum of squred residuls t Chebyshev nodes: minimize { n} N n=0 N (ŷ (t n ) ŷ(t n )) n=0 subject to ŷ(0) =. The figure below shows the log 0 reltive errors when T = 4 nd N = 3, 4,.... You cn see tht the reltive errors become smller s we increse the degree of polynomil pproximtion. References Jérôme Add nd Russel W. Cooper. Dynmic Economics: Quntittive Methods nd Applictions. MIT Press, Cmbridge, MA, 003. Jonthn M. Borwein nd Adrin S. Lewis. Dulity reltionships for entropylike minimiztion problems. SIAM Journl on Control nd Optimiztion, 9 ():35 338, Mrch 99. doi:0.37/ Philip J. Dvis nd Philip Rbinowitz. Methods of Numericl Integrtion. Acdemic Press, Orlndo, FL, second edition,

17 0 - log 0 reltive errors rd order 4th order -8 5th order 6th order 7th order -0 8th order t Lelnd E. Frmer nd Alexis Akir Tod. Discretizing nonliner, non-gussin Mrkov processes with exct conditionl moments. Quntittive Economics, 8():65 683, July 07. doi:0.398/qe737. Kenneth L. Judd. Projection methods for solving ggregte growth models. Journl of Economic Theory, 58():40 45, December 99. doi:0.06/00-053(9)9006-l. Solomon Kullbck nd Richrd A. Leibler. On informtion nd sufficiency. Annls of Mthemticl Sttistics, ():79 86, Mrch 95. doi:0.4/oms/ Wlter Pohl, Krl Schmedders, nd Ole Wilms. Higher-order effects in ssetpricing models with long-run risk. Journl of Finnce, 07. URL https: //ssrn.com/bstrct= Forthcoming. K. Geert Rouwenhorst. Asset pricing implictions of equilibrium business cycle models. In Thoms F. Cooley, editor, Frontiers of Business Cycle Reserch, chpter 0, pges Princeton University Press, 995. Ken ichiro Tnk nd Alexis Akir Tod. Discrete pproximtions of continuous distributions by mximum entropy. Economics Letters, 8(3): , Mrch 03. doi:0.06/j.econlet Ken ichiro Tnk nd Alexis Akir Tod. Discretizing distributions with exct moments: Error estimte nd convergence nlysis. SIAM Journl on Numericl Anlysis, 53(5):58 77, 05. doi:0.37/ George Tuchen. Finite stte Mrkov-chin pproximtions to univrite nd vector utoregressions. Economics Letters, 0():77 8, 986. doi:0.06/ (86) George Tuchen nd Robert Hussey. Qudrture-bsed methods for obtining pproximte solutions to nonliner sset pricing models. Econometric, 59 ():37 396, Mrch 99. doi:0.307/

Orthogonal Polynomials

Orthogonal Polynomials Mth 4401 Gussin Qudrture Pge 1 Orthogonl Polynomils Orthogonl polynomils rise from series solutions to differentil equtions, lthough they cn be rrived t in vriety of different mnners. Orthogonl polynomils

More information

Numerical integration

Numerical integration 2 Numericl integrtion This is pge i Printer: Opque this 2. Introduction Numericl integrtion is problem tht is prt of mny problems in the economics nd econometrics literture. The orgniztion of this chpter

More information

1 The Lagrange interpolation formula

1 The Lagrange interpolation formula Notes on Qudrture 1 The Lgrnge interpoltion formul We briefly recll the Lgrnge interpoltion formul. The strting point is collection of N + 1 rel points (x 0, y 0 ), (x 1, y 1 ),..., (x N, y N ), with x

More information

Lecture 6: Singular Integrals, Open Quadrature rules, and Gauss Quadrature

Lecture 6: Singular Integrals, Open Quadrature rules, and Gauss Quadrature Lecture notes on Vritionl nd Approximte Methods in Applied Mthemtics - A Peirce UBC Lecture 6: Singulr Integrls, Open Qudrture rules, nd Guss Qudrture (Compiled 6 August 7) In this lecture we discuss the

More information

Lecture 17. Integration: Gauss Quadrature. David Semeraro. University of Illinois at Urbana-Champaign. March 20, 2014

Lecture 17. Integration: Gauss Quadrature. David Semeraro. University of Illinois at Urbana-Champaign. March 20, 2014 Lecture 17 Integrtion: Guss Qudrture Dvid Semerro University of Illinois t Urbn-Chmpign Mrch 0, 014 Dvid Semerro (NCSA) CS 57 Mrch 0, 014 1 / 9 Tody: Objectives identify the most widely used qudrture method

More information

Orthogonal Polynomials and Least-Squares Approximations to Functions

Orthogonal Polynomials and Least-Squares Approximations to Functions Chpter Orthogonl Polynomils nd Lest-Squres Approximtions to Functions **4/5/3 ET. Discrete Lest-Squres Approximtions Given set of dt points (x,y ), (x,y ),..., (x m,y m ), norml nd useful prctice in mny

More information

CMDA 4604: Intermediate Topics in Mathematical Modeling Lecture 19: Interpolation and Quadrature

CMDA 4604: Intermediate Topics in Mathematical Modeling Lecture 19: Interpolation and Quadrature CMDA 4604: Intermedite Topics in Mthemticl Modeling Lecture 19: Interpoltion nd Qudrture In this lecture we mke brief diversion into the res of interpoltion nd qudrture. Given function f C[, b], we sy

More information

3.4 Numerical integration

3.4 Numerical integration 3.4. Numericl integrtion 63 3.4 Numericl integrtion In mny economic pplictions it is necessry to compute the definite integrl of relvlued function f with respect to "weight" function w over n intervl [,

More information

Numerical Analysis: Trapezoidal and Simpson s Rule

Numerical Analysis: Trapezoidal and Simpson s Rule nd Simpson s Mthemticl question we re interested in numericlly nswering How to we evlute I = f (x) dx? Clculus tells us tht if F(x) is the ntiderivtive of function f (x) on the intervl [, b], then I =

More information

Numerical Integration. 1 Introduction. 2 Midpoint Rule, Trapezoid Rule, Simpson Rule. AMSC/CMSC 460/466 T. von Petersdorff 1

Numerical Integration. 1 Introduction. 2 Midpoint Rule, Trapezoid Rule, Simpson Rule. AMSC/CMSC 460/466 T. von Petersdorff 1 AMSC/CMSC 46/466 T. von Petersdorff 1 umericl Integrtion 1 Introduction We wnt to pproximte the integrl I := f xdx where we re given, b nd the function f s subroutine. We evlute f t points x 1,...,x n

More information

NUMERICAL INTEGRATION. The inverse process to differentiation in calculus is integration. Mathematically, integration is represented by.

NUMERICAL INTEGRATION. The inverse process to differentiation in calculus is integration. Mathematically, integration is represented by. NUMERICAL INTEGRATION 1 Introduction The inverse process to differentition in clculus is integrtion. Mthemticlly, integrtion is represented by f(x) dx which stnds for the integrl of the function f(x) with

More information

Discrete Least-squares Approximations

Discrete Least-squares Approximations Discrete Lest-squres Approximtions Given set of dt points (x, y ), (x, y ),, (x m, y m ), norml nd useful prctice in mny pplictions in sttistics, engineering nd other pplied sciences is to construct curve

More information

Numerical Integration

Numerical Integration Chpter 5 Numericl Integrtion Numericl integrtion is the study of how the numericl vlue of n integrl cn be found. Methods of function pproximtion discussed in Chpter??, i.e., function pproximtion vi the

More information

Best Approximation. Chapter The General Case

Best Approximation. Chapter The General Case Chpter 4 Best Approximtion 4.1 The Generl Cse In the previous chpter, we hve seen how n interpolting polynomil cn be used s n pproximtion to given function. We now wnt to find the best pproximtion to given

More information

Theoretical foundations of Gaussian quadrature

Theoretical foundations of Gaussian quadrature Theoreticl foundtions of Gussin qudrture 1 Inner product vector spce Definition 1. A vector spce (or liner spce) is set V = {u, v, w,...} in which the following two opertions re defined: (A) Addition of

More information

Review of Calculus, cont d

Review of Calculus, cont d Jim Lmbers MAT 460 Fll Semester 2009-10 Lecture 3 Notes These notes correspond to Section 1.1 in the text. Review of Clculus, cont d Riemnn Sums nd the Definite Integrl There re mny cses in which some

More information

The Regulated and Riemann Integrals

The Regulated and Riemann Integrals Chpter 1 The Regulted nd Riemnn Integrls 1.1 Introduction We will consider severl different pproches to defining the definite integrl f(x) dx of function f(x). These definitions will ll ssign the sme vlue

More information

Numerical quadrature based on interpolating functions: A MATLAB implementation

Numerical quadrature based on interpolating functions: A MATLAB implementation SEMINAR REPORT Numericl qudrture bsed on interpolting functions: A MATLAB implementtion by Venkt Ayylsomyjul A seminr report submitted in prtil fulfillment for the degree of Mster of Science (M.Sc) in

More information

Advanced Computational Fluid Dynamics AA215A Lecture 3 Polynomial Interpolation: Numerical Differentiation and Integration.

Advanced Computational Fluid Dynamics AA215A Lecture 3 Polynomial Interpolation: Numerical Differentiation and Integration. Advnced Computtionl Fluid Dynmics AA215A Lecture 3 Polynomil Interpoltion: Numericl Differentition nd Integrtion Antony Jmeson Winter Qurter, 2016, Stnford, CA Lst revised on Jnury 7, 2016 Contents 3 Polynomil

More information

Lecture 14: Quadrature

Lecture 14: Quadrature Lecture 14: Qudrture This lecture is concerned with the evlution of integrls fx)dx 1) over finite intervl [, b] The integrnd fx) is ssumed to be rel-vlues nd smooth The pproximtion of n integrl by numericl

More information

Construction of Gauss Quadrature Rules

Construction of Gauss Quadrature Rules Jim Lmbers MAT 772 Fll Semester 2010-11 Lecture 15 Notes These notes correspond to Sections 10.2 nd 10.3 in the text. Construction of Guss Qudrture Rules Previously, we lerned tht Newton-Cotes qudrture

More information

1. Gauss-Jacobi quadrature and Legendre polynomials. p(t)w(t)dt, p {p(x 0 ),...p(x n )} p(t)w(t)dt = w k p(x k ),

1. Gauss-Jacobi quadrature and Legendre polynomials. p(t)w(t)dt, p {p(x 0 ),...p(x n )} p(t)w(t)dt = w k p(x k ), 1. Guss-Jcobi qudrture nd Legendre polynomils Simpson s rule for evluting n integrl f(t)dt gives the correct nswer with error of bout O(n 4 ) (with constnt tht depends on f, in prticulr, it depends on

More information

Continuous Random Variables

Continuous Random Variables STAT/MATH 395 A - PROBABILITY II UW Winter Qurter 217 Néhémy Lim Continuous Rndom Vribles Nottion. The indictor function of set S is rel-vlued function defined by : { 1 if x S 1 S (x) if x S Suppose tht

More information

Math& 152 Section Integration by Parts

Math& 152 Section Integration by Parts Mth& 5 Section 7. - Integrtion by Prts Integrtion by prts is rule tht trnsforms the integrl of the product of two functions into other (idelly simpler) integrls. Recll from Clculus I tht given two differentible

More information

NUMERICAL INTEGRATION

NUMERICAL INTEGRATION NUMERICAL INTEGRATION How do we evlute I = f (x) dx By the fundmentl theorem of clculus, if F (x) is n ntiderivtive of f (x), then I = f (x) dx = F (x) b = F (b) F () However, in prctice most integrls

More information

Physics 116C Solution of inhomogeneous ordinary differential equations using Green s functions

Physics 116C Solution of inhomogeneous ordinary differential equations using Green s functions Physics 6C Solution of inhomogeneous ordinry differentil equtions using Green s functions Peter Young November 5, 29 Homogeneous Equtions We hve studied, especilly in long HW problem, second order liner

More information

63. Representation of functions as power series Consider a power series. ( 1) n x 2n for all 1 < x < 1

63. Representation of functions as power series Consider a power series. ( 1) n x 2n for all 1 < x < 1 3 9. SEQUENCES AND SERIES 63. Representtion of functions s power series Consider power series x 2 + x 4 x 6 + x 8 + = ( ) n x 2n It is geometric series with q = x 2 nd therefore it converges for ll q =

More information

Lecture 19: Continuous Least Squares Approximation

Lecture 19: Continuous Least Squares Approximation Lecture 19: Continuous Lest Squres Approximtion 33 Continuous lest squres pproximtion We begn 31 with the problem of pproximting some f C[, b] with polynomil p P n t the discrete points x, x 1,, x m for

More information

Chapter 3 Polynomials

Chapter 3 Polynomials Dr M DRAIEF As described in the introduction of Chpter 1, pplictions of solving liner equtions rise in number of different settings In prticulr, we will in this chpter focus on the problem of modelling

More information

Matrices, Moments and Quadrature, cont d

Matrices, Moments and Quadrature, cont d Jim Lmbers MAT 285 Summer Session 2015-16 Lecture 2 Notes Mtrices, Moments nd Qudrture, cont d We hve described how Jcobi mtrices cn be used to compute nodes nd weights for Gussin qudrture rules for generl

More information

THE EXISTENCE-UNIQUENESS THEOREM FOR FIRST-ORDER DIFFERENTIAL EQUATIONS.

THE EXISTENCE-UNIQUENESS THEOREM FOR FIRST-ORDER DIFFERENTIAL EQUATIONS. THE EXISTENCE-UNIQUENESS THEOREM FOR FIRST-ORDER DIFFERENTIAL EQUATIONS RADON ROSBOROUGH https://intuitiveexplntionscom/picrd-lindelof-theorem/ This document is proof of the existence-uniqueness theorem

More information

Part IB Numerical Analysis

Part IB Numerical Analysis Prt IB Numericl Anlysis Theorems with proof Bsed on lectures by G. Moore Notes tken by Dexter Chu Lent 2016 These notes re not endorsed by the lecturers, nd I hve modified them (often significntly) fter

More information

Abstract inner product spaces

Abstract inner product spaces WEEK 4 Abstrct inner product spces Definition An inner product spce is vector spce V over the rel field R equipped with rule for multiplying vectors, such tht the product of two vectors is sclr, nd the

More information

Trapezoidal Rule, n = 1, x 0 = a, x 1 = b, h = b a. f (x)dx = h 2 (f (x 0) + f (x 1 )) h3

Trapezoidal Rule, n = 1, x 0 = a, x 1 = b, h = b a. f (x)dx = h 2 (f (x 0) + f (x 1 )) h3 Trpezoidl Rule, n = 1, x 0 =, x 1 = b, h = b f (x)dx = h 2 (f (x 0) + f (x 1 )) h3 12 f (ξ). Simpson s Rule: n = 3, x 0 =, x 1 = +b 2, x 2 = b, h = b 2. Qudrture Rule, double node t x 1 P 3 (x)dx = f (x

More information

New Expansion and Infinite Series

New Expansion and Infinite Series Interntionl Mthemticl Forum, Vol. 9, 204, no. 22, 06-073 HIKARI Ltd, www.m-hikri.com http://dx.doi.org/0.2988/imf.204.4502 New Expnsion nd Infinite Series Diyun Zhng College of Computer Nnjing University

More information

Exam 2, Mathematics 4701, Section ETY6 6:05 pm 7:40 pm, March 31, 2016, IH-1105 Instructor: Attila Máté 1

Exam 2, Mathematics 4701, Section ETY6 6:05 pm 7:40 pm, March 31, 2016, IH-1105 Instructor: Attila Máté 1 Exm, Mthemtics 471, Section ETY6 6:5 pm 7:4 pm, Mrch 1, 16, IH-115 Instructor: Attil Máté 1 17 copies 1. ) Stte the usul sufficient condition for the fixed-point itertion to converge when solving the eqution

More information

8 Laplace s Method and Local Limit Theorems

8 Laplace s Method and Local Limit Theorems 8 Lplce s Method nd Locl Limit Theorems 8. Fourier Anlysis in Higher DImensions Most of the theorems of Fourier nlysis tht we hve proved hve nturl generliztions to higher dimensions, nd these cn be proved

More information

Main topics for the First Midterm

Main topics for the First Midterm Min topics for the First Midterm The Midterm will cover Section 1.8, Chpters 2-3, Sections 4.1-4.8, nd Sections 5.1-5.3 (essentilly ll of the mteril covered in clss). Be sure to know the results of the

More information

Chapter 5 : Continuous Random Variables

Chapter 5 : Continuous Random Variables STAT/MATH 395 A - PROBABILITY II UW Winter Qurter 216 Néhémy Lim Chpter 5 : Continuous Rndom Vribles Nottions. N {, 1, 2,...}, set of nturl numbers (i.e. ll nonnegtive integers); N {1, 2,...}, set of ll

More information

Interpolation. Gaussian Quadrature. September 25, 2011

Interpolation. Gaussian Quadrature. September 25, 2011 Gussin Qudrture September 25, 2011 Approximtion of integrls Approximtion of integrls by qudrture Mny definite integrls cnnot be computed in closed form, nd must be pproximted numericlly. Bsic building

More information

Recitation 3: More Applications of the Derivative

Recitation 3: More Applications of the Derivative Mth 1c TA: Pdric Brtlett Recittion 3: More Applictions of the Derivtive Week 3 Cltech 2012 1 Rndom Question Question 1 A grph consists of the following: A set V of vertices. A set E of edges where ech

More information

Numerical Integration

Numerical Integration Numericl Integrtion Wouter J. Den Hn London School of Economics c 2011 by Wouter J. Den Hn June 3, 2011 Qudrture techniques I = f (x)dx n n w i f (x i ) = w i f i i=1 i=1 Nodes: x i Weights: w i Qudrture

More information

Z b. f(x)dx. Yet in the above two cases we know what f(x) is. Sometimes, engineers want to calculate an area by computing I, but...

Z b. f(x)dx. Yet in the above two cases we know what f(x) is. Sometimes, engineers want to calculate an area by computing I, but... Chpter 7 Numericl Methods 7. Introduction In mny cses the integrl f(x)dx cn be found by finding function F (x) such tht F 0 (x) =f(x), nd using f(x)dx = F (b) F () which is known s the nlyticl (exct) solution.

More information

1 Linear Least Squares

1 Linear Least Squares Lest Squres Pge 1 1 Liner Lest Squres I will try to be consistent in nottion, with n being the number of dt points, nd m < n being the number of prmeters in model function. We re interested in solving

More information

MATH 144: Business Calculus Final Review

MATH 144: Business Calculus Final Review MATH 144: Business Clculus Finl Review 1 Skills 1. Clculte severl limits. 2. Find verticl nd horizontl symptotes for given rtionl function. 3. Clculte derivtive by definition. 4. Clculte severl derivtives

More information

Advanced Calculus: MATH 410 Notes on Integrals and Integrability Professor David Levermore 17 October 2004

Advanced Calculus: MATH 410 Notes on Integrals and Integrability Professor David Levermore 17 October 2004 Advnced Clculus: MATH 410 Notes on Integrls nd Integrbility Professor Dvid Levermore 17 October 2004 1. Definite Integrls In this section we revisit the definite integrl tht you were introduced to when

More information

Best Approximation in the 2-norm

Best Approximation in the 2-norm Jim Lmbers MAT 77 Fll Semester 1-11 Lecture 1 Notes These notes correspond to Sections 9. nd 9.3 in the text. Best Approximtion in the -norm Suppose tht we wish to obtin function f n (x) tht is liner combintion

More information

Lecture 14 Numerical integration: advanced topics

Lecture 14 Numerical integration: advanced topics Lecture 14 Numericl integrtion: dvnced topics Weinn E 1,2 nd Tiejun Li 2 1 Deprtment of Mthemtics, Princeton University, weinn@princeton.edu 2 School of Mthemticl Sciences, Peking University, tieli@pku.edu.cn

More information

III. Lecture on Numerical Integration. File faclib/dattab/lecture-notes/numerical-inter03.tex /by EC, 3/14/2008 at 15:11, version 9

III. Lecture on Numerical Integration. File faclib/dattab/lecture-notes/numerical-inter03.tex /by EC, 3/14/2008 at 15:11, version 9 III Lecture on Numericl Integrtion File fclib/dttb/lecture-notes/numerical-inter03.tex /by EC, 3/14/008 t 15:11, version 9 1 Sttement of the Numericl Integrtion Problem In this lecture we consider the

More information

Lecture 12: Numerical Quadrature

Lecture 12: Numerical Quadrature Lecture 12: Numericl Qudrture J.K. Ryn@tudelft.nl WI3097TU Delft Institute of Applied Mthemtics Delft University of Technology 5 December 2012 () Numericl Qudrture 5 December 2012 1 / 46 Outline 1 Review

More information

Properties of Integrals, Indefinite Integrals. Goals: Definition of the Definite Integral Integral Calculations using Antiderivatives

Properties of Integrals, Indefinite Integrals. Goals: Definition of the Definite Integral Integral Calculations using Antiderivatives Block #6: Properties of Integrls, Indefinite Integrls Gols: Definition of the Definite Integrl Integrl Clcultions using Antiderivtives Properties of Integrls The Indefinite Integrl 1 Riemnn Sums - 1 Riemnn

More information

Numerical Analysis. Doron Levy. Department of Mathematics Stanford University

Numerical Analysis. Doron Levy. Department of Mathematics Stanford University Numericl Anlysis Doron Levy Deprtment of Mthemtics Stnford University December 1, 2005 D. Levy Prefce i D. Levy CONTENTS Contents Prefce i 1 Introduction 1 2 Interpoltion 2 2.1 Wht is Interpoltion?............................

More information

Lecture Note 4: Numerical differentiation and integration. Xiaoqun Zhang Shanghai Jiao Tong University

Lecture Note 4: Numerical differentiation and integration. Xiaoqun Zhang Shanghai Jiao Tong University Lecture Note 4: Numericl differentition nd integrtion Xioqun Zng Sngi Jio Tong University Lst updted: November, 0 Numericl Anlysis. Numericl differentition.. Introduction Find n pproximtion of f (x 0 ),

More information

Math 360: A primitive integral and elementary functions

Math 360: A primitive integral and elementary functions Mth 360: A primitive integrl nd elementry functions D. DeTurck University of Pennsylvni October 16, 2017 D. DeTurck Mth 360 001 2017C: Integrl/functions 1 / 32 Setup for the integrl prtitions Definition:

More information

Math 8 Winter 2015 Applications of Integration

Math 8 Winter 2015 Applications of Integration Mth 8 Winter 205 Applictions of Integrtion Here re few importnt pplictions of integrtion. The pplictions you my see on n exm in this course include only the Net Chnge Theorem (which is relly just the Fundmentl

More information

Review of Gaussian Quadrature method

Review of Gaussian Quadrature method Review of Gussin Qudrture method Nsser M. Asi Spring 006 compiled on Sundy Decemer 1, 017 t 09:1 PM 1 The prolem To find numericl vlue for the integrl of rel vlued function of rel vrile over specific rnge

More information

How can we approximate the area of a region in the plane? What is an interpretation of the area under the graph of a velocity function?

How can we approximate the area of a region in the plane? What is an interpretation of the area under the graph of a velocity function? Mth 125 Summry Here re some thoughts I ws hving while considering wht to put on the first midterm. The core of your studying should be the ssigned homework problems: mke sure you relly understnd those

More information

Math 270A: Numerical Linear Algebra

Math 270A: Numerical Linear Algebra Mth 70A: Numericl Liner Algebr Instructor: Michel Holst Fll Qurter 014 Homework Assignment #3 Due Give to TA t lest few dys before finl if you wnt feedbck. Exercise 3.1. (The Bsic Liner Method for Liner

More information

MATH34032: Green s Functions, Integral Equations and the Calculus of Variations 1

MATH34032: Green s Functions, Integral Equations and the Calculus of Variations 1 MATH34032: Green s Functions, Integrl Equtions nd the Clculus of Vritions 1 Section 1 Function spces nd opertors Here we gives some brief detils nd definitions, prticulrly relting to opertors. For further

More information

Math 61CM - Solutions to homework 9

Math 61CM - Solutions to homework 9 Mth 61CM - Solutions to homework 9 Cédric De Groote November 30 th, 2018 Problem 1: Recll tht the left limit of function f t point c is defined s follows: lim f(x) = l x c if for ny > 0 there exists δ

More information

ODE: Existence and Uniqueness of a Solution

ODE: Existence and Uniqueness of a Solution Mth 22 Fll 213 Jerry Kzdn ODE: Existence nd Uniqueness of Solution The Fundmentl Theorem of Clculus tells us how to solve the ordinry differentil eqution (ODE) du = f(t) dt with initil condition u() =

More information

p(x) = 3x 3 + x n 3 k=0 so the right hand side of the equality we have to show is obtained for r = b 0, s = b 1 and 2n 3 b k x k, q 2n 3 (x) =

p(x) = 3x 3 + x n 3 k=0 so the right hand side of the equality we have to show is obtained for r = b 0, s = b 1 and 2n 3 b k x k, q 2n 3 (x) = Norwegin University of Science nd Technology Deprtment of Mthemticl Sciences Pge 1 of 5 Contct during the exm: Elen Celledoni, tlf. 73593541, cell phone 48238584 PLESE NOTE: this solution is for the students

More information

Numerical Analysis. 10th ed. R L Burden, J D Faires, and A M Burden

Numerical Analysis. 10th ed. R L Burden, J D Faires, and A M Burden Numericl Anlysis 10th ed R L Burden, J D Fires, nd A M Burden Bemer Presenttion Slides Prepred by Dr. Annette M. Burden Youngstown Stte University July 9, 2015 Chpter 4.1: Numericl Differentition 1 Three-Point

More information

APPROXIMATE INTEGRATION

APPROXIMATE INTEGRATION APPROXIMATE INTEGRATION. Introduction We hve seen tht there re functions whose nti-derivtives cnnot be expressed in closed form. For these resons ny definite integrl involving these integrnds cnnot be

More information

221B Lecture Notes WKB Method

221B Lecture Notes WKB Method Clssicl Limit B Lecture Notes WKB Method Hmilton Jcobi Eqution We strt from the Schrödinger eqution for single prticle in potentil i h t ψ x, t = [ ] h m + V x ψ x, t. We cn rewrite this eqution by using

More information

Chapter 5. Numerical Integration

Chapter 5. Numerical Integration Chpter 5. Numericl Integrtion These re just summries of the lecture notes, nd few detils re included. Most of wht we include here is to be found in more detil in Anton. 5. Remrk. There re two topics with

More information

1 The Riemann Integral

1 The Riemann Integral The Riemnn Integrl. An exmple leding to the notion of integrl (res) We know how to find (i.e. define) the re of rectngle (bse height), tringle ( (sum of res of tringles). But how do we find/define n re

More information

Analytical Methods Exam: Preparatory Exercises

Analytical Methods Exam: Preparatory Exercises Anlyticl Methods Exm: Preprtory Exercises Question. Wht does it men tht (X, F, µ) is mesure spce? Show tht µ is monotone, tht is: if E F re mesurble sets then µ(e) µ(f). Question. Discuss if ech of the

More information

Lecture Notes: Orthogonal Polynomials, Gaussian Quadrature, and Integral Equations

Lecture Notes: Orthogonal Polynomials, Gaussian Quadrature, and Integral Equations 18330 Lecture Notes: Orthogonl Polynomils, Gussin Qudrture, nd Integrl Equtions Homer Reid My 1, 2014 In the previous set of notes we rrived t the definition of Chebyshev polynomils T n (x) vi the following

More information

Convex Sets and Functions

Convex Sets and Functions B Convex Sets nd Functions Definition B1 Let L, +, ) be rel liner spce nd let C be subset of L The set C is convex if, for ll x,y C nd ll [, 1], we hve 1 )x+y C In other words, every point on the line

More information

CS667 Lecture 6: Monte Carlo Integration 02/10/05

CS667 Lecture 6: Monte Carlo Integration 02/10/05 CS667 Lecture 6: Monte Crlo Integrtion 02/10/05 Venkt Krishnrj Lecturer: Steve Mrschner 1 Ide The min ide of Monte Crlo Integrtion is tht we cn estimte the vlue of n integrl by looking t lrge number of

More information

Numerical Integration

Numerical Integration Chpter 1 Numericl Integrtion Numericl differentition methods compute pproximtions to the derivtive of function from known vlues of the function. Numericl integrtion uses the sme informtion to compute numericl

More information

Definite integral. Mathematics FRDIS MENDELU

Definite integral. Mathematics FRDIS MENDELU Definite integrl Mthemtics FRDIS MENDELU Simon Fišnrová Brno 1 Motivtion - re under curve Suppose, for simplicity, tht y = f(x) is nonnegtive nd continuous function defined on [, b]. Wht is the re of the

More information

Math 1B, lecture 4: Error bounds for numerical methods

Math 1B, lecture 4: Error bounds for numerical methods Mth B, lecture 4: Error bounds for numericl methods Nthn Pflueger 4 September 0 Introduction The five numericl methods descried in the previous lecture ll operte by the sme principle: they pproximte the

More information

Euler, Ioachimescu and the trapezium rule. G.J.O. Jameson (Math. Gazette 96 (2012), )

Euler, Ioachimescu and the trapezium rule. G.J.O. Jameson (Math. Gazette 96 (2012), ) Euler, Iochimescu nd the trpezium rule G.J.O. Jmeson (Mth. Gzette 96 (0), 36 4) The following results were estblished in recent Gzette rticle [, Theorems, 3, 4]. Given > 0 nd 0 < s

More information

LECTURE. INTEGRATION AND ANTIDERIVATIVE.

LECTURE. INTEGRATION AND ANTIDERIVATIVE. ANALYSIS FOR HIGH SCHOOL TEACHERS LECTURE. INTEGRATION AND ANTIDERIVATIVE. ROTHSCHILD CAESARIA COURSE, 2015/6 1. Integrtion Historiclly, it ws the problem of computing res nd volumes, tht triggered development

More information

Definite integral. Mathematics FRDIS MENDELU. Simona Fišnarová (Mendel University) Definite integral MENDELU 1 / 30

Definite integral. Mathematics FRDIS MENDELU. Simona Fišnarová (Mendel University) Definite integral MENDELU 1 / 30 Definite integrl Mthemtics FRDIS MENDELU Simon Fišnrová (Mendel University) Definite integrl MENDELU / Motivtion - re under curve Suppose, for simplicity, tht y = f(x) is nonnegtive nd continuous function

More information

Review of basic calculus

Review of basic calculus Review of bsic clculus This brief review reclls some of the most importnt concepts, definitions, nd theorems from bsic clculus. It is not intended to tech bsic clculus from scrtch. If ny of the items below

More information

Unit #9 : Definite Integral Properties; Fundamental Theorem of Calculus

Unit #9 : Definite Integral Properties; Fundamental Theorem of Calculus Unit #9 : Definite Integrl Properties; Fundmentl Theorem of Clculus Gols: Identify properties of definite integrls Define odd nd even functions, nd reltionship to integrl vlues Introduce the Fundmentl

More information

Riemann Sums and Riemann Integrals

Riemann Sums and Riemann Integrals Riemnn Sums nd Riemnn Integrls Jmes K. Peterson Deprtment of Biologicl Sciences nd Deprtment of Mthemticl Sciences Clemson University August 26, 2013 Outline 1 Riemnn Sums 2 Riemnn Integrls 3 Properties

More information

Lecture 20: Numerical Integration III

Lecture 20: Numerical Integration III cs4: introduction to numericl nlysis /8/0 Lecture 0: Numericl Integrtion III Instructor: Professor Amos Ron Scribes: Mrk Cowlishw, Yunpeng Li, Nthnel Fillmore For the lst few lectures we hve discussed

More information

Lecture 1. Functional series. Pointwise and uniform convergence.

Lecture 1. Functional series. Pointwise and uniform convergence. 1 Introduction. Lecture 1. Functionl series. Pointwise nd uniform convergence. In this course we study mongst other things Fourier series. The Fourier series for periodic function f(x) with period 2π is

More information

Partial Derivatives. Limits. For a single variable function f (x), the limit lim

Partial Derivatives. Limits. For a single variable function f (x), the limit lim Limits Prtil Derivtives For single vrible function f (x), the limit lim x f (x) exists only if the right-hnd side limit equls to the left-hnd side limit, i.e., lim f (x) = lim f (x). x x + For two vribles

More information

Riemann Sums and Riemann Integrals

Riemann Sums and Riemann Integrals Riemnn Sums nd Riemnn Integrls Jmes K. Peterson Deprtment of Biologicl Sciences nd Deprtment of Mthemticl Sciences Clemson University August 26, 203 Outline Riemnn Sums Riemnn Integrls Properties Abstrct

More information

Calculus I-II Review Sheet

Calculus I-II Review Sheet Clculus I-II Review Sheet 1 Definitions 1.1 Functions A function is f is incresing on n intervl if x y implies f(x) f(y), nd decresing if x y implies f(x) f(y). It is clled monotonic if it is either incresing

More information

Section 4.8. D v(t j 1 ) t. (4.8.1) j=1

Section 4.8. D v(t j 1 ) t. (4.8.1) j=1 Difference Equtions to Differentil Equtions Section.8 Distnce, Position, nd the Length of Curves Although we motivted the definition of the definite integrl with the notion of re, there re mny pplictions

More information

Overview of Calculus I

Overview of Calculus I Overview of Clculus I Prof. Jim Swift Northern Arizon University There re three key concepts in clculus: The limit, the derivtive, nd the integrl. You need to understnd the definitions of these three things,

More information

Numerical Methods I Orthogonal Polynomials

Numerical Methods I Orthogonal Polynomials Numericl Methods I Orthogonl Polynomils Aleksndr Donev Cournt Institute, NYU 1 donev@cournt.nyu.edu 1 MATH-GA 2011.003 / CSCI-GA 2945.003, Fll 2014 Nov 6th, 2014 A. Donev (Cournt Institute) Lecture IX

More information

221A Lecture Notes WKB Method

221A Lecture Notes WKB Method A Lecture Notes WKB Method Hmilton Jcobi Eqution We strt from the Schrödinger eqution for single prticle in potentil i h t ψ x, t = [ ] h m + V x ψ x, t. We cn rewrite this eqution by using ψ x, t = e

More information

Sturm-Liouville Eigenvalue problem: Let p(x) > 0, q(x) 0, r(x) 0 in I = (a, b). Here we assume b > a. Let X C 2 1

Sturm-Liouville Eigenvalue problem: Let p(x) > 0, q(x) 0, r(x) 0 in I = (a, b). Here we assume b > a. Let X C 2 1 Ch.4. INTEGRAL EQUATIONS AND GREEN S FUNCTIONS Ronld B Guenther nd John W Lee, Prtil Differentil Equtions of Mthemticl Physics nd Integrl Equtions. Hildebrnd, Methods of Applied Mthemtics, second edition

More information

MORE FUNCTION GRAPHING; OPTIMIZATION. (Last edited October 28, 2013 at 11:09pm.)

MORE FUNCTION GRAPHING; OPTIMIZATION. (Last edited October 28, 2013 at 11:09pm.) MORE FUNCTION GRAPHING; OPTIMIZATION FRI, OCT 25, 203 (Lst edited October 28, 203 t :09pm.) Exercise. Let n be n rbitrry positive integer. Give n exmple of function with exctly n verticl symptotes. Give

More information

Lecture notes. Fundamental inequalities: techniques and applications

Lecture notes. Fundamental inequalities: techniques and applications Lecture notes Fundmentl inequlities: techniques nd pplictions Mnh Hong Duong Mthemtics Institute, University of Wrwick Emil: m.h.duong@wrwick.c.uk Februry 8, 207 2 Abstrct Inequlities re ubiquitous in

More information

4.4 Areas, Integrals and Antiderivatives

4.4 Areas, Integrals and Antiderivatives . res, integrls nd ntiderivtives 333. Ares, Integrls nd Antiderivtives This section explores properties of functions defined s res nd exmines some connections mong res, integrls nd ntiderivtives. In order

More information

Chapter 3 Solving Nonlinear Equations

Chapter 3 Solving Nonlinear Equations Chpter 3 Solving Nonliner Equtions 3.1 Introduction The nonliner function of unknown vrible x is in the form of where n could be non-integer. Root is the numericl vlue of x tht stisfies f ( x) 0. Grphiclly,

More information

Note 16. Stokes theorem Differential Geometry, 2005

Note 16. Stokes theorem Differential Geometry, 2005 Note 16. Stokes theorem ifferentil Geometry, 2005 Stokes theorem is the centrl result in the theory of integrtion on mnifolds. It gives the reltion between exterior differentition (see Note 14) nd integrtion

More information

An instructive toy model: two paradoxes

An instructive toy model: two paradoxes Tel Aviv University, 2006 Gussin rndom vectors 27 3 Level crossings... the fmous ice formul, undoubtedly one of the most importnt results in the ppliction of smooth stochstic processes..j. Adler nd J.E.

More information

440-2 Geometry/Topology: Differentiable Manifolds Northwestern University Solutions of Practice Problems for Final Exam

440-2 Geometry/Topology: Differentiable Manifolds Northwestern University Solutions of Practice Problems for Final Exam 440-2 Geometry/Topology: Differentible Mnifolds Northwestern University Solutions of Prctice Problems for Finl Exm 1) Using the cnonicl covering of RP n by {U α } 0 α n, where U α = {[x 0 : : x n ] RP

More information

W. We shall do so one by one, starting with I 1, and we shall do it greedily, trying

W. We shall do so one by one, starting with I 1, and we shall do it greedily, trying Vitli covers 1 Definition. A Vitli cover of set E R is set V of closed intervls with positive length so tht, for every δ > 0 nd every x E, there is some I V with λ(i ) < δ nd x I. 2 Lemm (Vitli covering)

More information

Math 520 Final Exam Topic Outline Sections 1 3 (Xiao/Dumas/Liaw) Spring 2008

Math 520 Final Exam Topic Outline Sections 1 3 (Xiao/Dumas/Liaw) Spring 2008 Mth 520 Finl Exm Topic Outline Sections 1 3 (Xio/Dums/Liw) Spring 2008 The finl exm will be held on Tuesdy, My 13, 2-5pm in 117 McMilln Wht will be covered The finl exm will cover the mteril from ll of

More information

COSC 3361 Numerical Analysis I Numerical Integration and Differentiation (III) - Gauss Quadrature and Adaptive Quadrature

COSC 3361 Numerical Analysis I Numerical Integration and Differentiation (III) - Gauss Quadrature and Adaptive Quadrature COSC 336 Numericl Anlysis I Numericl Integrtion nd Dierentition III - Guss Qudrture nd Adptive Qudrture Edgr Griel Fll 5 COSC 336 Numericl Anlysis I Edgr Griel Summry o the lst lecture I For pproximting

More information