Linear Algebra- Review And Beyond. Lecture 3

Size: px
Start display at page:

Download "Linear Algebra- Review And Beyond. Lecture 3"

Transcription

1 Linear Algebra- Review An Beyon Lecture 3 This lecture gives a wie range of materials relate to matrix. Matrix is the core of linear algebra, an it s useful in many other fiels. 1 Matrix Matrix is the concrete representation for a linear map between finite imensional vector spaces. Suppose we have two vector spaces V, W, an im V = m, im W = n, we can fin basis {α 1, α 2,, α m } of V an {β 1, β 2,, β n } of W. There is a linear map l : V W. For all v V, we have v = m j=1 x jα j, then l(v) = l( m x j α j ) = j=1 m x j l(α j ) So we just nee to consier l(α j ). l(α j ) is a vector in W, thus l(α j ) = n i=1 a ijβ i, an m m n n m l(v) = x j l(α j ) = x j a ij β i = ( a ij x j )β i More specifically, An j=1 j=1 i=1 j=1 v = {α 1, α 2,, α m } x 1 x 2. x m i=1 l(v) = {l(α 1 ), l(α 2 ),, l(α m )} l(α j ) = {β 1, β 2,, β n } l(v) = {β 1, β 2,, β n } a 1j a 2j. a nj j=1 x 1 x 2. x m a 11 a 12 a 1n a 21 a 22 a 2n... a n1 a n2 a nn 1 x 1 x 2. x m

2 Thus, for a linear mapping l : V W, the matrix uner basis {α j } an {β i } is A = (a ij ) where a ij = (l(α j )) βi The rule of aition an multiplication is omitte here. But you must be aware of the fact that the efinition of aition an multiplication is compatible with the meaning of linear mapping. Suppose U, V, W are all vector spaces with certain basis. Verify the following: If l : U V is a linear mapping with matrix A, then λa enotes the linear mapping λl. If l 1 : U V, l 2 : U V are linear mappings with matrices A 1, A 2, then A 2 + A 2 enotes the linear mapping l 1 + l 2. If l 1 : U V, l 2 : V W are linear mappings with matrices A 1, A 2, then A 2 A 1 enotes the linear mapping l 2 l 1. Remark The multiplication is associative because linear mapping is associative. proof is much clearer than the irect calculus. This way of Note that the multiplication of matrices is non-commutative. conition AB = BA is an interesting problem. However, uner what Verify that F m n is a vector space, an fin a basis. A R n n. Prove that if AB = BA for all B R n n, then there is some λ R such that A = λi. Definitions A is symmetric if A = A T. A is anti-symmetric if A = A T. A is Hermitian if A = ĀT. A is anti-hermitian if A = ĀT. A is nilpotent if A k = 0 for some k. A is iempotent if A 2 = A. A is involutory if A 2 = I. 2

3 A, B are square matrices of orer n, A = 2B I, then A is involutory if an only if B is iempotent. See F n n as a vector space Let S be the set of all symmetric matrices, an T be the set of all anti-symmetric matrices. Verify that S, T are subspaces, an fin im S, im T. Prove F n n = S T. Prove the following matrix is nilpotent: Suppose A F m n an rank(a) = 1, then α F m an β F n such that A = αβ T. This is useful ealing with matrices with rank 1. Definition(Invertible) BA = I n. A F m n is invertible if B F n m such that AB = I m an Fact A F m n is invertible if an only if m = n an et A 0. Definition(Ajoint Matrix) the ajoint matrix A = (a ij ) n n, an A ij is the algebraic cofactor of a ij, then A = A 11 A 21 A n1 A 12 A 22 A n2... A 1n A 2n A nn Fact AA = et A I. So if et A 0, A 1 = 1 et A A. Reprove Cramer theorem using x = A 1 β. I A I + A If A R n, an A k = 0 for some k. Fin the inverse of I + A + 1 2! A (k 1)! Ak 1 3

4 Definition(Elementary Transformation) Change two rows(columns) Multiply some row(column) with a non-zero number in F A λ times some row(column) to another row(column) Fin the corresponing matrices of elementary transformations. These matrices are calle elementary matrices. Remark The multiplication of matrix is non-commutative, thus you shoul be careful when oing elementary transformation by elementary matrix. Keep in min that left-multiplication is row transformation an right-multiplication is column transformation. (Schur s Formula) Suppose A F r r, B F r (n r), C F (n r) r an D F (n r) (n r), A is invertible. Prove: ( ) ( ) ( ) I r 0 A B A B CA 1 = I n r C D 0 D CA 1 B ( ) ( ) ( ) A B Ir A 1 B A 0 = C D 0 I n r C D CA 1 B ( ) ( ) ( ) ( ) I r 0 A B Ir A 1 B A 0 CA 1 = I n r C D 0 I n r 0 D CA 1 B A F n m, B F m n. Prove that λ m et(λi n AB) = λ n et(λi m BA). Suppose A F n n an rank(a) = 1. From the exercise above we know α, β F n such that A = αβ T. Prove that et(i A) = 1 β T α. Theorem(Equivalence Canonical Form) For any A F m n, we can fin P F m m, Q F n n such that ( ) Ir 0 P AQ = 0 0 where r = rank(a) an P is the prouct of elementary row transformation matrices, Q is the prouct of elementary column transformation matrices. Thus P, Q are invertible. Remark This theorem is extremely important. From now, when we want to stuy the property of matrix, we stuy the property of canonical form first. Canonical form makes problems easy to hanle. We also have other canonical form, but equivalence canonical form is the most funamental one. 4

5 Prove that equivalence is inee an equivalence relation. Theorem(Rank Inequality) ( ) A 0 rank = rank(a) + rank(b) 0 B ( ) A 0 rank rank(a) + rank(b) C B rank(ab) min{rank(a), rank(b)} If D is a submatrix of D, then rank(d ) rank(d) rank(a + B) rank(a) + rank(b) (Frobenius) rank(ab) + rank(bc) rank(b) rank(abc) If P, Q are invertible, then rank(p AQ) = rank(a) A is a matrix of orer n, prove: rank(a n ) rank(a n+1 ) rank(a n 1 ) rank(a n ) If rank(a m+1 ) = rank(a m ), then rank(a m ) = rank(a m+k ) for any integer k rank(a n ) = rank(a n+k ) for any integer k If A k = 0, then k n 2 Matrix analysis We have alreay known that F m n is a vector space. In lecture 1, we talke the structures on vector space, an norm is an important one. First we consier the norm of vector. Definition(Vector Norm) A function : R n R is a vector norm if x R n, x 0 an x = 0 if an only if x = 0 x R n, λ R, λx = λ x x, y R n, x + y x + y 5

