Matrix Analysis

Total Page:16

File Type:pdf, Size:1020Kb

Matrix Analysis Appendix A Matrix Analysis This appendix collects useful background from linear algebra and matrix analysis, such as vector and matrix norms, singular value decompositions, Gershgorin’s disk theorem, and matrix functions. Much more material can be found in various books on the subject including [47, 51, 231, 273, 280, 281, 475]. A.1 Vector and Matrix Norms We work with real or complex vector spaces X, usually X = Rn or X = Cn.We n usually write the vectors in C in boldface, x, while their entries are denoted xj , j ∈ [n],where[n]:={1,...,n}. The canonical unit vectors in Rn are denoted by e1,...,en. They have entries 1 if j = , (e ) = δ = j ,j 0 otherwise. Definition A.1. A nonnegative function ·: X → [0, ∞) is called a norm if (a) x =0if and only if x = 0 (definiteness). (b) λx = |λ|x for all scalars λ and all vectors x ∈ X (homogeneity). (c) x + y≤x + y for all vectors x, y ∈ X (triangle inequality). If only (b) and (c) hold, so that x =0does not necessarily imply x = 0,then· is called a seminorm. If (a) and (b) hold, but (c) is replaced by the weaker quasitriangle inequality x + y≤C(x + y) for some constant C ≥ 1,then·is called a quasinorm. The smallest constant C is called its quasinorm constant. S. Foucart and H. Rauhut, A Mathematical Introduction to Compressive Sensing, 515 Applied and Numerical Harmonic Analysis, DOI 10.1007/978-0-8176-4948-7, © Springer Science+Business Media New York 2013 516 A Matrix Analysis A space X endowed with a norm ·is called a normed space. Definition A.2. Let X be a set. A function d : X × X → [0, ∞) is called a metric if (a) d(x, y)=0if and only if x = y. (b) d(x, y)=d(y,x) for all x, y ∈ X. (c) d(x, z) ≤ d(x, y)+d(y,z) for all x, y, z ∈ X. If only (b) and (c) hold, then d is called a pseudometric. The set X endowed with a metric d is called a metric space. A norm ·on X induces a metric on X by d(x, y)=x − y. A seminorm induces a pseudometric in the same way. n n The p-norm (or simply p-norm) on R or C is defined for 1 ≤ p<∞ as n 1/p p xp := |xj | , (A.1) j=1 and for p = ∞ as x∞ := max |xj |. j∈[n] For 0 <p<1, the expression (A.1) only defines a quasinorm with quasinorm constant C =21/p−1. This is derived from the p-triangle inequality p ≤ p p x + y p x p + y p. − p Therefore, the p-quasinorm induces a metric via d(x, y)= x y p for 0 <p<1. We define a ball of radius t ≥ 0 around a point x in a metric space (X, d) by B(x,t)=Bd(x,t)={z ∈ X : d(x, z) ≤ t}. If the metric is induced by a norm ·on a vector space, then we also write B · (x,t)={z ∈ X : x − z≤t}. (A.2) If x = 0 and t =1,thenB = B · = B · (0, 1) is called unit ball. The canonical inner product on Cn is defined by n n x, y = xj yj , x, y ∈ C . j=1 A.1 Vector and Matrix Norms 517 Rn n ∈ Rn On ,itisgivenby x, y = j=1 xj yj, x, y .The2-norm is related to the canonical inner product by ' x2 = x, x. The Cauchy–Schwarz inequality states that n |x, y| ≤ x2y2 for all x, y ∈ C . More generally, for p, q ∈ [1, ∞] such that 1/p +1/q =1(with the convention that 1/∞ =0and 1/0=∞), Holder’s¨ inequality states that n |x, y| ≤ xpyq for all x, y ∈ C . Given 0 <p<q≤∞, applying the latter with x, y, p,andq replaced by | |p | |p − p ≤ p (q−p)/p [ x1 ,..., xn ] , [1,...,1] , q/p,andq/(q p) gives x p x qn , i.e., 1/p−1/q xp ≤ n xq. (A.3) We point out the important special cases √ √ x1 ≤ nx2 and x2 ≤ nx∞. If x has at most s nonzero entries, that is, x0 =card({ : x =0 }) ≤ s, then the 1/p−1/q above inequalities become xp ≤ s xq, and in particular, √ x1 ≤ sx2 ≤ sx∞. For 0 <p<q≤∞, we also have the reverse inequalities xq ≤xp, (A.4) and in particular, x∞ ≤x2 ≤x1. Indeed, the bound x∞ ≤xp is obvious, and for p<q<∞, n n n q | |q | |q−p| |p ≤ q−p | |p ≤ q−p p q x q = xj = xj xj x ∞ xj x p x p = x p. j=1 j=1 j=1 Both bounds (A.3)and(A.4) are sharp in general. Indeed, equality holds in (A.3) for vectors with constant absolute entries, while equality holds in (A.4) for scalar multiples of a canonical unit vector. n n Definition A.3. Let ·be a norm on R or C . Its dual norm ·∗ is defined by x∗ := sup |y, x|. y ≤1 518 A Matrix Analysis In the real case, the dual norm may equivalently be defined via x∗ =supy, x, y∈Rn, y ≤1 while in the complex case x∗ =supRe y, x. y∈Cn, y ≤1 The dual of the dual norm ·∗ is the norm ·itself. In particular, we have x =sup|x, y| =supRe x, y. (A.5) y ∗≤1 y ∗≤1 The dual of ·p is ·q with 1/p +1/q =1. In particular, ·2 is self-dual, i.e., x2 =sup|y, x|, (A.6) y 2≤1 while ·∞ is the dual norm of ·1 and vice versa. Given a subspace W of a vector space X,thequotient space X/W consists of the residue classes [x]:=x + W = {x + w, w ∈ W }, x ∈ X. The quotient map is the surjective linear map x → [x]=x + W ∈ X/W .The quotient norm on X/W is defined by [x]X/W := inf{v, v ∈ [x]=x + W }, [x] ∈ X/W. Let us now turn to norms of matrices (or more generally, linear mappings be- m×n tween normed spaces). The entries of A ∈ C are denoted Aj,k, j ∈ [m],k ∈ [n]. The columns of A are denoted ak,sothatA =[a1|···|an]. The transpose of m×n n×m A ∈ C is the matrix A ∈ C with entries (A )k,j = Aj,k. A matrix B ∈ Cn×n is called symmetric if B = B. The adjoint (or Hermitian transpose) m×n ∗ n×m ∗ n of A ∈ C is the matrix A ∈ C with entries (A )k,j = Aj,k.Forx ∈ C and y ∈ Cm,wehaveAx, y = x, A∗y. A matrix B ∈ Cn×n is called self- ∗ n adjoint (or Hermitian) if B = B. The identity matrix on C is denoted Id or Idn. AmatrixU ∈ Cn×n is called unitary if U∗U = UU∗ = Id. A self-adjoint matrix B ∈ Cn×n possesses an eigenvalue decomposition of the form B = U∗DU,where n×n U is a unitary matrix U ∈ C and D =diag[λ1,...,λn] is a diagonal matrix containing the real eigenvalues λ1,...,λn of B. Definition A.4. Let A : X → Y be a linear map between two normed spaces (X, ·) and (Y,||| · ||| ). The operator norm of A is defined as A.1 Vector and Matrix Norms 519 A := sup ||| Ax||| =sup||| Ax||| . (A.7) x ≤1 x =1 In particular, for a matrix A ∈ Cm×n and 1 ≤ p, q ≤∞, we define the matrix norm (or operator norm) between p and q as Ap→q := sup Axq =supAxq. (A.8) x p≤1 x p=1 For A : X → Y and x ∈ X, the definition implies that ||| Ax||| ≤ Ax.Itis an easy consequence of the definition that the norm of the product of two matrices A ∈ Cm×n and B ∈ Cn×k satisfies ABp→r ≤Aq→rBp→q, 1 ≤ p, q, r ≤∞. (A.9) We summarize formulas for the matrix norms Ap→q for some special choices of p and q. The lemma below also refers to the singular values of a matrix, which will be covered in the next section. Lemma A.5. Let A ∈ Cm×n. (a) We have ' ∗ A2→2 = λmax(A A)=σmax(A), ∗ ∗ where λmax(A A) is the largest eigenvalue of A A and σmax(A) the largest singular value of A. n×n In particular,if B ∈ C is self-adjoint, then B2→2 =maxj∈[n] |λj (B)|, where the λj (B) denote the eigenvalues of B. (b) For 1 ≤ p ≤∞, we have A1→p =maxk∈[n] akp. In particular, m A1→1 =max |Aj,k|, (A.10) k∈[n] j=1 A1→2 =maxak2. (A.11) k∈[n] (c) We have n A∞→∞ =max |Aj,k|. j∈[m] k=1 Proof. (a) Since A∗A ∈ Cn×n is self-adjoint, it can be diagonalized as A∗A = U∗DU with a unitary U and a diagonal D containing the eigenvalues ∗ n λ of A A on the diagonal. For x ∈ C with x2 =1, 2 ∗ ∗ Ax 2 = Ax, Ax = A Ax, x = U DUx, x = DUx, Ux . 520 A Matrix Analysis 2 ∗ 2 Since U is unitary, we have Ux 2 = Ux, Ux = x, U Ux = x 2 =1. Moreover, for an arbitrary vector z ∈ Cn, n n | |2 ≤ | |2 ∗ 2 Dz, z = λj zj max λj zj = λmax(A A) z 2. j∈[n] j=1 j=1 ' ∗ Combining these facts establishes the inequality A2→2 ≤ λmax(A A).
Recommended publications
  • Sobolev Spaces, Theory and Applications
    Sobolev spaces, theory and applications Piotr Haj lasz1 Introduction These are the notes that I prepared for the participants of the Summer School in Mathematics in Jyv¨askyl¨a,August, 1998. I thank Pekka Koskela for his kind invitation. This is the second summer course that I delivere in Finland. Last August I delivered a similar course entitled Sobolev spaces and calculus of variations in Helsinki. The subject was similar, so it was not posible to avoid overlapping. However, the overlapping is little. I estimate it as 25%. While preparing the notes I used partially the notes that I prepared for the previous course. Moreover Lectures 9 and 10 are based on the text of my joint work with Pekka Koskela [33]. The notes probably will not cover all the material presented during the course and at the some time not all the material written here will be presented during the School. This is however, not so bad: if some of the results presented on lectures will go beyond the notes, then there will be some reasons to listen the course and at the same time if some of the results will be explained in more details in notes, then it might be worth to look at them. The notes were prepared in hurry and so there are many bugs and they are not complete. Some of the sections and theorems are unfinished. At the end of the notes I enclosed some references together with comments. This section was also prepared in hurry and so probably many of the authors who contributed to the subject were not mentioned.
    [Show full text]
  • On Quasi Norm Attaining Operators Between Banach Spaces
    ON QUASI NORM ATTAINING OPERATORS BETWEEN BANACH SPACES GEUNSU CHOI, YUN SUNG CHOI, MINGU JUNG, AND MIGUEL MART´IN Abstract. We provide a characterization of the Radon-Nikod´ymproperty in terms of the denseness of bounded linear operators which attain their norm in a weak sense, which complement the one given by Bourgain and Huff in the 1970's. To this end, we introduce the following notion: an operator T : X ÝÑ Y between the Banach spaces X and Y is quasi norm attaining if there is a sequence pxnq of norm one elements in X such that pT xnq converges to some u P Y with }u}“}T }. Norm attaining operators in the usual (or strong) sense (i.e. operators for which there is a point in the unit ball where the norm of its image equals the norm of the operator) and also compact operators satisfy this definition. We prove that strong Radon-Nikod´ymoperators can be approximated by quasi norm attaining operators, a result which does not hold for norm attaining operators in the strong sense. This shows that this new notion of quasi norm attainment allows to characterize the Radon-Nikod´ymproperty in terms of denseness of quasi norm attaining operators for both domain and range spaces, completing thus a characterization by Bourgain and Huff in terms of norm attaining operators which is only valid for domain spaces and it is actually false for range spaces (due to a celebrated example by Gowers of 1990). A number of other related results are also included in the paper: we give some positive results on the denseness of norm attaining Lipschitz maps, norm attaining multilinear maps and norm attaining polynomials, characterize both finite dimensionality and reflexivity in terms of quasi norm attaining operators, discuss conditions to obtain that quasi norm attaining operators are actually norm attaining, study the relationship with the norm attainment of the adjoint operator and, finally, present some stability results.
    [Show full text]
  • On the Cone of a Finite Dimensional Compact Convex Set at a Point
    View metadata, citation and similar papers at core.ac.uk brought to you by CORE provided by Elsevier - Publisher Connector On the Cone of a Finite Dimensional Compact Convex Set at a Point C. H. Sung Department of Mathematics University of Califmia at San Diego La Joll41, California 92093 and Department of Mathematics San Diego State University San Diego, California 92182 and B. S. Tam* Department of Mathematics Tamkang University Taipei, Taiwan 25137, Republic of China Submitted by Robert C. Thompson ABSTRACT Four equivalent conditions for a convex cone in a Euclidean space to be an F,-set are given. Our result answers in the negative a recent open problem posed by Tam [5], characterizes the barrier cone of a convex set, and also provides an alternative proof for the known characterizations of the inner aperture of a convex set as given by BrBnsted [2] and Larman [3]. 1. INTRODUCTION Let V be a Euclidean space and C be a nonempty convex set in V. For each y E C, the cone of C at y, denoted by cone(y, C), is the cone *The work of this author was supported in part by the National Science Council of the Republic of China. LINEAR ALGEBRA AND ITS APPLICATIONS 90:47-55 (1987) 47 0 Elsevier Science Publishing Co., Inc., 1987 52 Vanderbilt Ave., New York, NY 10017 00243795/87/$3.50 48 C. H. SUNG AND B. S. TAM { a(r - Y) : o > 0 and x E C} (informally called a point’s cone). On 23 August 1983, at the International Congress of Mathematicians in Warsaw, in a short communication session, the second author presented the paper [5] and posed the following open question: Is it true that, given any cone K in V, there always exists a compact convex set C whose point’s cone at some given point y is equal to K? In view of the relation cone(y, C) = cone(0, C - { y }), the given point y may be taken to be the origin of the space.
    [Show full text]
  • Notes on Partial Differential Equations John K. Hunter
    Notes on Partial Differential Equations John K. Hunter Department of Mathematics, University of California at Davis Contents Chapter 1. Preliminaries 1 1.1. Euclidean space 1 1.2. Spaces of continuous functions 1 1.3. H¨olderspaces 2 1.4. Lp spaces 3 1.5. Compactness 6 1.6. Averages 7 1.7. Convolutions 7 1.8. Derivatives and multi-index notation 8 1.9. Mollifiers 10 1.10. Boundaries of open sets 12 1.11. Change of variables 16 1.12. Divergence theorem 16 Chapter 2. Laplace's equation 19 2.1. Mean value theorem 20 2.2. Derivative estimates and analyticity 23 2.3. Maximum principle 26 2.4. Harnack's inequality 31 2.5. Green's identities 32 2.6. Fundamental solution 33 2.7. The Newtonian potential 34 2.8. Singular integral operators 43 Chapter 3. Sobolev spaces 47 3.1. Weak derivatives 47 3.2. Examples 47 3.3. Distributions 50 3.4. Properties of weak derivatives 53 3.5. Sobolev spaces 56 3.6. Approximation of Sobolev functions 57 3.7. Sobolev embedding: p < n 57 3.8. Sobolev embedding: p > n 66 3.9. Boundary values of Sobolev functions 69 3.10. Compactness results 71 3.11. Sobolev functions on Ω ⊂ Rn 73 3.A. Lipschitz functions 75 3.B. Absolutely continuous functions 76 3.C. Functions of bounded variation 78 3.D. Borel measures on R 80 v vi CONTENTS 3.E. Radon measures on R 82 3.F. Lebesgue-Stieltjes measures 83 3.G. Integration 84 3.H. Summary 86 Chapter 4.
    [Show full text]
  • Boundedness in Linear Topological Spaces
    BOUNDEDNESS IN LINEAR TOPOLOGICAL SPACES BY S. SIMONS Introduction. Throughout this paper we use the symbol X for a (real or complex) linear space, and the symbol F to represent the basic field in question. We write R+ for the set of positive (i.e., ^ 0) real numbers. We use the term linear topological space with its usual meaning (not necessarily Tx), but we exclude the case where the space has the indiscrete topology (see [1, 3.3, pp. 123-127]). A linear topological space is said to be a locally bounded space if there is a bounded neighbourhood of 0—which comes to the same thing as saying that there is a neighbourhood U of 0 such that the sets {(1/n) U} (n = 1,2,—) form a base at 0. In §1 we give a necessary and sufficient condition, in terms of invariant pseudo- metrics, for a linear topological space to be locally bounded. In §2 we discuss the relationship of our results with other results known on the subject. In §3 we introduce two ways of classifying the locally bounded spaces into types in such a way that each type contains exactly one of the F spaces (0 < p ^ 1), and show that these two methods of classification turn out to be identical. Also in §3 we prove a metrization theorem for locally bounded spaces, which is related to the normal metrization theorem for uniform spaces, but which uses a different induction procedure. In §4 we introduce a large class of linear topological spaces which includes the locally convex spaces and the locally bounded spaces, and for which one of the more important results on boundedness in locally convex spaces is valid.
    [Show full text]
  • C H a P T E R § Methods Related to the Norm Al Equations
    ¡ ¢ £ ¤ ¥ ¦ § ¨ © © © © ¨ ©! "# $% &('*),+-)(./+-)0.21434576/),+98,:%;<)>=,'41/? @%3*)BAC:D8E+%=B891GF*),+H;I?H1KJ2.21K8L1GMNAPO45Q5R)S;S+T? =RU ?H1*)>./+EAVOKAPM ;<),5 ?H1G;P8W.XAVO4575R)S;S+Y? =Z8L1*)/[%\Z1*)]AB3*=,'Q;<)B=,'41/? @%3*)RAP8LU F*)BA(;S'*)Z)>@%3/? F*.4U ),1G;^U ?H1*)>./+ APOKAP;_),5a`Rbc`^dfeg`Rbih,jk=>.4U U )Blm;B'*)n1K84+o5R.EUp)B@%3*.K;q? 8L1KA>[r\0:D;_),1Ejp;B'/? A2.4s4s/+t8/.,=,' b ? A7.KFK84? l4)>lu?H1vs,+D.*=S;q? =>)m6/)>=>.43KA<)W;B'*)w=B8E)IxW=K? ),1G;W5R.K;S+Y? yn` `z? AW5Q3*=,'|{}84+-A_) =B8L1*l9? ;I? 891*)>lX;B'*.41Q`7[r~k8K{i)IF*),+NjL;B'*)71K8E+o5R.4U4)>@%3*.G;I? 891KA0.4s4s/+t8.*=,'w5R.BOw6/)Z.,l4)IM @%3*.K;_)7?H17A_8L5R)QAI? ;S3*.K;q? 8L1KA>[p1*l4)>)>lj9;B'*),+-)Q./+-)Q)SF*),1.Es4s4U ? =>.K;q? 8L1KA(?H1Q{R'/? =,'W? ;R? A s/+-)S:Y),+o+D)Blm;_8|;B'*)W3KAB3*.4Urc+HO4U 8,F|AS346KABs*.,=B)Q;_)>=,'41/? @%3*)BAB[&('/? A]=*'*.EsG;_),+}=B8*F*),+tA7? ;PM ),+-.K;q? F*)75R)S;S'K8ElAi{^'/? =,'Z./+-)R)K? ;B'*),+pl9?+D)B=S;BU OR84+k?H5Qs4U ? =K? ;BU O2+-),U .G;<)Bl7;_82;S'*)Q1K84+o5R.EU )>@%3*.G;I? 891KA>[ mWX(fQ - uK In order to solve the linear system 7 when is nonsymmetric, we can solve the equivalent system b b [¥K¦ ¡¢ £N¤ which is Symmetric Positive Definite. This system is known as the system of the normal equations associated with the least-squares problem, [ ­¦ £N¤ minimize §* R¨©7ª§*«9¬ Note that (8.1) is typically used to solve the least-squares problem (8.2) for over- ®°¯± ±²³® determined systems, i.e., when is a rectangular matrix of size , .
    [Show full text]
  • Surjective Isometries on Grassmann Spaces 11
    View metadata, citation and similar papers at core.ac.uk brought to you by CORE provided by Repository of the Academy's Library SURJECTIVE ISOMETRIES ON GRASSMANN SPACES FERNANDA BOTELHO, JAMES JAMISON, AND LAJOS MOLNAR´ Abstract. Let H be a complex Hilbert space, n a given positive integer and let Pn(H) be the set of all projections on H with rank n. Under the condition dim H ≥ 4n, we describe the surjective isometries of Pn(H) with respect to the gap metric (the metric induced by the operator norm). 1. Introduction The study of isometries of function spaces or operator algebras is an important research area in functional analysis with history dating back to the 1930's. The most classical results in the area are the Banach-Stone theorem describing the surjective linear isometries between Banach spaces of complex- valued continuous functions on compact Hausdorff spaces and its noncommutative extension for general C∗-algebras due to Kadison. This has the surprising and remarkable consequence that the surjective linear isometries between C∗-algebras are closely related to algebra isomorphisms. More precisely, every such surjective linear isometry is a Jordan *-isomorphism followed by multiplication by a fixed unitary element. We point out that in the aforementioned fundamental results the underlying structures are algebras and the isometries are assumed to be linear. However, descriptions of isometries of non-linear structures also play important roles in several areas. We only mention one example which is closely related with the subject matter of this paper. This is the famous Wigner's theorem that describes the structure of quantum mechanical symmetry transformations and plays a fundamental role in the probabilistic aspects of quantum theory.
    [Show full text]
  • POLARS and DUAL CONES 1. Convex Sets
    POLARS AND DUAL CONES VERA ROSHCHINA Abstract. The goal of this note is to remind the basic definitions of convex sets and their polars. For more details see the classic references [1, 2] and [3] for polytopes. 1. Convex sets and convex hulls A convex set has no indentations, i.e. it contains all line segments connecting points of this set. Definition 1 (Convex set). A set C ⊆ Rn is called convex if for any x; y 2 C the point λx+(1−λ)y also belongs to C for any λ 2 [0; 1]. The sets shown in Fig. 1 are convex: the first set has a smooth boundary, the second set is a Figure 1. Convex sets convex polygon. Singletons and lines are also convex sets, and linear subspaces are convex. Some nonconvex sets are shown in Fig. 2. Figure 2. Nonconvex sets A line segment connecting two points x; y 2 Rn is denoted by [x; y], so we have [x; y] = f(1 − α)x + αy; α 2 [0; 1]g: Likewise, we can consider open line segments (x; y) = f(1 − α)x + αy; α 2 (0; 1)g: and half open segments such as [x; y) and (x; y]. Clearly any line segment is a convex set. The notion of a line segment connecting two points can be generalised to an arbitrary finite set n n by means of a convex combination. Given a finite set fx1; x2; : : : ; xpg ⊂ R , a point x 2 R is the convex combination of x1; x2; : : : ; xp if it can be represented as p p X X x = αixi; αi ≥ 0 8i = 1; : : : ; p; αi = 1: i=1 i=1 Given an arbitrary set S ⊆ Rn, we can consider all possible finite convex combinations of points from this set.
    [Show full text]
  • Locally Solid Riesz Spaces with Applications to Economics / Charalambos D
    http://dx.doi.org/10.1090/surv/105 alambos D. Alipr Lie University \ Burkinshaw na University-Purdue EDITORIAL COMMITTEE Jerry L. Bona Michael P. Loss Peter S. Landweber, Chair Tudor Stefan Ratiu J. T. Stafford 2000 Mathematics Subject Classification. Primary 46A40, 46B40, 47B60, 47B65, 91B50; Secondary 28A33. Selected excerpts in this Second Edition are reprinted with the permissions of Cambridge University Press, the Canadian Mathematical Bulletin, Elsevier Science/Academic Press, and the Illinois Journal of Mathematics. For additional information and updates on this book, visit www.ams.org/bookpages/surv-105 Library of Congress Cataloging-in-Publication Data Aliprantis, Charalambos D. Locally solid Riesz spaces with applications to economics / Charalambos D. Aliprantis, Owen Burkinshaw.—2nd ed. p. cm. — (Mathematical surveys and monographs, ISSN 0076-5376 ; v. 105) Rev. ed. of: Locally solid Riesz spaces. 1978. Includes bibliographical references and index. ISBN 0-8218-3408-8 (alk. paper) 1. Riesz spaces. 2. Economics, Mathematical. I. Burkinshaw, Owen. II. Aliprantis, Char­ alambos D. III. Locally solid Riesz spaces. IV. Title. V. Mathematical surveys and mono­ graphs ; no. 105. QA322 .A39 2003 bib'.73—dc22 2003057948 Copying and reprinting. Individual readers of this publication, and nonprofit libraries acting for them, are permitted to make fair use of the material, such as to copy a chapter for use in teaching or research. Permission is granted to quote brief passages from this publication in reviews, provided the customary acknowledgment of the source is given. Republication, systematic copying, or multiple reproduction of any material in this publication is permitted only under license from the American Mathematical Society.
    [Show full text]
  • On the Ekeland Variational Principle with Applications and Detours
    Lectures on The Ekeland Variational Principle with Applications and Detours By D. G. De Figueiredo Tata Institute of Fundamental Research, Bombay 1989 Author D. G. De Figueiredo Departmento de Mathematica Universidade de Brasilia 70.910 – Brasilia-DF BRAZIL c Tata Institute of Fundamental Research, 1989 ISBN 3-540- 51179-2-Springer-Verlag, Berlin, Heidelberg. New York. Tokyo ISBN 0-387- 51179-2-Springer-Verlag, New York. Heidelberg. Berlin. Tokyo No part of this book may be reproduced in any form by print, microfilm or any other means with- out written permission from the Tata Institute of Fundamental Research, Colaba, Bombay 400 005 Printed by INSDOC Regional Centre, Indian Institute of Science Campus, Bangalore 560012 and published by H. Goetze, Springer-Verlag, Heidelberg, West Germany PRINTED IN INDIA Preface Since its appearance in 1972 the variational principle of Ekeland has found many applications in different fields in Analysis. The best refer- ences for those are by Ekeland himself: his survey article [23] and his book with J.-P. Aubin [2]. Not all material presented here appears in those places. Some are scattered around and there lies my motivation in writing these notes. Since they are intended to students I included a lot of related material. Those are the detours. A chapter on Nemyt- skii mappings may sound strange. However I believe it is useful, since their properties so often used are seldom proved. We always say to the students: go and look in Krasnoselskii or Vainberg! I think some of the proofs presented here are more straightforward. There are two chapters on applications to PDE.
    [Show full text]
  • Approximation Boundedness Surjectivity
    APPROXIMATION BOUNDEDNESS SURJECTIVITY Olav Kristian Nygaard Dr. scient. thesis, University of Bergen, 2001 Approximation, Boundedness, Surjectivity Olav Kr. Nygaard, 2001 ISBN 82-92-160-08-6 Contents 1Theframework 9 1.1 Separability, bases and the approximation property ....... 13 1.2Thecompletenessassumption................... 16 1.3Theoryofclosed,convexsets................... 19 2 Factorization of weakly compact operators and the approximation property 25 2.1Introduction............................. 25 2.2 Criteria of the approximation property in terms of the Davis- Figiel-Johnson-Pe'lczy´nskifactorization.............. 27 2.3Uniformisometricfactorization.................. 33 2.4 The approximation property and ideals of finite rank operators 36 2.5 The compact approximation property and ideals of compact operators.............................. 39 2.6 From approximation properties to metric approximation prop- erties................................. 41 3 Boundedness and surjectivity 49 3.1Introduction............................. 49 3.2Somemorepreliminaries...................... 52 3.3 The boundedness property in normed spaces . ....... 57 3.4ThesurjectivitypropertyinBanachspaces........... 59 3.5 The Seever property and the Nikod´ymproperty......... 63 3.6 Some results on thickness in L(X, Y )∗ .............. 63 3.7Somequestionsandremarks.................... 65 4 Slices in the unit ball of a uniform algebra 69 4.1Introduction............................. 69 4.2Thesliceshavediameter2..................... 70 4.3Someremarks...........................
    [Show full text]
  • The Column and Row Hilbert Operator Spaces
    The Column and Row Hilbert Operator Spaces Roy M. Araiza Department of Mathematics Purdue University Abstract Given a Hilbert space H we present the construction and some properties of the column and row Hilbert operator spaces Hc and Hr, respectively. The main proof of the survey is showing that CB(Hc; Kc) is completely isometric to B(H ; K ); in other words, the completely bounded maps be- tween the corresponding column Hilbert operator spaces is completely isometric to the bounded operators between the Hilbert spaces. A similar theorem for the row Hilbert operator spaces follows via duality of the operator spaces. In particular there exists a natural duality between the column and row Hilbert operator spaces which we also show. The presentation and proofs are due to Effros and Ruan [1]. 1 The Column Hilbert Operator Space Given a Hilbert space H , we define the column isometry C : H −! B(C; H ) given by ξ 7! C(ξ)α := αξ; α 2 C: Then given any n 2 N; we define the nth-matrix norm on Mn(H ); by (n) kξkc;n = C (ξ) ; ξ 2 Mn(H ): These are indeed operator space matrix norms by Ruan's Representation theorem and thus we define the column Hilbert operator space as n o Hc = H ; k·kc;n : n2N It follows that given ξ 2 Mn(H ) we have that the adjoint operator of C(ξ) is given by ∗ C(ξ) : H −! C; ζ 7! (ζj ξ) : Suppose C(ξ)∗(ζ) = d; c 2 C: Then we see that cd = (cj C(ξ)∗(ζ)) = (cξj ζ) = c(ζj ξ) = (cj (ζj ξ)) : We are also able to compute the matrix norms on rectangular matrices.
    [Show full text]