Real Symmetric Matrices

Total Page:16

File Type:pdf, Size:1020Kb

Real Symmetric Matrices Chapter 2 Real Symmetric Matrices 2.1 Special properties of real symmetric matrices A matrixA M n(C) (orM n(R)) is diagonalizable if it is similar to a diagonal matrix. If this ∈ happens, it means that there is a basis ofC n with respect to which the linear transformation ofC n defined by left multiplication byA has a diagonal matrix. Every element of such a basis is simply multiplied by a scalar when it is multiplied byA, which means exactly that the basis consists of eigenvectors ofA. n Lemma 2.1.1. A matrixA M n(C) is diagonalizable if and only ifC possesses a basis consisting of ∈ eigenvectors ofA. 1 1 Not all matrices are diagonalizable. For exampleA= is not. To see this note that 1 0 1 � � (occurring twice) is the only eigenvalue ofA, but that all eigenvectors ofA are scalar multiples of 1 2 2 0 , soC (orR ) does not contain a basis consisting of eigenvectors ofA, andA is not similar to a diagonal matrix. � � We note that a matrix can fail to be diagonalizable only if it has repeated eigenvalues, as the following lemma shows. Lemma 2.1.2. LetA M n(R) and suppose thatA has distinct eigenvaluesλ 1,...,λ n inC. ThenA is ∈ diagonalizable. Proof. Letv i be an eigenvector ofA corresponding toλ i. We will show thatS={v 1,...,v n} is a linearly independent set. Sincev 1 is not the zero vector, we know that{v 1} is linearly independent. IfS is linearly dependent, letk be the least for which{v 1,...,v k} is linearly dependent. This means that{v 1,...,v k−1} is a linearly independent set and v =a v + +a v k 1 1 ··· k−1 k−1 for somea i C, not all zero. Multiplying this equation on the left separately byA and byλk ∈ gives λkvk =a 1λ1v1 +a 2λ2v2 +a k−1λk−1vk−1 a1λkv1 +a 2λkv2 +a k−1λkvk−1 = 0=a (λ −λ )v +a (λ −λ ) + +a (λ −λ )v . ⇒ 1 1 k 1 2 2 k ··· k k−1 k k−1 Since the complex numbersλ i −λ k are non-zero fori= 1, . ,k− 1 and at least one of thesea i is non-zero, the above is an expression for the zero vector as a nontrivial linear combination of v1,...,v k−1, contrary to the choice ofk. We conclude thatS is linearly independent and hence that it is a basis ofC n. 13 Definition 2.1.3. A matrixA M n(R) is symmetric if it is equal to its transpose, i.e. ifA ij =A ji for ∈ alli andj. Symmetric matrices arise naturally in various contexts, including as adjacency matrices of undirected graphs. Fortunately they have lots of nice properties. To explore some of these we need a slightly more general concept, that of a complex Hermitian matrix. Definition 2.1.4. LetA M n(C). The Hermitian transpose, or conjugate transpose ofA is the ∈ matrixA ∗ obtained by taking the transpose ofA and then taking the complex conjugate of each entry. The matrixA is said to be Hermitian ifA=A ∗. Notes 2+i4−i 2−i3 1. Example: IfA= , thenA ∗ = 3 3−i 4+i3+i � � � � 2. The Hermitian transpose ofA is equal to its (ordinary) transpose if and only ifA M n(R). ∈ In some contexts the Hermitian transpose is the appropriate analogue inC of the concept of transpose of a real matrix. 3. IfA M n(C), then the trace of the productA ∗A is the sum of all the entries ofA, each ∈ multiplied by its own complex conjugate (check this). This is a non-negative real number T and it is zero only ifA= 0. In particular, ifA M n(R), then trace(A A) is the sum of the ∈ squares of all the entries ofA. 4. Suppose thatA andB are two matrices for which the productAB exists. Then(AB) T = T T B A and(AB) ∗ =B ∗A∗ (it is routine but worthwile to prove these statements). In particu- lar, ifA is any matrix at all, then T T T T T T (A A) =A (A ) =A A, and(A ∗A)∗ =A ∗(A∗)∗ =A ∗A, T T soA A andA ∗A are respectively symmetric and Hermitian (so areAA andAA ∗). The following theorem is the start of the story of what makes real symmetric matrices so special. Theorem 2.1.5. The eigenvalues of a real symmetric matrix are all real. Proof. We will prove the stronger statement that the eigenvalues of a complex Hermitian matrix are all real. LetA be a Hermitian matrix inM n(C) and letλ be an eigenvalue ofA with corre- n sponding eigenvectorv. Soλ C andv is a non-zero vector inC . Look at the productv ∗Av. ∈ This is a complex number. v∗Av=v ∗λv=λv ∗v. The expressionv ∗v is a positive real number, since it is the sum of the expressions ¯ivvi over all entriesv i ofv. We have not yet used the fact thatA ∗ =A. Now look at the Hermitian transpose of the matrix productv ∗Av. (v∗Av)∗ =v ∗A∗(v∗)∗ =v ∗Av. This is saying thatv ∗Av is a complex number that is equal to its own Hermitian transpose, i.e. equal to its own complex conjugate. This means exactly thatv ∗Av R. ∈ We also know thatv ∗Av=λv ∗v, and sincev ∗v is a non-zero real number, this means that λ R. ∈ So the eigenvalues of a real symmetric matrix are real numbers. This means in particular that the eigenvalues of the adjacency matrix of an undirected graph are real numbers, they can be arranged in order and we can ask questions about (for example) the greatest eigenvalue, the least eigenvalue, etc. 14 Another concept that is often mentioned in connection with real symmetric matrices is that T of positive definiteness. We mentioned above that ifA M m n(R), thenA A is a symmetric ∈ × matrix. However not every symmetric matrix has the formA T A, since for example the entries on the main diagonal ofA T A do not. It turns out that those symmetric matrices that have the form AT A (even for a non-squareA) can be characterized in another way. Definition 2.1.6. LetA be a symmetric matrix inM n(R). ThenA is called positive semidefinite (PSD) ifv T Av 0 for allv R n. In addition, ifv T Av is strictly positive wheneverv=0, thenA is called � ∈ � positive definite (PD). Notes 1. The identity matrixI n is the classical example of a positive definite symmetric matrix, since n T T for anyv R ,v Inv=v v=v v 0, andv v= 0 only ifv is the zero vector. ∈ · � · 1 2 2. The matrix is an example of a matrix that is not positive semidefinite, since 2 1 � � 1 2 −1 −1 1 =−2. 2 1 1 � � � � � � So positive (semi)definite is not the same thing as positive - a symmetric matrix can have all of its entries positive and still fail to be positive (semi)definite. 3. A symmetric matrix can have negative entries and still be positive definite, for example the 1−1 matrixA= is SPD (symmetric positive definite). To see this observe that for −1 2 � � real numbersa andb we have 1−1 a a b =a 2 − ab− ab+2b 2 = (a−b) 2 +b 2. −1 2 b � � � � � � Since(a−b) 2 +b 2 cannot be negative and is zero only if botha andb are equal to zero, the matrixA is positive definite. The importance of the concept of positive definiteness is not really obvious atfirst glance, it takes a little bit of discussion. We will defer this discussion for now, and mention two observations related to positive (semi)definiteness that have a connection to spectral graph theory. Lemma 2.1.7. The eigenvalues of a real symmetric positive semidefinite matrix are non-negative (positive if positive definite). Proof. Letλ be an eigenvalue of the real symmetric positive semidefinite matrixA, and letv R n ∈ be a corresponding eigenvector. Then T T T 0�v Av=v λv=λv v. Thusλ is nonnegative sincev T v is a positive real number. Lemma 2.1.8. LetB M n m(R) for some positive integersm andn. Then the symmetric matrix T ∈ × A=BB inM n(R) is positive semidefinite. Proof. Letu R n. Then ∈ uT Au=u T BBT u=(u T B)(BT u) = (BT u)T (BT u) = (BT u) (B T u) 0, · � soA is positive semidefinite. The next section will contain a more detailed discussion of positive (semi)definiteness, includ- ing the converses of the two statements above. First we digress to look at an application of what we know so far to spectral graph theory. 15 Definition 2.1.9. LetG be a graph. The line graph ofG, denoted byL(G), has a vertex for every edge ofG, and two vertices ofL(G) are adjacent if and only if their corresponding edges inG share an incident vertex. Example 2.1.10.K 4 (left) and its line graph (right). Choose an edge ofK 4. Since each of its incident vertices has degree 3, there are four other edges with which it shares a vertex. So the vertex that represents it inL(K 4) has degree 4. In general, if a graphG is regular of degreek, thenL(G) will be regular of degree 2k− 2. For any graphG, a vertex of degreed inG corresponds to a copy of the complete graphK d withinL(G). Not every graph can be a line graph.
Recommended publications
  • Math 221: LINEAR ALGEBRA
    Math 221: LINEAR ALGEBRA Chapter 8. Orthogonality §8-3. Positive Definite Matrices Le Chen1 Emory University, 2020 Fall (last updated on 11/10/2020) Creative Commons License (CC BY-NC-SA) 1 Slides are adapted from those by Karen Seyffarth from University of Calgary. Positive Definite Matrices Cholesky factorization – Square Root of a Matrix Positive Definite Matrices Definition An n × n matrix A is positive definite if it is symmetric and has positive eigenvalues, i.e., if λ is a eigenvalue of A, then λ > 0. Theorem If A is a positive definite matrix, then det(A) > 0 and A is invertible. Proof. Let λ1; λ2; : : : ; λn denote the (not necessarily distinct) eigenvalues of A. Since A is symmetric, A is orthogonally diagonalizable. In particular, A ∼ D, where D = diag(λ1; λ2; : : : ; λn). Similar matrices have the same determinant, so det(A) = det(D) = λ1λ2 ··· λn: Since A is positive definite, λi > 0 for all i, 1 ≤ i ≤ n; it follows that det(A) > 0, and therefore A is invertible. Theorem A symmetric matrix A is positive definite if and only if ~xTA~x > 0 for all n ~x 2 R , ~x 6= ~0. Proof. Since A is symmetric, there exists an orthogonal matrix P so that T P AP = diag(λ1; λ2; : : : ; λn) = D; where λ1; λ2; : : : ; λn are the (not necessarily distinct) eigenvalues of A. Let n T ~x 2 R , ~x 6= ~0, and define ~y = P ~x. Then ~xTA~x = ~xT(PDPT)~x = (~xTP)D(PT~x) = (PT~x)TD(PT~x) = ~yTD~y: T Writing ~y = y1 y2 ··· yn , 2 y1 3 6 y2 7 ~xTA~x = y y ··· y diag(λ ; λ ; : : : ; λ ) 6 7 1 2 n 1 2 n 6 .
    [Show full text]
  • Handout 9 More Matrix Properties; the Transpose
    Handout 9 More matrix properties; the transpose Square matrix properties These properties only apply to a square matrix, i.e. n £ n. ² The leading diagonal is the diagonal line consisting of the entries a11, a22, a33, . ann. ² A diagonal matrix has zeros everywhere except the leading diagonal. ² The identity matrix I has zeros o® the leading diagonal, and 1 for each entry on the diagonal. It is a special case of a diagonal matrix, and A I = I A = A for any n £ n matrix A. ² An upper triangular matrix has all its non-zero entries on or above the leading diagonal. ² A lower triangular matrix has all its non-zero entries on or below the leading diagonal. ² A symmetric matrix has the same entries below and above the diagonal: aij = aji for any values of i and j between 1 and n. ² An antisymmetric or skew-symmetric matrix has the opposite entries below and above the diagonal: aij = ¡aji for any values of i and j between 1 and n. This automatically means the digaonal entries must all be zero. Transpose To transpose a matrix, we reect it across the line given by the leading diagonal a11, a22 etc. In general the result is a di®erent shape to the original matrix: a11 a21 a11 a12 a13 > > A = A = 0 a12 a22 1 [A ]ij = A : µ a21 a22 a23 ¶ ji a13 a23 @ A > ² If A is m £ n then A is n £ m. > ² The transpose of a symmetric matrix is itself: A = A (recalling that only square matrices can be symmetric).
    [Show full text]
  • On the Eigenvalues of Euclidean Distance Matrices
    “main” — 2008/10/13 — 23:12 — page 237 — #1 Volume 27, N. 3, pp. 237–250, 2008 Copyright © 2008 SBMAC ISSN 0101-8205 www.scielo.br/cam On the eigenvalues of Euclidean distance matrices A.Y. ALFAKIH∗ Department of Mathematics and Statistics University of Windsor, Windsor, Ontario N9B 3P4, Canada E-mail: [email protected] Abstract. In this paper, the notion of equitable partitions (EP) is used to study the eigenvalues of Euclidean distance matrices (EDMs). In particular, EP is used to obtain the characteristic poly- nomials of regular EDMs and non-spherical centrally symmetric EDMs. The paper also presents methods for constructing cospectral EDMs and EDMs with exactly three distinct eigenvalues. Mathematical subject classification: 51K05, 15A18, 05C50. Key words: Euclidean distance matrices, eigenvalues, equitable partitions, characteristic poly- nomial. 1 Introduction ( ) An n ×n nonzero matrix D = di j is called a Euclidean distance matrix (EDM) 1, 2,..., n r if there exist points p p p in some Euclidean space < such that i j 2 , ,..., , di j = ||p − p || for all i j = 1 n where || || denotes the Euclidean norm. i , ,..., Let p , i ∈ N = {1 2 n}, be the set of points that generate an EDM π π ( , ,..., ) D. An m-partition of D is an ordered sequence = N1 N2 Nm of ,..., nonempty disjoint subsets of N whose union is N. The subsets N1 Nm are called the cells of the partition. The n-partition of D where each cell consists #760/08. Received: 07/IV/08. Accepted: 17/VI/08. ∗Research supported by the Natural Sciences and Engineering Research Council of Canada and MITACS.
    [Show full text]
  • Rotation Matrix - Wikipedia, the Free Encyclopedia Page 1 of 22
    Rotation matrix - Wikipedia, the free encyclopedia Page 1 of 22 Rotation matrix From Wikipedia, the free encyclopedia In linear algebra, a rotation matrix is a matrix that is used to perform a rotation in Euclidean space. For example the matrix rotates points in the xy -Cartesian plane counterclockwise through an angle θ about the origin of the Cartesian coordinate system. To perform the rotation, the position of each point must be represented by a column vector v, containing the coordinates of the point. A rotated vector is obtained by using the matrix multiplication Rv (see below for details). In two and three dimensions, rotation matrices are among the simplest algebraic descriptions of rotations, and are used extensively for computations in geometry, physics, and computer graphics. Though most applications involve rotations in two or three dimensions, rotation matrices can be defined for n-dimensional space. Rotation matrices are always square, with real entries. Algebraically, a rotation matrix in n-dimensions is a n × n special orthogonal matrix, i.e. an orthogonal matrix whose determinant is 1: . The set of all rotation matrices forms a group, known as the rotation group or the special orthogonal group. It is a subset of the orthogonal group, which includes reflections and consists of all orthogonal matrices with determinant 1 or -1, and of the special linear group, which includes all volume-preserving transformations and consists of matrices with determinant 1. Contents 1 Rotations in two dimensions 1.1 Non-standard orientation
    [Show full text]
  • Matrices and Matrix Operations with TI-Nspire™ CAS
    Matrices and Matrix Operations with TI-Nspire™ CAS Forest W. Arnold June 2020 Typeset in LATEX. Copyright © 2020 Forest W. Arnold This work is licensed under the Creative Commons Attribution-Noncommercial-Share Alike 4.0 International License. To view a copy of this license, visit http://creativecommons. org/licenses/by-nc-sa/4.0/legalcode/ or send a letter to Creative Commons, 171 Second Street, Suite 300, San Francisco, California, 94105, USA. You can use, print, duplicate, share this work as much as you want. You can base your own work on it and reuse parts if you keep the license the same. Trademarks TI-Nspire is a registered trademark of Texas Instruments, Inc. Attribution Most of the examples in this article are from A First Course in Linear Algebra an Open Text by Lyrix Learning, base textbook version 2017 - revision A, by K. Kuttler. The text is licensed under the Creative Commons License (CC BY) and is available for download at the link https://lyryx.com/first-course-linear-algebra/. 1 Introduction The article Systems of Equations with TI-Nspire™ CAS: Matrices and Gaussian Elim- ination described how to represent and solve systems of linear equations with matrices and elementary row operations. By defining arithmetic and algebraic operations with matrices, applications of matrices can be expanded to include more than simply solving linear systems. This article describes and demonstrates how to use TI-Nspire’s builtin matrix functions to • add and subtract matrices, • multiply matrices by scalars, • multiply matrices, • transpose matrices, • find matrix inverses, and • use matrix equations. The TI-Nspire examples in this article require the CAS version of TI-Nspire.
    [Show full text]
  • Notes on Symmetric Matrices 1 Symmetric Matrices
    CPSC 536N: Randomized Algorithms 2011-12 Term 2 Notes on Symmetric Matrices Prof. Nick Harvey University of British Columbia 1 Symmetric Matrices We review some basic results concerning symmetric matrices. All matrices that we discuss are over the real numbers. Let A be a real, symmetric matrix of size d × d and let I denote the d × d identity matrix. Perhaps the most important and useful property of symmetric matrices is that their eigenvalues behave very nicely. Definition 1 Let U be a d × d matrix. The matrix U is called an orthogonal matrix if U TU = I. This implies that UU T = I, by uniqueness of inverses. Fact 2 (Spectral Theorem). Let A be any d × d symmetric matrix. There exists an orthogonal matrix U and a (real) diagonal matrix D such that A = UDU T: This is called a spectral decomposition of A. Let ui be the ith column of U and let λi denote the ith diagonal entry of D. Then fu1; : : : ; udg is an orthonormal basis consisting of eigenvectors of A, and λi is the eigenvalue corresponding to ui. We can also write d X T A = λiuiui : (1) i=1 The eigenvalues λ are uniquely determined by A, up to reordering. Caution. The product of two symmetric matrices is usually not symmetric. 1.1 Positive semi-definite matrices Definition 3 Let A be any d × d symmetric matrix. The matrix A is called positive semi-definite if all of its eigenvalues are non-negative. This is denoted A 0, where here 0 denotes the zero matrix.
    [Show full text]
  • On the Uniqueness of Euclidean Distance Matrix Completions Abdo Y
    View metadata, citation and similar papers at core.ac.uk brought to you by CORE provided by Elsevier - Publisher Connector Linear Algebra and its Applications 370 (2003) 1–14 www.elsevier.com/locate/laa On the uniqueness of Euclidean distance matrix completions Abdo Y. Alfakih Bell Laboratories, Lucent Technologies, Room 3J-310, 101 Crawfords Corner Road, Holmdel, NJ 07733-3030, USA Received 28 December 2001; accepted 18 December 2002 Submitted by R.A. Brualdi Abstract The Euclidean distance matrix completion problem (EDMCP) is the problem of determin- ing whether or not a given partial matrix can be completed into a Euclidean distance matrix. In this paper, we present necessary and sufficient conditions for a given solution of the EDMCP to be unique. © 2003 Elsevier Inc. All rights reserved. AMS classification: 51K05; 15A48; 52A05; 52B35 Keywords: Matrix completion problems; Euclidean distance matrices; Semidefinite matrices; Convex sets; Singleton sets; Gale transform 1. Introduction All matrices considered in this paper are real. An n × n matrix D = (dij ) is said to be a Euclidean distance matrix (EDM) iff there exist points p1,p2,...,pn in some i j 2 Euclidean space such that dij =p − p for all i, j = 1,...,n. It immediately follows that if D is EDM then D is symmetric with positive entries and with zero diagonal. We say matrix A = (aij ) is symmetric partial if only some of its entries are specified and aji is specified and equal to aij whenever aij is specified. The unspecified entries of A are said to be free. Given an n × n symmetric partial matrix A,ann × n matrix D is said to be a EDM completion of A iff D is EDM and Email address: [email protected] (A.Y.
    [Show full text]
  • Rotations in 3-Space
    Rotations in 3-space A. Eremenko March 13, 2020 These facts of the combinations of rotations, and what they produce, are hard to grasp intuitively. It is rather strange, because we live in three dimensions, but it is hard for us to appreciate what happens if we turn this way and then that way. Perhaps, if we were fish or birds and had a real appreciation of what happens when we turn somersaults in space, we could more easily appreciate these things. Feynman’s lectures on physics, vol. 3, 6.5. O(3) pervades all the essential properties of the physical world. But we remain intellectually blind to this symmetry, even if we encounter it frequently and use it in everyday life, for instance when we experience or engender mechanical movements, such as walking. This is due in part to the non commutativity of O(3), which is difficult to grasp. M. Gromov, Notices AMS, 45, 846-847. Rotations in 3-space are more complicated than rotations in a plane. One reason for this is that rotations in 3-space in general do not commute. (Give an example!) We consider rotations with fixed center which we place at the origin. Then rotations are linear transformations of the space represented by orthogonal matrices with determinant 1. Orthogonality means that all distances and angles are preserved. The determinant of an orthogonal matrix is always 1 or -1. (Think why.) The 1 condition that determinant equals 1 means that orientation is preserved. An orthogonal transformation with determinant -1 will map a right shoe onto a left shoe; such orthogonal transformations are called sometimes improper rotations, we cannot actually perform them on real objects.
    [Show full text]
  • Exam 3 Review
    Exam 3 review The exam will cover the material through the singular value decomposition. Linear transformations and change of basis will be covered on the final. The main topics on this exam are: • Eigenvalues and eigenvectors du At • Differential equations dt = Au and exponentials e • Symmetric matrices A = AT: These always have real eigenvalues, and they always have “enough” eigenvectors. The eigenvector matrix Q can be an orthogonal matrix, with A = QLQT . • Positive definite matrices • Similar matrices B = M−1 AM. Matrices A and B have the same eigen­ values; powers of A will “look like” powers of B. • Singular value decomposition Sample problems 1. This is a question about a differential equation with a skew symmetric matrix. Suppose 2 0 −1 0 3 du = Au = 4 1 0 −1 5 u. dt 0 1 0 The general solution to this equation will look like l1t l2t l3t u(t) = c1e x1 + c2e x2 + cee x3. a) What are the eigenvalues of A? The matrix A is singular; the first and third rows are dependent, so one eigenvalue is l1 = 0. We might also notice that A is antisymmet­ ric (AT = −A) and realize that its eigenvalues will be imaginary. To find the other two eigenvalues, we’ll solve the equation jA − lIj = 0. � � � −l −1 0 � � � � 1 −l −1 � = −l3 − 2l = 0. � � � 0 1 −l � p p We conclude l2 = 2 i and l3 = − 2 i. 1 At this point we know that our solution will look like: p p 2 it − 2 it u(t) = c1x1 + c2e x2 + cee x3.
    [Show full text]
  • Spectral Properties of Sign Symmetric Matrices∗
    Electronic Journal of Linear Algebra ISSN 1081-3810 A publication of the International Linear Algebra Society Volume 13, pp. 90-110, March 2005 ELA www.math.technion.ac.il/iic/ela SPECTRAL PROPERTIES OF SIGN SYMMETRIC MATRICES∗ DANIEL HERSHKOWITZ† AND NATHAN KELLER‡ Abstract. Spectral properties of sign symmetric matrices are studied.A criterion for sign symmetry of shifted basic circulant permutation matrices is proven, and is then used to answer the question which complex numbers can serve as eigenvalues of sign symmetric 3 × 3matrices.The results are applied in the discussion of the eigenvalues of QM-matrices.In particular, it is shown that for every positive integer n there exists a QM-matrix A such that Ak is a sign symmetric P -matrix for all k ≤ n, but not all the eigenvalues of A are positive real numbers. Key words. Spectrum, Sign symmetric matrices, Circulant matrices, Basic circulant permuta- tion matrices, P -matrices, PM-matrices, Q-matrices, QM-matrices. AMS subject classifications. 15A18, 15A29. 1. Introduction. A square complex matrix A is called a Q-matrix [Q0-matrix] if the sums of principal minors of A of the same order are positive [nonnegative]. Equivalently, Q-matrices can be defined as matrices whose characteristic polynomials have coefficients with alternating signs. A square complex matrix is called a P -matrix [P0-matrix] if all its principal minors are positive [nonnegative]. A square complex matrix is said to be stable if its spectrum lies in the open right half plane. Let A be an n×n matrix. For subsets α and β of {1, ..., n} we denote by A(α|β)the submatrix of A with rows indexed by α and columns indexed by β.If|α| = |β| then we denote by A[α|β] the corresponding minor.
    [Show full text]
  • Definite Matrices
    John Nachbar September 2, 2014 Definite Matrices1 1 Basic Definitions. An N × N symmetric matrix A is positive definite iff for any v 6= 0, v0Av > 0. For example, if a b A = b c then the statement is that for any v = (v1; v2) 6= 0, 0 a b v1 v Av = [ v1 v2 ] b c v2 av1 + bv2 = [ v1 v2 ] bv1 + cv2 2 2 = av1 + 2bv1v2 + cv2 > 0 2 2 (The expression av1 +2bv1v2 +cv2 is called a quadratic form.) An N ×N symmetric matrix A is negative definite iff −A is positive definite. The definition of a positive semidefinite matrix relaxes > to ≥, and similarly for negative semi-definiteness. If N = 1 then A is just a number and a number is positive definite iff it is positive. For N > 1 the condition of being positive definite is somewhat subtle. For example, the matrix 1 3 A = 3 1 is not positive definite. If v = (1; −1) then v0Av = −4. Loosely, a matrix is positive definite iff (a) it has a diagonal that is positive and (b) off diagonal terms are not too large in absolute value relative to the terms on the diagonal. I won't formalize this assertion but it should be plausible given the example. The canonical positive definite matrix is the identity matrix, where all the off diagonal terms are zero. A useful fact is the following. If S is any M ×N matrix then A = S0S is positive semi-definite. To see this, note that S0S is symmetric N × N. To see that it is N positive semi-definite, note that for any v 2 R , v0Av = v0[S0S]v = (v0S0)(Sv) = (Sv)0(Sv) ≥ 0: 1cbna.
    [Show full text]
  • Matrices and Linear Algebra
    Chapter 2 Matrices and Linear Algebra 2.1 Basics Definition 2.1.1. A matrix is an m n array of scalars from a given field F . The individual values in the matrix× are called entries. Examples. 213 12 A = B = 124 34 − The size of the array is–written as m n,where × m n × number of rows number of columns Notation a11 a12 ... a1n a21 a22 ... a2n rows ←− A = a a ... a n1 n2 mn columns A := uppercase denotes a matrix a := lower case denotes an entry of a matrix a F. ∈ Special matrices 33 34 CHAPTER 2. MATRICES AND LINEAR ALGEBRA (1) If m = n, the matrix is called square.Inthiscasewehave (1a) A matrix A is said to be diagonal if aij =0 i = j. (1b) A diagonal matrix A may be denoted by diag(d1,d2,... ,dn) where aii = di aij =0 j = i. The diagonal matrix diag(1, 1,... ,1) is called the identity matrix and is usually denoted by 10... 0 01 In = . . .. 01 or simply I,whenn is assumed to be known. 0 = diag(0,... ,0) is called the zero matrix. (1c) A square matrix L is said to be lower triangular if ij =0 i<j. (1d) A square matrix U is said to be upper triangular if uij =0 i>j. (1e) A square matrix A is called symmetric if aij = aji. (1f) A square matrix A is called Hermitian if aij =¯aji (¯z := complex conjugate of z). (1g) Eij has a 1 in the (i, j) position and zeros in all other positions.
    [Show full text]