6 Example For p 1, x p = ( n i=1 x i p ) 1 p is a vector norm. Specially, x 1 = n i=1 x i x 2 = ( n i=1 x i 2 ) 1 2 x = max 1 i n { x i } Remark The proof of triangle inequality is complicate. When p = 2, you can prove it by Cauchy-Schwarz inequality, which is the special case of Holer inequality. An one more wor, Holer inequality is a useful tool in real analysis an probability. Theorem(Holer Inequality) For p, q > 1, 1 p + 1 q = 1, xt y x p y q. We have efine many norms, but the following result tells us that all of them are equivalent. Theorem(Equivalent Norm) Suppose we have two norms α, β on R n, then there exists c 1, c 2 R such that for all x R n c 1 x α x β c 2 x α Suppose x k = (x 1 k,, xn k ) Rn an x = (x 1,, x n ) R n. Prove that lim x k x = 0 lim x i k x i = 0, i n n Although we have given the general efinition of norm, the matrix norm is ifferent, because we nee to consier the multiplication between matrices. To ensure the matrix norm has nice properties, we nee some more requirements. Definition(Matrix Norm) A function : R n n R is a matrix norm if A R n n, A 0 an A = 0 if an only if A = 0 A R n n, λ R, λa = λ A A, B R n n, A + B A + B A, B R n n, AB A B Remark Note that any matrix norm on R n n is also a vector norm on R n2. Thus matrix norm has all properties of vector norm. 6

7 Definition(Compatible) We have a matrix norm M on R n n an a vector norm v on R n, we say they are compatible if Example Define Ax v A M x v, A R n n, x R n A M = max Ax Ax v v = max x v=1 x x v This is a compatible matrix norm. This is calle the operator norm, an it will appear in functional analysis again. Actually, we often efine norm of linear operator between norme vector space in this way. Example In the last example, we can take v = 1, 2 an. In fact v = 1, then the inuce matrix norm is A 1 = max 1 j n n i=1 a ij v =, then the inuce matrix norm is A = max 1 i n n j=1 a ij A, B R n an A is invertible. If A B < 1 A 1 then B is also invertible. Definition(Convergence) say A n converges to A. A n, A R n, is a matrix norm, if lim n A n A = 0, we We claim that R n n with a matrix norm is a Banach space. Thus, any Cauchy sequence is convergent. A R n n, is a matrix norm, then A k A k. If A < 1, then I A is invertible, an (I A) 1 1. (Compare with 1 A the nilpotent case) For matrix A R n n, we efine e A = A k k=0. k! Prove that this is well-efine. Fin the inverse of e A. (Compare with the nilpotent case) Prove that if AB = BA, then e A+B = e A e B (Use convolution) Fin a counterexample such that e A+B e A e B 7

8 3 Calculus for vector an matrix value function In mathematical analysis, you have learne many things about vector value function. Suppose x(t) = (x 1 (t), x 2 (t),, x n (t)) is a vector value function of t in R n, we can iscuss continuity an erivative using the norm we learne above. Definition(Continuity) x(t) is continuous at t 0 if lim t t0 x(t) x(t 0 ) = 0. Definition(Derivative) If lim h 0 x(t 0+h) x(t 0 ) h at t 0, an the erivative at t 0 is x (t 0 ). x (t 0 ) = 0, we say x(t) is ifferentiable The case of matrix value function is all the same because we can see matrix as a vector. But note that when we put ifferentiation an linear function together, something nice appears. l is a linear function on R n, x(t) is a ifferentiable vector value function in R n, then t l(x(t)) = l( t x(t)) A(t) is a matrix value function, then t tr(a(t)) = tr( t A(t)) Theorem Suppose A(t) is a ifferentiable an invertible matrix value function, then A 1 (t) is ifferentiable, an t A 1 = A 1 ( t A)A 1 Remark Note that chain rule is not true for matrix value function because matrix multiplication is not commutative. An when we ifferentiate the prouct of matrix/vector, the orer can t be change. Prove by inuction that t Ak = A A k 1 + AA A k A k 1 A Theorem Suppose p is a polynomial, A(t) is a matrix value function, If A(t 0 ) is commutative with A (t 0 ), then the chain rule hols at t 0 : t tr(p(a)) = tr(p (A)A ) t p(a) t 0 = p (A)A t0 8

9 Now we come to consier multiple linear function L(a 1,, a n ). If x 1 (t),, x n (t) are ifferentiable vector value function, then L(x 1 (t),, x n (t)) is also ifferentiable. An it s not har to prove: t L(x 1(t),, x n (t)) = L(x 1(t),, x n (t)) + + L(x 1 (t),, x n(t)) As you may have guesse, an application of this formula is eterminant. Determinant is a multiple linear function, so t et(x 1(t),, x n (t)) = et(x 1(t),, x n (t)) + + et(x 1 (t),, x n(t)) Use the ifferentiation formula of eterminant, prove: X(t) is a ifferentiable matrix value function an X(0) = I, then t et X(t) t=0= tr(x (0)) X(t) is a ifferentiable matrix value function an X(t) is always invertible, then t ln et Y (t) = tr(y 1 (t)y (t)) 4 Applications in ifferential geometry I will introuce some basic ieas of ifferential geometry here. Definition(Curve) A mapping r : (a, b) R 3, t (x(t), y(t), z(t)) is a smooth curve if it s infinitely ifferentiable an r/t 0. We can take parameter s such that T (s) = r is the unit tangent vector. Because (T, T ) = 1, s ifferentiate, we know (T, T ) = 0, thus T T. Let N = 1 T, we immeiately know N T T an N = 1. Let κ = T = x 2 + y 2 + z 2, T = κn. An let B = T N, consier the relations between (T, N, B ) an (T, N, B). Differentiate (N, T ) = 0, we get (N, T ) = (N, T ) = κ. Let τ = (N, B), from (N, N ) = 0 an (T, N, B) is orthogonal, we know N = κt + τb. An B = T N + T N = T ( κt + τb) = τn Thus, using the language of matrix, we get T N = κ s B κ τ τ T N B 9

10 Suppose {e 1 (t), e 2 (t),, e n (t)} is a stanar orthogonal basis of R n, an e 1 (t) e 1 (t) e 2 (t) e 2 (t) t. e n (t) = A. e n (t) Prove that A + A T = 0. Definition(Smooth surface) A mapping r : D = {(u, v)} R 3, (u, v) (x(u, v), y(u, v), z(u, v)) is a smooth surface, if it s infinitely ifferentiable an r u r v 0 everywhere. Fix u = a, we get a curve r(a, v), an the tangent vector is r v (a, v). Similarly, r u (u, b) is a tangent vector. Consier a curve on u, say r(u(t), v(t)), then the tangent vector is r u +r t v v, t it s a linear combination of r u, r v. Thus, r u, r v span the tangent surface of, we enote this by T p. By the meaning of ifferentiation, a small arc r = r u u + r v v. To calculate the length, We let then (r, r) = (r u u + r v v, r u u + r v v) = (r u, r u )u 2 + 2(r u, r v )uv + (r v, r v )v 2 E = (r u, r u ) = ( x u )2 + ( y u )2 + ( z u )2 F = (r u, r v ) = x x u v + y y u v + z z u v G = (r v, r v ) = ( x v )2 + ( y v )2 + ( z v )2 ( E F r 2 = (u, v) F G This is calle the first funamental form of surface. ) ( u v ) Calculate the first funamental form Cyliner: r(u, v) = (x(u), y(u), v) Plane:r(u, v) = (u, v, 0) 10

