Lecture 2 — Convexity

Total Page:16

File Type:pdf, Size:1020Kb

Lecture 2 — Convexity TMA947 / MMG621 – Nonlinear optimisation Lecture 2 TMA947 / MMG621 — Nonlinear optimisation Lecture 2 — Convexity Emil Gustavsson October 28, 2013 Convex sets We begin by defining the notion of a convex set. Definition (convex set). The set S ⊆ Rn is convex if x1, x2 ∈ S ⇒ λx1 + (1 − λ)x2 ∈ S. λ ∈ (0, 1) A set is thus convex if all convex combination of any two points in the set lies in the set, see Figure 1. x2 λx1 + (1 − λ)x2 S x1 Figure 1: A convex set Examples: – The empty set is a convex set. – The set {x ∈ Rn |kxk≤ a} is convex for any a ∈ R. – The set {x ∈ Rn |kxk = a} is non-convex for any a> 0. – The set {0, 1, 2, 3} is non-convex. Rn Proposition. Let Sk ⊆ , k ∈ K be a collection of convex sets. Then the intersection k∈K Sk is also a convex set. T Proof. See Proposition 3.3. in the book. 1 TMA947 / MMG621 – Nonlinear optimisation Lecture 2 We define the affine hull of a finite set V = {v1, v2,..., vk} as k 1 k aff V := λ1v + ··· + λkv λ1,...,λk ∈ R, λi =1 ( i ) =1 X We define the convex hull of a finite set V = {v1, v2,..., vk} as k 1 k conv V := λ1v + ··· + λkv λ1,...,λk ≥ 0, λi =1 ( i ) =1 X The sets are defined by all possible affine (convex) combinations of the k points. v2 v2 v2 v1 v1 v1 V aff V conv V 1 2 Figure 2: The set V = {v , v }, the affine hull of V , and the convex hull of V . In general, we can define the convex hull of a set S as a) the unique minimal convex set containing S, b) the intersection of all convex sets containing S, or c) the set of all convex combinations of points in S. Any point x ∈ conv S, where S ⊆ Rn can thus be expressed as a convex combination of points in S. But how many points are required? The answer is, according to the following theorem, n +1 points. Theorem (Caratheodory’s theorem). Let x ∈ conv S, where S ⊆ Rn. Then x can be expressed as a convex combination of n +1 or fewer points of S. Proof. See Theorem 3.11. in the book. We now define the notion of a polytope. Definition (polytope). A set P is a polytope if it is the convex hull of finitely many points in Rn. A cube and a tetrahedron are examples of polytopes in R3. In Figure 3, a polytope in R2 generated by seven points is illustrated. 2 TMA947 / MMG621 – Nonlinear optimisation Lecture 2 v2 v6 v5 v3 v1 v7 v4 Figure 3: A polytope generated by seven point. The red dots are the extreme points Definition (extreme point). A point v of a convex set P is an extreme point if whenever v = λx1 + (1 − λ)x2 x1, x2 ∈ P =⇒ v = x1 = x2. λ ∈ (0, 1) An extreme point of P is thus a point in P that can not be represented as a convex combination of two other points, see Figure 3 for an example. We can now formulate the following intuitive theorem. Theorem. Let P be the polytope conv V , where V = {v1,..., vk}⊂ Rn. Then P is equal to the convex hull of its extreme points. The theorem basically says that the interesting points in a polytope are the extreme points. By combining the two last theorems, we can deduce that any point in a polytope P can be described as a convex combination of at most n +1 extreme points of P . This is often denoted as the inner representation of P . We now try to describe a polytope as linear inequalities instead of extreme points (exterior representation). Definition (polyhedron). A set P is a polyhedron if there exists a matrix A ∈ Rm×n and a vector b ∈ Rm such that P = {x ∈ Rn | Ax ≤ b}. – Ax ≤ b ⇐⇒ aix ≤ bi, i =1,...,m. (ai row i of A) n – {x ∈ R | aix ≤ bi}, i =1,...,m are half-spaces, so – P is the intersection of m half-spaces. 1 2 6 – Figure 4 shows the bounded polyhedron defined by A = −2 1 and b = −2 0 −1 −1 −2 1 −2 – Figure 5 shows the undounded polyhedron defined by A = and b = . 0 −1 −1 To make the distinction between a polytope and a polyhedron clearer, we have that 3 TMA947 / MMG621 – Nonlinear optimisation Lecture 2 x1 2x1 − x2 =2 x1 +2x2 =6 3 2 P 1 x2 =1 x2 1 2 3 4 5 Figure 4: A bounded polyhedron described by three linear inequalities. x1 2x1 − x2 =2 3 2 P 1 x2 =1 x2 1 2 3 4 5 Figure 5: An unbounded polyhedron described by two linear inequalities. – A polytope = The convex hull of finitely many points. – A polyhedron = The intersection of finitely many half-spaces. We can now define the extreme points of a polyhedron algebraically Theorem. Let x¯ ∈ P = {x ∈ Rn | Ax ≤ b}, where rank A = n and b ∈ Rm. Further, let A¯ x¯ = b¯ be the equality subsystem of Ax ≤ b. Then x¯ is an extreme point of P if and only if rank A¯ = n Proof. See Theorem 3.21 in the book. Note that the equality subsystem is obtained if one strikes out all rows i with aix¯ <bi, and require equality for the rest of the rows. That the equality subsystem has rank n basically means that there should be at least n linearly independent half-spaces going through the point in order for it to be an extreme point. In Figure 6, two half-spaces goes through the point x¯. Hence, it is an extreme point. In Figure 7, however, only one half-space goes through x¯, meaning that it is not an extreme point. How many extreme points can there exist in a polyhedron P = {x ∈ Rn | Ax ≤ b}? How many m ways can we choose n linearly independent rows from the m existing rows? At most . n Definition (cone). A set C ⊆ Rn is a cone if λx ∈ C whenever x ∈ C and λ> 0. 4 TMA947 / MMG621 – Nonlinear optimisation Lecture 2 x1 2x1 − x2 =2 x1 +2x2 =6 3 2 P 1 x2 =1 x¯ = (3/2, 1)T x2 1 2 3 4 5 Figure 6: x¯ = (3/2, 1)T is an extreme point of P x1 2x1 − x2 =2 x1 +2x2 =6 3 2 P 1 x2 =1 x¯ = (2, 1)T x2 1 2 3 4 5 Figure 7: x¯ = (2, 1)T is not an extreme point of P Example: The set {x ∈ Rn | Ax ≤ 0} is a polyhedral cone. In Figure 11 one convex and one non-convex cone are illustrated. C C C (a) A convex cone (b) A non-convex cone Figure 8: Two cones. We can now formulate a very important theorem which basically says that a polyhedron = a polytope + a polyhedral cone Theorem (The representation theorem). Let the polyhedron Q = {x ∈ Rn | Ax ≤ b} and let {v1,..., vk} be its extreme points. Define P := conv {v1,..., vk} and C := {x ∈ Rn | Ax ≤ 0}. Then Q = P + C = {x ∈ Rn | x = u + v for some u ∈ P and v ∈ C} Proof. See Theorem 3.26 in the book. 5 TMA947 / MMG621 – Nonlinear optimisation Lecture 2 T x2 y = (2, 2) T π x = α ⇔ x1 + x2 =2 S x1 T T T Figure 9: The hyperplane π x = α separates the point y = (2, 2) from the unit disc. π = (1, 1) and α = 2. Now we will present a very useful theorem for convex sets which says that: "If a point y does not lie in a closed convex set S, then there exist a hyperplane separating y from S". Mathematically, this amounts to the following. Theorem (The separation theorem). Suppose that the set S ⊆ Rn is closed and convex, and that the n point y does not lie in S. Then there exist α ∈ R and π 6= 0 such that πT y > α and πT x ≤ α for all x ∈ S. Proof. Later in the course. One last important theorem related to convex set is Farkas’ Lemma. Theorem (Farkas’ Lemma). Let A ∈ Rm×n and b ∈ Rm. Then exactly one of the systems Ax = b, (A) x ≥ 0, and T A π ≤ 0, T (B) b π > 0, has a feasible solution, and the other is inconsistent. Proof. See Theorem 3.37 in the book. Farkas’ Lemma says that: (A) Either b lies in the cone spanned by the columns of A, i.e., b = Ax, for some x ≥ 0, (B) or, b does not lie in the cone, meaning that there exists a hyperplane π separating b from the cone, i.e., ATπ ≤ 0, bTπ > 0. 6 TMA947 / MMG621 – Nonlinear optimisation Lecture 2 y y = f(x) f(x1) λf(x1)+(1 − λ)f(x2) f(x2) f(λx1 + (1 − λ)x2) x x1 λx1 + (1 − λ)x2 x2 Figure 10: A convex function Convex functions Definition (convex function). Suppose S ⊆ Rn is convex. A function f : Rn → R is convex on S if x1, x2 ∈ S =⇒ f λx1 + (1 − λ)x2 ≤ λf(x1)+(1 − λ)f(x2). λ ∈ (0, 1) – A function is strictly convex on S if < holds in place of ≤ for all x1 6= x2. – A function f is concave if −f is convex. The linear interpolation between two points on the function never is lower than the function. Two important examples: – f(x)= cTx + d, where c ∈ Rn, d ∈ R is both convex and concave.
Recommended publications
  • 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]
  • Notes on Convex Sets, Polytopes, Polyhedra, Combinatorial Topology, Voronoi Diagrams and Delaunay Triangulations
    Notes on Convex Sets, Polytopes, Polyhedra, Combinatorial Topology, Voronoi Diagrams and Delaunay Triangulations Jean Gallier and Jocelyn Quaintance Department of Computer and Information Science University of Pennsylvania Philadelphia, PA 19104, USA e-mail: [email protected] April 20, 2017 2 3 Notes on Convex Sets, Polytopes, Polyhedra, Combinatorial Topology, Voronoi Diagrams and Delaunay Triangulations Jean Gallier Abstract: Some basic mathematical tools such as convex sets, polytopes and combinatorial topology, are used quite heavily in applied fields such as geometric modeling, meshing, com- puter vision, medical imaging and robotics. This report may be viewed as a tutorial and a set of notes on convex sets, polytopes, polyhedra, combinatorial topology, Voronoi Diagrams and Delaunay Triangulations. It is intended for a broad audience of mathematically inclined readers. One of my (selfish!) motivations in writing these notes was to understand the concept of shelling and how it is used to prove the famous Euler-Poincar´eformula (Poincar´e,1899) and the more recent Upper Bound Theorem (McMullen, 1970) for polytopes. Another of my motivations was to give a \correct" account of Delaunay triangulations and Voronoi diagrams in terms of (direct and inverse) stereographic projections onto a sphere and prove rigorously that the projective map that sends the (projective) sphere to the (projective) paraboloid works correctly, that is, maps the Delaunay triangulation and Voronoi diagram w.r.t. the lifting onto the sphere to the Delaunay diagram and Voronoi diagrams w.r.t. the traditional lifting onto the paraboloid. Here, the problem is that this map is only well defined (total) in projective space and we are forced to define the notion of convex polyhedron in projective space.
    [Show full text]
  • Convex Sets and Convex Functions 1 Convex Sets
    Convex Sets and Convex Functions 1 Convex Sets, In this section, we introduce one of the most important ideas in economic modelling, in the theory of optimization and, indeed in much of modern analysis and computatyional mathematics: that of a convex set. Almost every situation we will meet will depend on this geometric idea. As an independent idea, the notion of convexity appeared at the end of the 19th century, particularly in the works of Minkowski who is supposed to have said: \Everything that is convex interests me." We discuss other ideas which stem from the basic definition, and in particular, the notion of a convex and concave functions which which are so prevalent in economic models. The geometric definition, as we will see, makes sense in any vector space. Since, for the most of our work we deal only with Rn, the definitions will be stated in that context. The interested student may, however, reformulate the definitions either, in an ab stract setting or in some concrete vector space as, for example, C([0; 1]; R)1. Intuitively if we think of R2 or R3, a convex set of vectors is a set that contains all the points of any line segment joining two points of the set (see the next figure). Here is the definition. Definition 1.1 Let u; v 2 V . Then the set of all convex combinations of u and v is the set of points fwλ 2 V : wλ = (1 − λ)u + λv; 0 ≤ λ ≤ 1g: (1.1) In, say, R2 or R3, this set is exactly the line segment joining the two points u and v.
    [Show full text]
  • OPTIMIZATION METHODS: CLASS 3 Linearity, Convexity, ANity
    OPTIMIZATION METHODS: CLASS 3 Linearity, convexity, anity The exercises are on the opposite side. D: A set A ⊆ Rd is an ane space, if A is of the form L + v for some linear space L and a shift vector v 2 Rd. By A is of the form L + v we mean a bijection between vectors of L and vectors of A given as b(u) = u + v. Each ane space has a dimension, dened as the dimension of its associated linear space L. D: A vector is an ane combination of a nite set of vectors if Pn , where x a1; a2; : : : an x = i=1 αiai are real number satisfying Pn . αi i=1 αi = 1 A set of vectors V ⊆ Rd is anely independent if it holds that no vector v 2 V is an ane combination of the rest. D: GIven a set of vectors V ⊆ Rd, we can think of its ane span, which is a set of vectors A that are all possible ane combinations of any nite subset of V . Similar to the linear spaces, ane spaces have a nite basis, so we do not need to consider all nite subsets of V , but we can generate the ane span as ane combinations of the base. D: A hyperplane is any ane space in Rd of dimension d − 1. Thus, on a 2D plane, any line is a hyperplane. In the 3D space, any plane is a hyperplane, and so on. A hyperplane splits the space Rd into two halfspaces. We count the hyperplane itself as a part of both halfspaces.
    [Show full text]
  • Vector Space and Affine Space
    Preliminary Mathematics of Geometric Modeling (1) Hongxin Zhang & Jieqing Feng State Key Lab of CAD&CG Zhejiang University Contents Coordinate Systems Vector and Affine Spaces Vector Spaces Points and Vectors Affine Combinations, Barycentric Coordinates and Convex Combinations Frames 11/20/2006 State Key Lab of CAD&CG 2 Coordinate Systems Cartesian coordinate system 11/20/2006 State Key Lab of CAD&CG 3 Coordinate Systems Frame Origin O Three Linear-Independent r rur Vectors ( uvw ,, ) 11/20/2006 State Key Lab of CAD&CG 4 Vector Spaces Definition A nonempty set ς of elements is called a vector space if in ς there are two algebraic operations, namely addition and scalar multiplication Examples of vector space Linear Independence and Bases 11/20/2006 State Key Lab of CAD&CG 5 Vector Spaces Addition Addition associates with every pair of vectors and a unique vector which is called the sum of and and is written For 2D vectors, the summation is componentwise, i.e., if and , then 11/20/2006 State Key Lab of CAD&CG 6 Vector Spaces Addition parallelogram illustration 11/20/2006 State Key Lab of CAD&CG 7 Addition Properties Commutativity Associativity Zero Vector Additive Inverse Vector Subtraction 11/20/2006 State Key Lab of CAD&CG 8 Commutativity for any two vectors and in ς , 11/20/2006 State Key Lab of CAD&CG 9 Associativity for any three vectors , and in ς, 11/20/2006 State Key Lab of CAD&CG 10 Zero Vector There is a unique vector in ς called the zero vector and denoted such that for every vector 11/20/2006 State Key Lab of CAD&CG 11 Additive
    [Show full text]
  • Convex Sets and Convex Functions (Part I)
    Convex Sets and Convex Functions (part I) Prof. Dan A. Simovici UMB 1 / 79 Outline 1 Convex and Affine Sets 2 The Convex and Affine Closures 3 Operations on Convex Sets 4 Cones 5 Extreme Points 2 / 79 Convex and Affine Sets n Special Subsets in R Let L be a real linear space and let x; y 2 L. The closed segment determined by x and y is the set [x; y] = f(1 − a)x + ay j 0 6 a 6 1g: The half-closed segments determined by x and y are the sets [x; y) = f(1 − a)x + ay j 0 6 a < 1g; and (x; y] = f(1 − a)x + ay j 0 < a 6 1g: The open segment determined by x and y is (x; y) = f(1 − a)x + ay j 0 < a < 1g: The line determined by x and y is the set `x;y = f(1 − a)x + ay j a 2 Rg: 3 / 79 Convex and Affine Sets Definition A subset C of L is convex if we have [x; y] ⊆ C for all x; y 2 C. Note that the empty subset and every singleton fxg of L are convex. 4 / 79 Convex and Affine Sets Convex vs. Non-convex x3 x4 x2 x4 x x y x2 x3 y x1 x1 (a) (b) 5 / 79 Convex and Affine Sets Example The set n of all vectors of n having non-negative components is a R>0 R n convex set called the non-negative orthant of R . 6 / 79 Convex and Affine Sets Example The convex subsets of (R; +; ·) are the intervals of R.
    [Show full text]
  • Lecture 2 - Introduction to Polytopes
    Lecture 2 - Introduction to Polytopes Optimization and Approximation - ENS M1 Nicolas Bousquet 1 Reminder of Linear Algebra definitions n Pm Let x1; : : : ; xm be points in R and λ1; : : : ; λm be real numbers. Then x = i=1 λixi is said to be a: • Linear combination (of x1; : : : ; xm) if the λi are arbitrary scalars. • Conic combination if λi ≥ 0 for every i. Pm • Convex combination if i=1 λi = 1 and λi ≥ 0 for every i. In the following, λ will still denote a scalar (since we consider in real spaces, λ is a real number). The linear space spanned by X = fx1; : : : ; xmg (also called the span of X), denoted by Span(X), is the set of n n points x of R which can be expressed as linear combinations of x1; : : : ; xm. Given a set X of R , the span of X is the smallest vectorial space containing the set X. In the following we will consider a little bit further the other types of combinations. Pm A set x1; : : : ; xm of vectors are linearly independent if i=1 λixi = 0 implies that for every i ≤ m, λi = 0. The dimension of the space spanned by x1; : : : ; xm is the cardinality of a maximum subfamily of x1; : : : ; xm which is linearly independent. The points x0; : : : ; x` of an affine space are said to be affinely independent if the vectors x1−x0; : : : ; x`− x0 are linearly independent. In other words, if we consider the space to be “centered” on x0 then the vectors corresponding to the other points in the vectorial space are independent.
    [Show full text]
  • An Introduction to Convex Polytopes
    Graduate Texts in Mathematics Arne Brondsted An Introduction to Convex Polytopes 9, New YorkHefdelbergBerlin Graduate Texts in Mathematics90 Editorial Board F. W. GehringP. R. Halmos (Managing Editor) C. C. Moore Arne Brondsted An Introduction to Convex Polytopes Springer-Verlag New York Heidelberg Berlin Arne Brondsted K, benhavns Universitets Matematiske Institut Universitetsparken 5 2100 Kobenhavn 0 Danmark Editorial Board P. R. Halmos F. W. Gehring C. C. Moore Managing Editor University of Michigan University of California Indiana University Department of at Berkeley Department of Mathematics Department of Mathematics Ann Arbor, MI 48104 Mathematics Bloomington, IN 47405 U.S.A. Berkeley, CA 94720 U.S.A. U.S.A. AMS Subject Classifications (1980): 52-01, 52A25 Library of Congress Cataloging in Publication Data Brondsted, Arne. An introduction to convex polytopes. (Graduate texts in mathematics; 90) Bibliography : p. 1. Convex polytopes.I. Title.II. Series. QA64.0.3.B76 1982 514'.223 82-10585 With 3 Illustrations. © 1983 by Springer-Verlag New York Inc. All rights reserved. No part of this book may be translated or reproduced in any form without written permission from Springer-Verlag, 175 Fifth Avenue, New York, New York 10010, U.S.A. Typeset by Composition House Ltd., Salisbury, England. Printed and bound by R. R. Donnelley & Sons, Harrisonburg, VA. Printed in the United States of America. 987654321 ISBN 0-387-90722-X Springer-Verlag New York Heidelberg Berlin ISBN 3-540-90722-X Springer-Verlag Berlin Heidelberg New York Preface The aim of this book is to introduce the reader to the fascinating world of convex polytopes. The highlights of the book are three main theorems in the combinatorial theory of convex polytopes, known as the Dehn-Sommerville Relations, the Upper Bound Theorem and the Lower Bound Theorem.
    [Show full text]
  • Weak Matrix Majorization Francisco D
    Linear Algebra and its Applications 403 (2005) 343–368 www.elsevier.com/locate/laa Weak matrix majorization Francisco D. Martínez Pería a,∗, Pedro G. Massey a, Luis E. Silvestre b aDepartamento de Matemática, Facultad de Ciencias Exactas, Universidad Nacional de La Plata, CC 172, La Plata, Argentina bDepartment of Mathematics, University of Texas at Austin, Austin, USA Received 19 May 2004; accepted 10 February 2005 Available online 31 March 2005 Submitted by R.A. Brualdi Abstract × Given X, Y ∈ Rn m we introduce the following notion of matrix majorization, called weak matrix majorization, n×n X w Y if there exists a row-stochastic matrix A ∈ R such that AX = Y, and consider the relations between this concept, strong majorization (s) and directional maj- orization (). It is verified that s⇒⇒w, but none of the reciprocal implications is true. Nevertheless, we study the implications w⇒s and ⇒s under additional hypotheses. We give characterizations of strong, directional and weak matrix majorization in terms of convexity. We also introduce definitions for majorization between Abelian families of selfadjoint matrices, called joint majorizations. They are induced by the previously mentioned matrix majorizations. We obtain descriptions of these relations using convexity arguments. © 2005 Elsevier Inc. All rights reserved. AMS classification: Primary 15A51; 15A60; 15A45 Keywords: Multivariate and directional matrix majorizations; Row stochastic matrices; Mutually com- muting selfadjoint matrices; Convex sets and functions ∗ Corresponding author. E-mail addresses: [email protected] (F.D. Mart´ınez Per´ıa), [email protected] (P.G. Massey), [email protected] (L.E. Silvestre).
    [Show full text]
  • Lecture 2: Convex Sets
    Lecture 2: Convex sets August 28, 2008 Lecture 2 Outline • Review basic topology in Rn • Open Set and Interior • Closed Set and Closure • Dual Cone • Convex set • Cones • Affine sets • Half-Spaces, Hyperplanes, Polyhedra • Ellipsoids and Norm Cones • Convex, Conical, and Affine Hulls • Simplex • Verifying Convexity Convex Optimization 1 Lecture 2 Topology Review n Let {xk} be a sequence of vectors in R n n Def. The sequence {xk} ⊆ R converges to a vector xˆ ∈ R when kxk − xˆk tends to 0 as k → ∞ • Notation: When {xk} converges to a vector xˆ, we write xk → xˆ n • The sequence {xk} converges xˆ ∈ R if and only if for each component i: the i-th components of xk converge to the i-th component of xˆ i i |xk − xˆ | tends to 0 as k → ∞ Convex Optimization 2 Lecture 2 Open Set and Interior Let X ⊆ Rn be a nonempty set Def. The set X is open if for every x ∈ X there is an open ball B(x, r) that entirely lies in the set X, i.e., for each x ∈ X there is r > 0 s.th. for all z with kz − xk < r, we have z ∈ X Def. A vector x0 is an interior point of the set X, if there is a ball B(x0, r) contained entirely in the set X Def. The interior of the set X is the set of all interior points of X, denoted by R (X) • How is R (X) related to X? 2 • Example X = {x ∈ R | x1 ≥ 0, x2 > 0} R 2 (X) = {x ∈ R | x1 > 0, x2 > 0} R n 0 (S) of a probability simplex S = {x ∈ R | x 0, e x = 1} Th.
    [Show full text]
  • Lecture 3 Convex Functions
    Lecture 3 Convex functions (Basic properties; Calculus; Closed functions; Continuity of convex functions; Subgradients; Optimality conditions) 3.1 First acquaintance Definition 3.1.1 [Convex function] A function f : M ! R defined on a nonempty subset M of Rn and taking real values is called convex, if • the domain M of the function is convex; • for any x; y 2 M and every λ 2 [0; 1] one has f(λx + (1 − λ)y) ≤ λf(x) + (1 − λ)f(y): (3.1.1) If the above inequality is strict whenever x 6= y and 0 < λ < 1, f is called strictly convex. A function f such that −f is convex is called concave; the domain M of a concave function should be convex, and the function itself should satisfy the inequality opposite to (3.1.1): f(λx + (1 − λ)y) ≥ λf(x) + (1 − λ)f(y); x; y 2 M; λ 2 [0; 1]: The simplest example of a convex function is an affine function f(x) = aT x + b { the sum of a linear form and a constant. This function clearly is convex on the entire space, and the \convexity inequality" for it is equality; the affine function is also concave. It is easily seen that the function which is both convex and concave on the entire space is an affine function. Here are several elementary examples of \nonlinear" convex functions of one variable: 53 54 LECTURE 3. CONVEX FUNCTIONS • functions convex on the whole axis: x2p, p being positive integer; expfxg; • functions convex on the nonnegative ray: xp, 1 ≤ p; −xp, 0 ≤ p ≤ 1; x ln x; • functions convex on the positive ray: 1=xp, p > 0; − ln x.
    [Show full text]
  • Proquest Dissertations
    u Ottawa L'Universitd canadienne Canada's university FACULTE DES ETUDES SUPERIEURES l==I FACULTY OF GRADUATE AND ET POSTOCTORALES U Ottawa POSDOCTORAL STUDIES L'Universit6 canadienne Canada's university Guy Beaulieu "MEWDE"UATH£S17XUTHORWTHE"STS" Ph.D. (Mathematics) GRADE/DEGREE Department of Mathematics and Statistics 7ACulTirfc6L17bT^ Probabilistic Completion of Nondeterministic Models TITRE DE LA THESE / TITLE OF THESIS Philip Scott DIREWEURlbTRECTRicirDE'iSTHESE"/ THESIS SUPERVISOR EXAMINATEURS (EXAMINATRICES) DE LA THESE /THESIS EXAMINERS Richard Blute _ _ Paul-Eugene Parent Michael Mislove Benjamin Steinberg G ^y.W:.Slater.. Le Doyen de la Faculte des etudes superieures et postdoctorales / Dean of the Faculty of Graduate and Postdoctoral Studies PROBABILISTIC COMPLETION OF NONDETERMINISTIC MODELS By Guy Beaulieu, B.Sc, M.S. Thesis submitted to the Faculty of Graduate and Postdoctoral Studies University of Ottawa in partial fulfillment of the requirements for the PhD degree in the Ottawa-Carleton Institute for Graduate Studies and Research in Mathematics and Statistics ©2008 Guy Beaulieu, B.Sc, M.S. Library and Bibliotheque et 1*1 Archives Canada Archives Canada Published Heritage Direction du Branch Patrimoine de I'edition 395 Wellington Street 395, rue Wellington Ottawa ON K1A0N4 Ottawa ON K1A0N4 Canada Canada Your file Votre reference ISBN: 978-0-494-48387-9 Our file Notre reference ISBN: 978-0-494-48387-9 NOTICE: AVIS: The author has granted a non­ L'auteur a accorde une licence non exclusive exclusive license allowing Library
    [Show full text]