11 5 Matrix group Suppose V is a vector space on fiel F, we use M n (F ) to enote all square matrices of orer n on F, an use GL n (F ) to enote all invertible matrices of orer n on F. M n (F ) is an abelian group uner matrix aition, but it s not a group uner matrix multiplication because not every matrix have an inverse. However, GL n (F ) is a group uner matrix multiplication, we call it general linear group. Example For n = 1, GL n (F ) = F. For a prime p, F p is a fiel. Fin GL n (F p ). We often stuy the subgroup of GL n (F ), which is calle classical group. Definition(Special Linear Group) SL n (F ) = {A GL n (F ) et A = 1}. ( a b Example SL 2 (Z/nZ) = { c ) a, b, c, Z/nZ, a bc = 1} Given the stanar inner prouct on R n, say, < x, y >= x T y, then A GL n (R) is an orthogonal matrix if A contains the inner prouct, i.e., < Ax, Ay >= x T A T Ay = x T y. Thus A T A = AA T = I. Definition(Orthogonal Group) O n (R) = {A GL n (R) A T A = AA T = I}. We have other inner prouct other than the stanar inner prouct, more specifically, bilinear form. An we know that for a nonegenerately bilinear form Q, there exists a basis such that Q(x, y) = x T ( Ip I q ) y In this case, the matrices satisfying Q(x, y) = Q(Ax, Ay) form a group. Definition(Generalize Orthogonal Group) O p,q = {A GL n (R) A T ( Ip I q ) A = ( Ip I q ) } An SO n (R) = O n (R) SL n (R) is calle the special orthogonal group, SO p,q (R) = O p,q (R) SL n (R) is calle the generalize special orthogonal group. 11

12 Example ( cos θ sin θ SO 2 (R) = { sin θ cos θ ) θ R} Prove that ϕ : R R, t e ta is a homomorphism for a fixe a. An all homomorphism from R to R must be of this form. Prove that ϕ : R GL n (R), t e ta is a homomorphism for a fixe A R n n. An all homomorphism from R to GL n (R) must be of this form. Let S n enote the symmetric group of egree n, an let F be an arbitrary fiel. To each permutation σ S n, efine M(σ) = n i=1 E σ(i),i. Show that M is a homomorphism from S n to GL n (K). 6 Numerical linear algebra 6.1 Perturbation You can regar this part as an introuction to computational mathematic. We focus on solving linear system Ax = b on a computer. Actually we can t get accurate solution because of the truncation error. Consier the linear system Ax = b an a perturbation on A an b we get (A + δa)(x + δx) = b + δb. Plugging in Ax = b, we get (A + δa)δx = δb δax Note that A+δA = A(I +A 1 δa). The perturbation is small enough such that A 1 δa < 1. Accoring to the result in exercise, we know I + A 1 δa is invertible, an Thus, (I + A 1 δa) A 1 δa δx = (A + δa) 1 (δb δax) = (I + A 1 δa) 1 A 1 (δb δax) δx (I +A 1 δa) 1 A 1 δb δax Diviing by x an note that b A x, 1 1 A 1 δa A 1 ( δb + δa x ) δx x A 1 A 1 A 1 δa ( δb + δa b A ) The number A A 1, name conition number gives an upper boun of the perturbation of solution, an we use κ(a) to enote it. The smaller κ(a) is, the more accurate the numerical solution is. 12

13 Solving a linear system is perfect theoretically, for example, Cramer s theorem, x = A 1 b. But we have mentione that these methos are awful in practice. So we nee to fin numerical methos. Generally speaking, there are two types of numerical metho:irectly an iteratively. 6.2 Direct metho The main iea of irect metho is ecomposition. First, consier the conition that A is upper triangle or lower triangle, then the linear system is easy to solve. For general coefficient matrix A, if we can ecompose A into LU where L is lower triangle, U is upper triangle, then the problem is easy. Suppose A R n n, we have n 2 elements in total. Both L an U have n 2 +n elements, so if we want to solve LU = A, we have n 2 equations an n 2 + n unknown 2 number. It has solution in general! In fact, we can assume the number of L in the iagonal positions are all 1. 1 l l n1 l n2 1 u 11 u 1,n 1 u 1n..... u n 1,n 1 u n 1,n u nn = a 11 a 12 a 1n a 21 a 22 a 2n... a n1 a n2 a nn We can get the first row of U, then the first column of L, then the secon row of U, the secon column of L an repeat this until we are one. On the other han, we can get the first column of U then the first row of L instea. However, this process is a little bit stupi. Recall the Gauss cancelation, we can o this by elementary row transformation. Let L k = I l k e T k, where l k = (0,, 0, l k+1,, l n ) T. Then for x = (x 1,, x n ) T R n, L k x = (x 1,, x k, x k+1 l k+1,k x k,, x n l n,k x k ) T Take l i,k = x i x k, i = k+1,, n, we have L k x = (x 1,, x k, 0,, 0) T. Thus, we can transform A into an upper triangle matrix U with prouct of such L k. An obviously the prouct of such L k, enote by L is lower triangle. So we get an LA = U. Note that Ax = b LAx = Lb Ux = Lb, we only nee to solve Ux = Lb. 6.3 Iterative metho For Ax = b, we ecompose A into three parts:a = D L U, where D is the iagonal elements of A, an L is lower triangle, U is upper triangle. Then we have (D L U)x = b. That is x = D 1 (L + U)x + D 1 b. For an initial value x 0 R n, let x k+1 = D 1 (L + U)x k + D 1 b we get a sequence of vectors. This is calle Jacobi iteration. 13

14 Another iea is we can use new terms of x k+1 to o iteration. That is x k+1 = D 1 Lx k+1 + D 1 Ux k + D 1 b. By calculation we know This is calle Gauss-Seiel iteration. x k+1 = (D L) 1 Ux k + (D L) 1 b Note that both iteration have the form x k+1 = Mx k + g. Suppose the accurate solution is x, we must have x = Mx = g. Let e k = x k x, we get e k+1 = Me k. If e k 0, then the iteration converges to the accurate solution. Note that e k = M k e 0, so if M < 1, the iteration must be efficient! 14

SYSTEMS OF DIFFERENTIAL EQUATIONS, EULER S FORMULA. where L is some constant, usually called the Lipschitz constant. An example is

SYSTEMS OF DIFFERENTIAL EQUATIONS, EULER S FORMULA. where L is some constant, usually called the Lipschitz constant. An example is SYSTEMS OF DIFFERENTIAL EQUATIONS, EULER S FORMULA. Uniqueness for solutions of ifferential equations. We consier the system of ifferential equations given by x = v( x), () t with a given initial conition

More information

Euler equations for multiple integrals

Euler equations for multiple integrals Euler equations for multiple integrals January 22, 2013 Contents 1 Reminer of multivariable calculus 2 1.1 Vector ifferentiation......................... 2 1.2 Matrix ifferentiation........................

More information

The derivative of a function f(x) is another function, defined in terms of a limiting expression: f(x + δx) f(x)

The derivative of a function f(x) is another function, defined in terms of a limiting expression: f(x + δx) f(x) Y. D. Chong (2016) MH2801: Complex Methos for the Sciences 1. Derivatives The erivative of a function f(x) is another function, efine in terms of a limiting expression: f (x) f (x) lim x δx 0 f(x + δx)

More information

6 General properties of an autonomous system of two first order ODE

6 General properties of an autonomous system of two first order ODE 6 General properties of an autonomous system of two first orer ODE Here we embark on stuying the autonomous system of two first orer ifferential equations of the form ẋ 1 = f 1 (, x 2 ), ẋ 2 = f 2 (, x

More information

Sturm-Liouville Theory

Sturm-Liouville Theory LECTURE 5 Sturm-Liouville Theory In the three preceing lectures I emonstrate the utility of Fourier series in solving PDE/BVPs. As we ll now see, Fourier series are just the tip of the iceberg of the theory

More information

JUST THE MATHS UNIT NUMBER DIFFERENTIATION 2 (Rates of change) A.J.Hobson

JUST THE MATHS UNIT NUMBER DIFFERENTIATION 2 (Rates of change) A.J.Hobson JUST THE MATHS UNIT NUMBER 10.2 DIFFERENTIATION 2 (Rates of change) by A.J.Hobson 10.2.1 Introuction 10.2.2 Average rates of change 10.2.3 Instantaneous rates of change 10.2.4 Derivatives 10.2.5 Exercises

More information

Problem Sheet 2: Eigenvalues and eigenvectors and their use in solving linear ODEs

Problem Sheet 2: Eigenvalues and eigenvectors and their use in solving linear ODEs Problem Sheet 2: Eigenvalues an eigenvectors an their use in solving linear ODEs If you fin any typos/errors in this problem sheet please email jk28@icacuk The material in this problem sheet is not examinable

More information

Calculus of Variations

Calculus of Variations 16.323 Lecture 5 Calculus of Variations Calculus of Variations Most books cover this material well, but Kirk Chapter 4 oes a particularly nice job. x(t) x* x*+ αδx (1) x*- αδx (1) αδx (1) αδx (1) t f t

More information

The Exact Form and General Integrating Factors

The Exact Form and General Integrating Factors 7 The Exact Form an General Integrating Factors In the previous chapters, we ve seen how separable an linear ifferential equations can be solve using methos for converting them to forms that can be easily

More information

Integration Review. May 11, 2013

Integration Review. May 11, 2013 Integration Review May 11, 2013 Goals: Review the funamental theorem of calculus. Review u-substitution. Review integration by parts. Do lots of integration eamples. 1 Funamental Theorem of Calculus In

More information

Linear First-Order Equations

Linear First-Order Equations 5 Linear First-Orer Equations Linear first-orer ifferential equations make up another important class of ifferential equations that commonly arise in applications an are relatively easy to solve (in theory)

More information

Implicit Differentiation

Implicit Differentiation Implicit Differentiation Thus far, the functions we have been concerne with have been efine explicitly. A function is efine explicitly if the output is given irectly in terms of the input. For instance,

More information

Agmon Kolmogorov Inequalities on l 2 (Z d )

Agmon Kolmogorov Inequalities on l 2 (Z d ) Journal of Mathematics Research; Vol. 6, No. ; 04 ISSN 96-9795 E-ISSN 96-9809 Publishe by Canaian Center of Science an Eucation Agmon Kolmogorov Inequalities on l (Z ) Arman Sahovic Mathematics Department,

More information

Lecture 6: Calculus. In Song Kim. September 7, 2011

Lecture 6: Calculus. In Song Kim. September 7, 2011 Lecture 6: Calculus In Song Kim September 7, 20 Introuction to Differential Calculus In our previous lecture we came up with several ways to analyze functions. We saw previously that the slope of a linear

More information

CHAPTER 1 : DIFFERENTIABLE MANIFOLDS. 1.1 The definition of a differentiable manifold

CHAPTER 1 : DIFFERENTIABLE MANIFOLDS. 1.1 The definition of a differentiable manifold CHAPTER 1 : DIFFERENTIABLE MANIFOLDS 1.1 The efinition of a ifferentiable manifol Let M be a topological space. This means that we have a family Ω of open sets efine on M. These satisfy (1), M Ω (2) the

More information

Rank, Trace, Determinant, Transpose an Inverse of a Matrix Let A be an n n square matrix: A = a11 a1 a1n a1 a an a n1 a n a nn nn where is the jth col

Rank, Trace, Determinant, Transpose an Inverse of a Matrix Let A be an n n square matrix: A = a11 a1 a1n a1 a an a n1 a n a nn nn where is the jth col Review of Linear Algebra { E18 Hanout Vectors an Their Inner Proucts Let X an Y be two vectors: an Their inner prouct is ene as X =[x1; ;x n ] T Y =[y1; ;y n ] T (X; Y ) = X T Y = x k y k k=1 where T an

More information

PDE Notes, Lecture #11

PDE Notes, Lecture #11 PDE Notes, Lecture # from Professor Jalal Shatah s Lectures Febuary 9th, 2009 Sobolev Spaces Recall that for u L loc we can efine the weak erivative Du by Du, φ := udφ φ C0 If v L loc such that Du, φ =

More information

Math Notes on differentials, the Chain Rule, gradients, directional derivative, and normal vectors

Math Notes on differentials, the Chain Rule, gradients, directional derivative, and normal vectors Math 18.02 Notes on ifferentials, the Chain Rule, graients, irectional erivative, an normal vectors Tangent plane an linear approximation We efine the partial erivatives of f( xy, ) as follows: f f( x+

More information

Many problems in physics, engineering, and chemistry fall in a general class of equations of the form. d dx. d dx

Many problems in physics, engineering, and chemistry fall in a general class of equations of the form. d dx. d dx Math 53 Notes on turm-liouville equations Many problems in physics, engineering, an chemistry fall in a general class of equations of the form w(x)p(x) u ] + (q(x) λ) u = w(x) on an interval a, b], plus

More information

Lectures - Week 10 Introduction to Ordinary Differential Equations (ODES) First Order Linear ODEs

Lectures - Week 10 Introduction to Ordinary Differential Equations (ODES) First Order Linear ODEs Lectures - Week 10 Introuction to Orinary Differential Equations (ODES) First Orer Linear ODEs When stuying ODEs we are consiering functions of one inepenent variable, e.g., f(x), where x is the inepenent

More information

Notes on Lie Groups, Lie algebras, and the Exponentiation Map Mitchell Faulk

Notes on Lie Groups, Lie algebras, and the Exponentiation Map Mitchell Faulk Notes on Lie Groups, Lie algebras, an the Exponentiation Map Mitchell Faulk 1. Preliminaries. In these notes, we concern ourselves with special objects calle matrix Lie groups an their corresponing Lie

More information

Math 11 Fall 2016 Section 1 Monday, September 19, Definition: A vector parametric equation for the line parallel to vector v = x v, y v, z v

Math 11 Fall 2016 Section 1 Monday, September 19, Definition: A vector parametric equation for the line parallel to vector v = x v, y v, z v Math Fall 06 Section Monay, September 9, 06 First, some important points from the last class: Definition: A vector parametric equation for the line parallel to vector v = x v, y v, z v passing through

More information

Two formulas for the Euler ϕ-function

Two formulas for the Euler ϕ-function Two formulas for the Euler ϕ-function Robert Frieman A multiplication formula for ϕ(n) The first formula we want to prove is the following: Theorem 1. If n 1 an n 2 are relatively prime positive integers,

More information

Math 300 Winter 2011 Advanced Boundary Value Problems I. Bessel s Equation and Bessel Functions

Math 300 Winter 2011 Advanced Boundary Value Problems I. Bessel s Equation and Bessel Functions Math 3 Winter 2 Avance Bounary Value Problems I Bessel s Equation an Bessel Functions Department of Mathematical an Statistical Sciences University of Alberta Bessel s Equation an Bessel Functions We use

More information

Matrix Theory. A.Holst, V.Ufnarovski

Matrix Theory. A.Holst, V.Ufnarovski Matrix Theory AHolst, VUfnarovski 55 HINTS AND ANSWERS 9 55 Hints and answers There are two different approaches In the first one write A as a block of rows and note that in B = E ij A all rows different

More information

The Non-abelian Hodge Correspondence for Non-Compact Curves

The Non-abelian Hodge Correspondence for Non-Compact Curves 1 Section 1 Setup The Non-abelian Hoge Corresponence for Non-Compact Curves Chris Elliott May 8, 2011 1 Setup In this talk I will escribe the non-abelian Hoge theory of a non-compact curve. This was worke

More information

Section 7.1: Integration by Parts

Section 7.1: Integration by Parts Section 7.1: Integration by Parts 1. Introuction to Integration Techniques Unlike ifferentiation where there are a large number of rules which allow you (in principle) to ifferentiate any function, the

More information

MAT 545: Complex Geometry Fall 2008

MAT 545: Complex Geometry Fall 2008 MAT 545: Complex Geometry Fall 2008 Notes on Lefschetz Decomposition 1 Statement Let (M, J, ω) be a Kahler manifol. Since ω is a close 2-form, it inuces a well-efine homomorphism L: H k (M) H k+2 (M),

More information

Lecture 2 Lagrangian formulation of classical mechanics Mechanics

Lecture 2 Lagrangian formulation of classical mechanics Mechanics Lecture Lagrangian formulation of classical mechanics 70.00 Mechanics Principle of stationary action MATH-GA To specify a motion uniquely in classical mechanics, it suffices to give, at some time t 0,

More information

Designing Information Devices and Systems II Fall 2017 Note Theorem: Existence and Uniqueness of Solutions to Differential Equations

Designing Information Devices and Systems II Fall 2017 Note Theorem: Existence and Uniqueness of Solutions to Differential Equations EECS 6B Designing Information Devices an Systems II Fall 07 Note 3 Secon Orer Differential Equations Secon orer ifferential equations appear everywhere in the real worl. In this note, we will walk through

More information

DIFFERENTIAL GEOMETRY, LECTURE 15, JULY 10

DIFFERENTIAL GEOMETRY, LECTURE 15, JULY 10 DIFFERENTIAL GEOMETRY, LECTURE 15, JULY 10 5. Levi-Civita connection From now on we are intereste in connections on the tangent bunle T X of a Riemanninam manifol (X, g). Out main result will be a construction

More information

ELEC3114 Control Systems 1

ELEC3114 Control Systems 1 ELEC34 Control Systems Linear Systems - Moelling - Some Issues Session 2, 2007 Introuction Linear systems may be represente in a number of ifferent ways. Figure shows the relationship between various representations.

More information

Exam 2 Review Solutions

Exam 2 Review Solutions Exam Review Solutions 1. True or False, an explain: (a) There exists a function f with continuous secon partial erivatives such that f x (x, y) = x + y f y = x y False. If the function has continuous secon

More information

The Natural Logarithm

The Natural Logarithm The Natural Logarithm -28-208 In earlier courses, you may have seen logarithms efine in terms of raising bases to powers. For eample, log 2 8 = 3 because 2 3 = 8. In those terms, the natural logarithm

More information

First Order Linear Differential Equations

First Order Linear Differential Equations LECTURE 6 First Orer Linear Differential Equations A linear first orer orinary ifferential equation is a ifferential equation of the form ( a(xy + b(xy = c(x. Here y represents the unknown function, y

More information

2.1 Derivatives and Rates of Change

2.1 Derivatives and Rates of Change 1a 1b 2.1 Derivatives an Rates of Change Tangent Lines Example. Consier y f x x 2 0 2 x-, 0 4 y-, f(x) axes, curve C Consier a smooth curve C. A line tangent to C at a point P both intersects C at P an

More information

Schrödinger s equation.

Schrödinger s equation. Physics 342 Lecture 5 Schröinger s Equation Lecture 5 Physics 342 Quantum Mechanics I Wenesay, February 3r, 2010 Toay we iscuss Schröinger s equation an show that it supports the basic interpretation of

More information

Math 1271 Solutions for Fall 2005 Final Exam

Math 1271 Solutions for Fall 2005 Final Exam Math 7 Solutions for Fall 5 Final Eam ) Since the equation + y = e y cannot be rearrange algebraically in orer to write y as an eplicit function of, we must instea ifferentiate this relation implicitly

More information

Math 1B, lecture 8: Integration by parts

Math 1B, lecture 8: Integration by parts Math B, lecture 8: Integration by parts Nathan Pflueger 23 September 2 Introuction Integration by parts, similarly to integration by substitution, reverses a well-known technique of ifferentiation an explores

More information

Pure Further Mathematics 1. Revision Notes

Pure Further Mathematics 1. Revision Notes Pure Further Mathematics Revision Notes June 20 2 FP JUNE 20 SDB Further Pure Complex Numbers... 3 Definitions an arithmetical operations... 3 Complex conjugate... 3 Properties... 3 Complex number plane,

More information

d dx But have you ever seen a derivation of these results? We ll prove the first result below. cos h 1

d dx But have you ever seen a derivation of these results? We ll prove the first result below. cos h 1 Lecture 5 Some ifferentiation rules Trigonometric functions (Relevant section from Stewart, Seventh Eition: Section 3.3) You all know that sin = cos cos = sin. () But have you ever seen a erivation of

More information

Applications of the Wronskian to ordinary linear differential equations

Applications of the Wronskian to ordinary linear differential equations Physics 116C Fall 2011 Applications of the Wronskian to orinary linear ifferential equations Consier a of n continuous functions y i (x) [i = 1,2,3,...,n], each of which is ifferentiable at least n times.

More information

ALGEBRAIC AND ANALYTIC PROPERTIES OF ARITHMETIC FUNCTIONS

ALGEBRAIC AND ANALYTIC PROPERTIES OF ARITHMETIC FUNCTIONS ALGEBRAIC AND ANALYTIC PROPERTIES OF ARITHMETIC FUNCTIONS MARK SCHACHNER Abstract. When consiere as an algebraic space, the set of arithmetic functions equippe with the operations of pointwise aition an

More information

Review of Differentiation and Integration for Ordinary Differential Equations

Review of Differentiation and Integration for Ordinary Differential Equations Schreyer Fall 208 Review of Differentiation an Integration for Orinary Differential Equations In this course you will be expecte to be able to ifferentiate an integrate quickly an accurately. Many stuents

More information

A. Incorrect! The letter t does not appear in the expression of the given integral

A. Incorrect! The letter t does not appear in the expression of the given integral AP Physics C - Problem Drill 1: The Funamental Theorem of Calculus Question No. 1 of 1 Instruction: (1) Rea the problem statement an answer choices carefully () Work the problems on paper as neee (3) Question

More information

Knowledge Discovery and Data Mining 1 (VO) ( )

Knowledge Discovery and Data Mining 1 (VO) ( ) Knowledge Discovery and Data Mining 1 (VO) (707.003) Review of Linear Algebra Denis Helic KTI, TU Graz Oct 9, 2014 Denis Helic (KTI, TU Graz) KDDM1 Oct 9, 2014 1 / 74 Big picture: KDDM Probability Theory

More information

Tractability results for weighted Banach spaces of smooth functions

Tractability results for weighted Banach spaces of smooth functions Tractability results for weighte Banach spaces of smooth functions Markus Weimar Mathematisches Institut, Universität Jena Ernst-Abbe-Platz 2, 07740 Jena, Germany email: markus.weimar@uni-jena.e March

More information

QF101: Quantitative Finance September 5, Week 3: Derivatives. Facilitator: Christopher Ting AY 2017/2018. f ( x + ) f(x) f(x) = lim

QF101: Quantitative Finance September 5, Week 3: Derivatives. Facilitator: Christopher Ting AY 2017/2018. f ( x + ) f(x) f(x) = lim QF101: Quantitative Finance September 5, 2017 Week 3: Derivatives Facilitator: Christopher Ting AY 2017/2018 I recoil with ismay an horror at this lamentable plague of functions which o not have erivatives.

More information

Similar Operators and a Functional Calculus for the First-Order Linear Differential Operator

Similar Operators and a Functional Calculus for the First-Order Linear Differential Operator Avances in Applie Mathematics, 9 47 999 Article ID aama.998.067, available online at http: www.iealibrary.com on Similar Operators an a Functional Calculus for the First-Orer Linear Differential Operator

More information

Final Exam Study Guide and Practice Problems Solutions

Final Exam Study Guide and Practice Problems Solutions Final Exam Stuy Guie an Practice Problems Solutions Note: These problems are just some of the types of problems that might appear on the exam. However, to fully prepare for the exam, in aition to making

More information

First Order Linear Differential Equations

First Order Linear Differential Equations LECTURE 8 First Orer Linear Differential Equations We now turn our attention to the problem of constructing analytic solutions of ifferential equations; that is to say,solutions that can be epresse in

More information

The Principle of Least Action

The Principle of Least Action Chapter 7. The Principle of Least Action 7.1 Force Methos vs. Energy Methos We have so far stuie two istinct ways of analyzing physics problems: force methos, basically consisting of the application of

More information

Math 115 Section 018 Course Note

Math 115 Section 018 Course Note Course Note 1 General Functions Definition 1.1. A function is a rule that takes certain numbers as inputs an assigns to each a efinite output number. The set of all input numbers is calle the omain of

More information

Lecture 1 Review: Linear models have the form (in matrix notation) Y = Xβ + ε,

Lecture 1 Review: Linear models have the form (in matrix notation) Y = Xβ + ε, 2. REVIEW OF LINEAR ALGEBRA 1 Lecture 1 Review: Linear models have the form (in matrix notation) Y = Xβ + ε, where Y n 1 response vector and X n p is the model matrix (or design matrix ) with one row for

More information

19 Eigenvalues, Eigenvectors, Ordinary Differential Equations, and Control

19 Eigenvalues, Eigenvectors, Ordinary Differential Equations, and Control 19 Eigenvalues, Eigenvectors, Orinary Differential Equations, an Control This section introuces eigenvalues an eigenvectors of a matrix, an iscusses the role of the eigenvalues in etermining the behavior

More information

Assignment 1. g i (x 1,..., x n ) dx i = 0. i=1

Assignment 1. g i (x 1,..., x n ) dx i = 0. i=1 Assignment 1 Golstein 1.4 The equations of motion for the rolling isk are special cases of general linear ifferential equations of constraint of the form g i (x 1,..., x n x i = 0. i=1 A constraint conition

More information

Calculus of Variations

Calculus of Variations Calculus of Variations Lagrangian formalism is the main tool of theoretical classical mechanics. Calculus of Variations is a part of Mathematics which Lagrangian formalism is base on. In this section,

More information

Acute sets in Euclidean spaces

Acute sets in Euclidean spaces Acute sets in Eucliean spaces Viktor Harangi April, 011 Abstract A finite set H in R is calle an acute set if any angle etermine by three points of H is acute. We examine the maximal carinality α() of

More information

NORMS ON SPACE OF MATRICES

NORMS ON SPACE OF MATRICES NORMS ON SPACE OF MATRICES. Operator Norms on Space of linear maps Let A be an n n real matrix and x 0 be a vector in R n. We would like to use the Picard iteration method to solve for the following system

More information

HOMEWORK PROBLEMS FROM STRANG S LINEAR ALGEBRA AND ITS APPLICATIONS (4TH EDITION)

HOMEWORK PROBLEMS FROM STRANG S LINEAR ALGEBRA AND ITS APPLICATIONS (4TH EDITION) HOMEWORK PROBLEMS FROM STRANG S LINEAR ALGEBRA AND ITS APPLICATIONS (4TH EDITION) PROFESSOR STEVEN MILLER: BROWN UNIVERSITY: SPRING 2007 1. CHAPTER 1: MATRICES AND GAUSSIAN ELIMINATION Page 9, # 3: Describe

More information

Robustness and Perturbations of Minimal Bases

Robustness and Perturbations of Minimal Bases Robustness an Perturbations of Minimal Bases Paul Van Dooren an Froilán M Dopico December 9, 2016 Abstract Polynomial minimal bases of rational vector subspaces are a classical concept that plays an important

More information

A Constructive Inversion Framework for Twisted Convolution

A Constructive Inversion Framework for Twisted Convolution A Constructive Inversion Framework for Twiste Convolution Yonina C. Elar, Ewa Matusiak, Tobias Werther June 30, 2006 Subject Classification: 44A35, 15A30, 42C15 Key Wors: Twiste convolution, Wiener s Lemma,

More information

Witten s Proof of Morse Inequalities

Witten s Proof of Morse Inequalities Witten s Proof of Morse Inequalities by Igor Prokhorenkov Let M be a smooth, compact, oriente manifol with imension n. A Morse function is a smooth function f : M R such that all of its critical points

More information

model considered before, but the prey obey logistic growth in the absence of predators. In

model considered before, but the prey obey logistic growth in the absence of predators. In 5.2. First Orer Systems of Differential Equations. Phase Portraits an Linearity. Section Objective(s): Moifie Preator-Prey Moel. Graphical Representations of Solutions. Phase Portraits. Vector Fiels an

More information

Characteristic classes of vector bundles

Characteristic classes of vector bundles Characteristic classes of vector bunles Yoshinori Hashimoto 1 Introuction Let be a smooth, connecte, compact manifol of imension n without bounary, an p : E be a real or complex vector bunle of rank k

More information

Function Spaces. 1 Hilbert Spaces

Function Spaces. 1 Hilbert Spaces Function Spaces A function space is a set of functions F that has some structure. Often a nonparametric regression function or classifier is chosen to lie in some function space, where the assume structure

More information

Orthogonal $*$-basis of relative symmetry classes of polynomials

Orthogonal $*$-basis of relative symmetry classes of polynomials Electronic Journal of Linear Algebra Volume 30 Volume 30 (2015) Article 11 2015 Orthogonal $*$-basis of relative symmetry classes of polynomials Kijti Rotes Department of Mathematics, Faculty of Science,

More information

Table of Common Derivatives By David Abraham

Table of Common Derivatives By David Abraham Prouct an Quotient Rules: Table of Common Derivatives By Davi Abraham [ f ( g( ] = [ f ( ] g( + f ( [ g( ] f ( = g( [ f ( ] g( g( f ( [ g( ] Trigonometric Functions: sin( = cos( cos( = sin( tan( = sec

More information

SYDE 112, LECTURE 1: Review & Antidifferentiation

SYDE 112, LECTURE 1: Review & Antidifferentiation SYDE 112, LECTURE 1: Review & Antiifferentiation 1 Course Information For a etaile breakown of the course content an available resources, see the Course Outline. Other relevant information for this section

More information

Integration by Parts

Integration by Parts Integration by Parts 6-3-207 If u an v are functions of, the Prouct Rule says that (uv) = uv +vu Integrate both sies: (uv) = uv = uv + u v + uv = uv vu, vu v u, I ve written u an v as shorthan for u an

More information

Chapter 6: Integration: partial fractions and improper integrals

Chapter 6: Integration: partial fractions and improper integrals Chapter 6: Integration: partial fractions an improper integrals Course S3, 006 07 April 5, 007 These are just summaries of the lecture notes, an few etails are inclue. Most of what we inclue here is to

More information

Topic 2.3: The Geometry of Derivatives of Vector Functions

Topic 2.3: The Geometry of Derivatives of Vector Functions BSU Math 275 Notes Topic 2.3: The Geometry of Derivatives of Vector Functions Textbook Sections: 13.2 From the Toolbox (what you nee from previous classes): Be able to compute erivatives scalar-value functions

More information

Free rotation of a rigid body 1 D. E. Soper 2 University of Oregon Physics 611, Theoretical Mechanics 5 November 2012

Free rotation of a rigid body 1 D. E. Soper 2 University of Oregon Physics 611, Theoretical Mechanics 5 November 2012 Free rotation of a rigi boy 1 D. E. Soper 2 University of Oregon Physics 611, Theoretical Mechanics 5 November 2012 1 Introuction In this section, we escribe the motion of a rigi boy that is free to rotate

More information

Calculus in the AP Physics C Course The Derivative

Calculus in the AP Physics C Course The Derivative Limits an Derivatives Calculus in the AP Physics C Course The Derivative In physics, the ieas of the rate change of a quantity (along with the slope of a tangent line) an the area uner a curve are essential.

More information

12.11 Laplace s Equation in Cylindrical and

12.11 Laplace s Equation in Cylindrical and SEC. 2. Laplace s Equation in Cylinrical an Spherical Coorinates. Potential 593 2. Laplace s Equation in Cylinrical an Spherical Coorinates. Potential One of the most important PDEs in physics an engineering

More information

1. General Vector Spaces

1. General Vector Spaces 1.1. Vector space axioms. 1. General Vector Spaces Definition 1.1. Let V be a nonempty set of objects on which the operations of addition and scalar multiplication are defined. By addition we mean a rule

More information

Differentiation Rules Derivatives of Polynomials and Exponential Functions

Differentiation Rules Derivatives of Polynomials and Exponential Functions Derivatives of Polynomials an Exponential Functions Differentiation Rules Derivatives of Polynomials an Exponential Functions Let s start with the simplest of all functions, the constant function f(x)

More information

Linear Algebra Highlights

Linear Algebra Highlights Linear Algebra Highlights Chapter 1 A linear equation in n variables is of the form a 1 x 1 + a 2 x 2 + + a n x n. We can have m equations in n variables, a system of linear equations, which we want to

More information

Math 32A Review Sheet

Math 32A Review Sheet Review Sheet Tau Beta Pi - Boelter 6266 Contents 1 Parametric Equation 2 1.1 Line.................................................. 2 1.2 Circle................................................. 2 1.3 Ellipse.................................................

More information

Differentiation ( , 9.5)

Differentiation ( , 9.5) Chapter 2 Differentiation (8.1 8.3, 9.5) 2.1 Rate of Change (8.2.1 5) Recall that the equation of a straight line can be written as y = mx + c, where m is the slope or graient of the line, an c is the

More information

Calculus and optimization

Calculus and optimization Calculus an optimization These notes essentially correspon to mathematical appenix 2 in the text. 1 Functions of a single variable Now that we have e ne functions we turn our attention to calculus. A function

More information

Computing Exact Confidence Coefficients of Simultaneous Confidence Intervals for Multinomial Proportions and their Functions

Computing Exact Confidence Coefficients of Simultaneous Confidence Intervals for Multinomial Proportions and their Functions Working Paper 2013:5 Department of Statistics Computing Exact Confience Coefficients of Simultaneous Confience Intervals for Multinomial Proportions an their Functions Shaobo Jin Working Paper 2013:5

More information

NOTES ON EULER-BOOLE SUMMATION (1) f (l 1) (n) f (l 1) (m) + ( 1)k 1 k! B k (y) f (k) (y) dy,

NOTES ON EULER-BOOLE SUMMATION (1) f (l 1) (n) f (l 1) (m) + ( 1)k 1 k! B k (y) f (k) (y) dy, NOTES ON EULER-BOOLE SUMMATION JONATHAN M BORWEIN, NEIL J CALKIN, AND DANTE MANNA Abstract We stuy a connection between Euler-MacLaurin Summation an Boole Summation suggeste in an AMM note from 196, which

More information

Systems & Control Letters

Systems & Control Letters Systems & ontrol Letters ( ) ontents lists available at ScienceDirect Systems & ontrol Letters journal homepage: www.elsevier.com/locate/sysconle A converse to the eterministic separation principle Jochen

More information

cosh x sinh x So writing t = tan(x/2) we have 6.4 Integration using tan(x/2) 2t 1 + t 2 cos x = 1 t2 sin x =

cosh x sinh x So writing t = tan(x/2) we have 6.4 Integration using tan(x/2) 2t 1 + t 2 cos x = 1 t2 sin x = 6.4 Integration using tan/ We will revisit the ouble angle ientities: sin = sin/ cos/ = tan/ sec / = tan/ + tan / cos = cos / sin / tan = = tan / sec / tan/ tan /. = tan / + tan / So writing t = tan/ we

More information

Permanent vs. Determinant

Permanent vs. Determinant Permanent vs. Determinant Frank Ban Introuction A major problem in theoretical computer science is the Permanent vs. Determinant problem. It asks: given an n by n matrix of ineterminates A = (a i,j ) an

More information

Chapter 2 Lagrangian Modeling

Chapter 2 Lagrangian Modeling Chapter 2 Lagrangian Moeling The basic laws of physics are use to moel every system whether it is electrical, mechanical, hyraulic, or any other energy omain. In mechanics, Newton s laws of motion provie

More information

Introduction to the Vlasov-Poisson system

Introduction to the Vlasov-Poisson system Introuction to the Vlasov-Poisson system Simone Calogero 1 The Vlasov equation Consier a particle with mass m > 0. Let x(t) R 3 enote the position of the particle at time t R an v(t) = ẋ(t) = x(t)/t its

More information

Vectors in two dimensions

Vectors in two dimensions Vectors in two imensions Until now, we have been working in one imension only The main reason for this is to become familiar with the main physical ieas like Newton s secon law, without the aitional complication

More information

Linear and quadratic approximation

Linear and quadratic approximation Linear an quaratic approximation November 11, 2013 Definition: Suppose f is a function that is ifferentiable on an interval I containing the point a. The linear approximation to f at a is the linear function

More information

Physics 5153 Classical Mechanics. The Virial Theorem and The Poisson Bracket-1

Physics 5153 Classical Mechanics. The Virial Theorem and The Poisson Bracket-1 Physics 5153 Classical Mechanics The Virial Theorem an The Poisson Bracket 1 Introuction In this lecture we will consier two applications of the Hamiltonian. The first, the Virial Theorem, applies to systems

More information

Solutions to Math 41 Second Exam November 4, 2010

Solutions to Math 41 Second Exam November 4, 2010 Solutions to Math 41 Secon Exam November 4, 2010 1. (13 points) Differentiate, using the metho of your choice. (a) p(t) = ln(sec t + tan t) + log 2 (2 + t) (4 points) Using the rule for the erivative of

More information

05 The Continuum Limit and the Wave Equation

05 The Continuum Limit and the Wave Equation Utah State University DigitalCommons@USU Founations of Wave Phenomena Physics, Department of 1-1-2004 05 The Continuum Limit an the Wave Equation Charles G. Torre Department of Physics, Utah State University,

More information

A FURTHER REFINEMENT OF MORDELL S BOUND ON EXPONENTIAL SUMS

A FURTHER REFINEMENT OF MORDELL S BOUND ON EXPONENTIAL SUMS A FURTHER REFINEMENT OF MORDELL S BOUND ON EXPONENTIAL SUMS TODD COCHRANE, JEREMY COFFELT, AND CHRISTOPHER PINNER 1. Introuction For a prime p, integer Laurent polynomial (1.1) f(x) = a 1 x k 1 + + a r

More information

Characterizing Real-Valued Multivariate Complex Polynomials and Their Symmetric Tensor Representations

Characterizing Real-Valued Multivariate Complex Polynomials and Their Symmetric Tensor Representations Characterizing Real-Value Multivariate Complex Polynomials an Their Symmetric Tensor Representations Bo JIANG Zhening LI Shuzhong ZHANG December 31, 2014 Abstract In this paper we stuy multivariate polynomial

More information

The Press-Schechter mass function

The Press-Schechter mass function The Press-Schechter mass function To state the obvious: It is important to relate our theories to what we can observe. We have looke at linear perturbation theory, an we have consiere a simple moel for

More information

Section 2.7 Derivatives of powers of functions

Section 2.7 Derivatives of powers of functions Section 2.7 Derivatives of powers of functions (3/19/08) Overview: In this section we iscuss the Chain Rule formula for the erivatives of composite functions that are forme by taking powers of other functions.

More information

Convergence of Random Walks

Convergence of Random Walks Chapter 16 Convergence of Ranom Walks This lecture examines the convergence of ranom walks to the Wiener process. This is very important both physically an statistically, an illustrates the utility of

More information

Lecture Introduction. 2 Examples of Measure Concentration. 3 The Johnson-Lindenstrauss Lemma. CS-621 Theory Gems November 28, 2012

Lecture Introduction. 2 Examples of Measure Concentration. 3 The Johnson-Lindenstrauss Lemma. CS-621 Theory Gems November 28, 2012 CS-6 Theory Gems November 8, 0 Lecture Lecturer: Alesaner Mąry Scribes: Alhussein Fawzi, Dorina Thanou Introuction Toay, we will briefly iscuss an important technique in probability theory measure concentration

More information

MAT 2037 LINEAR ALGEBRA I web:

MAT 2037 LINEAR ALGEBRA I web: MAT 237 LINEAR ALGEBRA I 2625 Dokuz Eylül University, Faculty of Science, Department of Mathematics web: Instructor: Engin Mermut http://kisideuedutr/enginmermut/ HOMEWORK 2 MATRIX ALGEBRA Textbook: Linear

More information