Numerical Optimization

Size: px
Start display at page:

Download "Numerical Optimization"

Transcription

1 Convex Sets Computer Science and Automation Indian Institute of Science Bangalore , India. NPTEL Course on

2 Let x 1, x 2 R n, x 1 x 2. Line and line segment Line passing through x 1 and x 2 : {y R n : y = λx 1 + (1 λ)x 2, λ R} Line Segment, LS[x 1, x 2 ]: {y R n : y = λx 1 + (1 λ)x 2, λ [0, 1]}

3 Affine sets Definition A set X R n is affine if for any x 1, x 2 X, and λ R, λx 1 + (1 λ)x 2 X. If X R n is an affine set, x 1, x 2,..., x k X and i λ i = 1, then the point λ 1 x 1 + λ 2 x λ k x k X. Examples Solution set of linear equations: {x R n : Ax = b} where A R m n, b R m. A subspace or a translated subspace

4

5 Result If X is an affine set and x 0 X, then {x x 0 : x X} forms a subspace. Proof. Let Y = {x x 0 : x X}. To show that Y is a subspace, we need to show, αy 1 + βy 2 Y for any y 1, y 2 Y and α, β R. Let y 1, y 2 Y and α, β R. Therefore, y 1 + x 0 X and y 2 + x 0 X. αy 1 + βy 2 = α(y 1 + x 0 ) + β(y 2 + x 0 ) (α + β)x 0. αy 1 + βy 2 + x 0 = α(y 1 + x 0 ) + β(y 2 + x 0 ) + (1 α β)x 0. Since X is an affine set, αy 1 + βy 2 + x 0 X. Thus, αy 1 + βy 2 Y Y is a subspace.

6 Definition Let X = {x 1, x 2,..., x k }. A point x is said to be an affine combination of points in X if x = k λ i x i, i=1 k λ i = 1. i=1 Definition Let X R n. The set of all affine combinations of points in X is called the affine hull of X. aff(x) = { k λ i x i : x 1,..., x k X, i i=1 λ i = 1}

7 Convex Sets Definition A set C R n is convex if for any x 1, x 2 C and any scalar λ with 0 λ 1, we have Examples Some simple convex sets λx 1 + (1 λ)x 2 C.

8 Some examples of nonconvex sets

9 Convex sets Examples: The empty set φ, any singleton set {x 0 } and R n are convex subsets of R n. A closed ball in R n, B[x 0, r] and an open ball in R n, B(x 0, r), are convex sets. Any affine set is a convex set. A line segment is a convex set, but not an affine set.

10 Possible to construct new convex sets using given convex sets Definition Let P R n, Q R n, α R. The scalar multiple αp of the set P is defined as αp = {x : x = αp, p P} The sum of two sets P and Q is the set, P + Q = {x : x = p + q, p P, q Q}.

11 Theorem If {C i }, i A, is any collection of convex sets, then i A C i is a convex set. Proof. Let C = i A C i. Case 1. If C is empty or singleton, then clearly C is a convex set. Case 2. To show that, for any x 1, x 2 C and λ [0, 1], λx 1 + (1 λ)x 2 C. Let x 1, x 2 C. Clearly, x 1, x 2 C i for every i A. Since every C i is convex, λx 1 + (1 λ)x 2 C i, i A, λ [0, 1] λx 1 + (1 λ)x 2 i A C i, λ [0, 1] λx 1 + (1 λ)x 2 C, λ [0, 1].

12 Theorem If C 1 and C 2 are convex sets, then C 1 + C 2 is a convex set. Proof. Let x 1, y 1 C 1 and x 2, y 2 C 2. So, x 1 + x 2, y 1 + y 2 C 1 + C 2. We need to show, λ(x 1 + x 2 ) + (1 λ)(y 1 + y 2 ) C 1 + C 2 λ [0, 1]. Since C 1 and C 2 are convex, z 1 = λx 1 + (1 λ)y 1 C 1 λ [0, 1], and z 2 = λx 2 + (1 λ)y 2 C 2 λ [0, 1]. Thus, z 1 + z 2 C 1 + C (1) Now, x 1 + x 2 C 1 + C 2 and y 1 + y 2 C 1 + C 2. Therefore, from (1), z 1 + z 2 = λ(x 1 + x 2 ) + (1 λ)(y 1 + y 2 ) C 1 + C 2 λ [0, 1]. Thus, C 1 + C 2 is a convex set.

13 Theorem If C is a convex set and α R, then αc is a convex set. Proof. Let x 1, x 2 C. Since C is convex, λx 1 + (1 λ)x 2 C λ [0, 1]. Also, αx 1, αx 2 αc. Therefore, λ(αx 1 ) + (1 λ)(αx 2 ) = α(λx 1 + (1 λ)x 2 ) αc for any λ [0, 1]. Therefore, αc is a convex set.

14 Hyperplane Definition Let b R and a R n, a 0. Then, the set is said to be a hyperplane in R n. H = {x : a T x = b} a denotes the normal to the hyperplane H. If a = 1, then b is the distance of H from the origin. In R 2, hyperplane is a line In R 3, hyperplane is a plane

15

16

17

18 Half-spaces The sets H + = {x : a T x b} and H = {x : a T x b} are called closed positive and negative half-spaces generated by H.

19

20 Some more examples of convex sets H = {x : a T x = b} is a convex set Let a 1, a 2,..., a m R n and b 1, b 2,..., b m R a T 1 b 1 a T 2 Define, A =. and b = b 2. a T m Then, {x : Ax = b} is a convex set. H + = {x : a T x b} and H = {x : a T x b} are convex sets. b m {x : Ax b} and {x : Ax b} are convex sets.

21

22

23

24

25 Convex Hull Definition The convex hull of a set S is the intersection of all the convex sets which contain S and is denoted by conv(s). Note: Convex Hull of a set S is the convex set. The smallest convex set that contains S is called the convex hull of the set S. Examples: conv({x, y}) = LS[x, y] where x and y are two points Let S = {(x, 0) : x R} {(0, y) : y R}. Then conv(s) = R 2.

26

27

28

29 S = {(x 1, x 2 ) : x 2 = x 2 1} conv(s) = {(x 1, x 2 ) : x 2 x 2 1}

30 Theorem CS1 Let S R n be a nonempty, closed convex set and y / S. Then there exists a unique point x 0 S with minimum distance from y. Further, x 0 is the minimizing point iff (y x 0 ) T (x x 0 ) 0 for all x S.

31 Proof Sketch Given S R n, a closed convex set and y / S. First show that there exists a minimizing point x 0 in S that is closest to y. Let δ = inf x S x y. Note that S is not bounded.

32 Proof Sketch (continued) Consider the set S B[y, 2δ]. By Weierstrass Theorem, there exists a minimizing point x 0 in S that is closest to y. x 0 = arg min x S B[y,2δ] x y

33 Proof Sketch (continued) Show uniqueness using triangle inequality Assume that there exists ˆx S such that y x 0 = y ˆx = δ. Since S is convex, 1 2 (x 0 + ˆx) S. Using triangle inequality, 2 y (x 0 + ˆx) y x 0 + y ˆx = 2δ 2 We have a contradiction if strict inequality holds.

34 Proof Sketch (continued) To show that x 0 is the unique minimizing point iff (y x 0 ) T (x x 0 ) 0 for all x S. Let x S. Assume (y x 0 ) T (x x 0 ) 0. y x 2 = y x 0 + x 0 x 2 = y x x 0 x 2 + 2(y x 0 ) T (x 0 x) Using the assumption, (y x 0 ) T (x 0 x) 0, we get y x 2 y x 0 2 This implies that x 0 is the minimizing point.

35 Proof Sketch (continued) Assume that x 0 is the minimizing point, that is, y x 0 2 y z 2 z S. Consider any x S. Since S is convex, λx + (1 λ)x 0 S λ [0, 1]. Therefore, y x 0 2 y x 0 λ(x x 0 ) 2 That is, y x 0 2 y x 0 2 +λ 2 x x 0 ) 2 2λ(y x 0 ) T (x x 0 ) 2(y x 0 ) T (x x 0 ) λ x x 0 ) 2 Letting λ 0 +, the result follows.

36 Theorem CS1 Let S R n be a nonempty, closed convex set and y / S. Then there exists a unique point x 0 S with minimum distance from y. Further, x 0 is the minimizing point iff (y x 0 ) T (x x 0 ) 0 for all x S.

37 Separating hyperplanes Definition Let S 1 and S 2 be nonempty subsets in R n and H = {x : a T x = b} be a hyperplane. 1 The hyperplane H is said to separate S 1 and S 2, if a T x b x S 1 and a T x b x S 2. 2 If a T x > b x S 1 and a T x < b x S 2, then the hyperplane H is said to strictly separate S 1 and S 2. 3 The hyperplane H is said to strongly separate S 1 and S 2 if a T x b + ɛ x S 1 and a T x b x S 2 where ɛ is a positive scalar.

38 H: Separating hyperplane The hyperplane H = {x : a T x = b} is said to separate S 1 and S 2, if a T x b x S 1 and a T x b x S 2.

39 H: Strictly separating hyperplane If a T x > b x S 1 and a T x < b x S 2, then the hyperplane H = {x : a T x = b} is said to strictly separate S 1 and S 2.

40 H: Strongly separating hyperplane The hyperplane H = {x : a T x = b} is said to strongly separate S 1 and S 2 if a T x b + ɛ x S 1 and a T x b x S 2 where ɛ is a positive scalar.

41 Separation of a closed convex set and a point Result Let S be a nonempty closed convex set in R n and y / S. Then there exists a nonzero vector a and a scalar b such that a T y > b and a T x b x S. Proof. By Theorem CS1, there exists a unique minimizing point x 0 S such that (x x 0 ) T (y x 0 ) 0 for each x S. Letting a = (y x 0 ) and b = a T x 0, we get a T x b for each x S and a T y b = (y x 0 ) T (y x 0 ) > 0 (since y x 0 ).

42 Cone Definition A set K R n is called a cone if for every x K and λ 0, we have λx K. K is a convex cone if it is convex and a cone.

43 Some examples of cones

44 Farkas Lemma Farkas Lemma Let A R m n and c R n. Then, exactly one of the following two systems has a solution: (I) Ax 0, c T x > 0 for some x R n (II) A T y = c, y 0 for some y R m.

45 Let a 1, a 2,..., a m R n. a T 1 a T 2 Define, A =.. a T m For example,

46

47

48 Farkas Lemma (Geometrical Interpretation) Exactly one of the following two systems has a solution: (I) Ax 0, c T x > 0 for some x R n (II) A T y = c, y 0 for some y R m

49 Farkas Lemma Let A R m n and c R n. Then, exactly one of the following two systems has a solution: (I) Ax 0, c T x > 0 (II) A T y = c, y 0 for some x R n for some y R m Proof of Farkas Lemma (a) Suppose, system (II) has a solution. Therefore, y 0 such that c = A T y. Consider x R n such that Ax 0. So, c T x = y T Ax 0. That is, System I has no solution.

50 Farkas Lemma Let A R m n and c R n. Then, exactly one of the following two systems has a solution: (I) Ax 0, c T x > 0 (II) A T y = c, y 0 for some x R n for some y R m Proof of Farkas Lemma (continued) (b) Suppose, system (II) has no solution. Let S = {x : x = A T y, y 0}, a closed convex set and c / S. Therefore, p R n and α R such that p T x α x S and c T p > α. This means, α 0 (Since 0 S) c T p > 0. Also, α p T A T y = y T Ap y 0. Since y 0, Ap 0 (as y can be made arbitrarily large). Thus, p R n such that Ap 0, c T p > 0 System (I) has a solution.

51 Farkas Lemma Let A R m n and c R n. Then, exactly one of the following two systems has a solution: (I) Ax 0, c T x > 0 for some x R n (II) A T y = c, y 0 for some y R m. Corollary Let A R m n. Then exactly one of the following systems has a solution: (I) Ax < 0 for some x R n (II) A T y = 0, y 0 for some nonzero y R m.

52 Corollary Let A R m n. Then exactly one of the following systems has a solution: (I) Ax < 0 for some x R n (II) A T y = 0, y 0 for some nonzero y R m. Proof. We can write system I as Ax + ze 0 for some x R n, z > 0 where e is a m-dimensional vector containing all 1 s. That is, ( ) ( ) x x (A e) 0, (0,..., 0, 1) > 0 z z for some (x z) T R n+1.

53 Proof. (continued) Recall Farkas Lemma. Therefore, System II is ( ) A T y = (0,..., 0, 1) T, y 0 for some y R m. e T That is A T y = 0, e T y = 1 and y 0 for some y R m. Using Farkas Lemma, the result follows.

54 Supporting Hyperplanes of sets at boundary points Definition Let S R n, S φ. Let x 0 be a boundary point of S. A hyperplane H = {x : a T (x x 0 ) = 0} is called a supporting hyperplane of S at x 0, if either S H + (that is, a T (x x 0 ) 0 x S), or S H (that is, a T (x x 0 ) 0 x S).

55 Theorem Let S be a nonempty convex set in R n and x 0 be a boundary point of S. Then, there exists a hyperplane that supports S at x 0.

56 Theorem Let S 1 and S 2 be two nonempty disjoint convex sets in R n. Then, there exists a hyperplane that separates S 1 and S 2. Proof. Consider the set S = S 1 S 2 = {x 1 x 2 : x 1 S 1, x 2 S 2 }. Note that S is a convex set and 0 / S. Thus, we have a convex set and a point not in that set. So, there exists a vector a such that a T x 0 x S. In other words, a T x 1 a T x 2 x 1 S 1, x 2 S 2.

EC 521 MATHEMATICAL METHODS FOR ECONOMICS. Lecture 2: Convex Sets

EC 521 MATHEMATICAL METHODS FOR ECONOMICS. Lecture 2: Convex Sets EC 51 MATHEMATICAL METHODS FOR ECONOMICS Lecture : Convex Sets Murat YILMAZ Boğaziçi University In this section, we focus on convex sets, separating hyperplane theorems and Farkas Lemma. And as an application

More information

Math 5593 Linear Programming Lecture Notes

Math 5593 Linear Programming Lecture Notes Math 5593 Linear Programming Lecture Notes Unit II: Theory & Foundations (Convex Analysis) University of Colorado Denver, Fall 2013 Topics 1 Convex Sets 1 1.1 Basic Properties (Luenberger-Ye Appendix B.1).........................

More information

Lecture 2 - Introduction to Polytopes

Lecture 2 - Introduction to Polytopes Lecture 2 - Introduction to Polytopes Optimization and Approximation - ENS M1 Nicolas Bousquet 1 Reminder of Linear Algebra definitions Let x 1,..., x m be points in R n and λ 1,..., λ m be real numbers.

More information

Lecture 2. Topology of Sets in R n. August 27, 2008

Lecture 2. Topology of Sets in R n. August 27, 2008 Lecture 2 Topology of Sets in R n August 27, 2008 Outline Vectors, Matrices, Norms, Convergence Open and Closed Sets Special Sets: Subspace, Affine Set, Cone, Convex Set Special Convex Sets: Hyperplane,

More information

Lecture 5: Duality Theory

Lecture 5: Duality Theory Lecture 5: Duality Theory Rajat Mittal IIT Kanpur The objective of this lecture note will be to learn duality theory of linear programming. We are planning to answer following questions. What are hyperplane

More information

Division of the Humanities and Social Sciences. Convex Analysis and Economic Theory Winter Separation theorems

Division of the Humanities and Social Sciences. Convex Analysis and Economic Theory Winter Separation theorems Division of the Humanities and Social Sciences Ec 181 KC Border Convex Analysis and Economic Theory Winter 2018 Topic 8: Separation theorems 8.1 Hyperplanes and half spaces Recall that a hyperplane in

More information

Convex Sets. CSCI5254: Convex Optimization & Its Applications. subspaces, affine sets, and convex sets. operations that preserve convexity

Convex Sets. CSCI5254: Convex Optimization & Its Applications. subspaces, affine sets, and convex sets. operations that preserve convexity CSCI5254: Convex Optimization & Its Applications Convex Sets subspaces, affine sets, and convex sets operations that preserve convexity generalized inequalities separating and supporting hyperplanes dual

More information

However, this is not always true! For example, this fails if both A and B are closed and unbounded (find an example).

However, this is not always true! For example, this fails if both A and B are closed and unbounded (find an example). 98 CHAPTER 3. PROPERTIES OF CONVEX SETS: A GLIMPSE 3.2 Separation Theorems It seems intuitively rather obvious that if A and B are two nonempty disjoint convex sets in A 2, then there is a line, H, separating

More information

Convex Sets. Pontus Giselsson

Convex Sets. Pontus Giselsson Convex Sets Pontus Giselsson 1 Today s lecture convex sets convex, affine, conical hulls closure, interior, relative interior, boundary, relative boundary separating and supporting hyperplane theorems

More information

Convex Geometry arising in Optimization

Convex Geometry arising in Optimization Convex Geometry arising in Optimization Jesús A. De Loera University of California, Davis Berlin Mathematical School Summer 2015 WHAT IS THIS COURSE ABOUT? Combinatorial Convexity and Optimization PLAN

More information

Conic Duality. yyye

Conic Duality.  yyye Conic Linear Optimization and Appl. MS&E314 Lecture Note #02 1 Conic Duality Yinyu Ye Department of Management Science and Engineering Stanford University Stanford, CA 94305, U.S.A. http://www.stanford.edu/

More information

Convexity: an introduction

Convexity: an introduction Convexity: an introduction Geir Dahl CMA, Dept. of Mathematics and Dept. of Informatics University of Oslo 1 / 74 1. Introduction 1. Introduction what is convexity where does it arise main concepts and

More information

REVIEW OF FUZZY SETS

REVIEW OF FUZZY SETS REVIEW OF FUZZY SETS CONNER HANSEN 1. Introduction L. A. Zadeh s paper Fuzzy Sets* [1] introduces the concept of a fuzzy set, provides definitions for various fuzzy set operations, and proves several properties

More information

Locally convex topological vector spaces

Locally convex topological vector spaces Chapter 4 Locally convex topological vector spaces 4.1 Definition by neighbourhoods Let us start this section by briefly recalling some basic properties of convex subsets of a vector space over K (where

More information

Chapter 4 Concepts from Geometry

Chapter 4 Concepts from Geometry Chapter 4 Concepts from Geometry An Introduction to Optimization Spring, 2014 Wei-Ta Chu 1 Line Segments The line segment between two points and in R n is the set of points on the straight line joining

More information

FACES OF CONVEX SETS

FACES OF CONVEX SETS FACES OF CONVEX SETS VERA ROSHCHINA Abstract. We remind the basic definitions of faces of convex sets and their basic properties. For more details see the classic references [1, 2] and [4] for polytopes.

More information

Advanced Operations Research Techniques IE316. Quiz 1 Review. Dr. Ted Ralphs

Advanced Operations Research Techniques IE316. Quiz 1 Review. Dr. Ted Ralphs Advanced Operations Research Techniques IE316 Quiz 1 Review Dr. Ted Ralphs IE316 Quiz 1 Review 1 Reading for The Quiz Material covered in detail in lecture. 1.1, 1.4, 2.1-2.6, 3.1-3.3, 3.5 Background material

More information

2. Convex sets. x 1. x 2. affine set: contains the line through any two distinct points in the set

2. Convex sets. x 1. x 2. affine set: contains the line through any two distinct points in the set 2. Convex sets Convex Optimization Boyd & Vandenberghe affine and convex sets some important examples operations that preserve convexity generalized inequalities separating and supporting hyperplanes dual

More information

Math 414 Lecture 2 Everyone have a laptop?

Math 414 Lecture 2 Everyone have a laptop? Math 44 Lecture 2 Everyone have a laptop? THEOREM. Let v,...,v k be k vectors in an n-dimensional space and A = [v ;...; v k ] v,..., v k independent v,..., v k span the space v,..., v k a basis v,...,

More information

Lecture 3: Convex sets

Lecture 3: Convex sets Lecture 3: Convex sets Rajat Mittal IIT Kanpur We denote the set of real numbers as R. Most of the time we will be working with space R n and its elements will be called vectors. Remember that a subspace

More information

2. Convex sets. affine and convex sets. some important examples. operations that preserve convexity. generalized inequalities

2. Convex sets. affine and convex sets. some important examples. operations that preserve convexity. generalized inequalities 2. Convex sets Convex Optimization Boyd & Vandenberghe affine and convex sets some important examples operations that preserve convexity generalized inequalities separating and supporting hyperplanes dual

More information

maximize c, x subject to Ax b,

maximize c, x subject to Ax b, Lecture 8 Linear programming is about problems of the form maximize c, x subject to Ax b, where A R m n, x R n, c R n, and b R m, and the inequality sign means inequality in each row. The feasible set

More information

POLYHEDRAL GEOMETRY. Convex functions and sets. Mathematical Programming Niels Lauritzen Recall that a subset C R n is convex if

POLYHEDRAL GEOMETRY. Convex functions and sets. Mathematical Programming Niels Lauritzen Recall that a subset C R n is convex if POLYHEDRAL GEOMETRY Mathematical Programming Niels Lauritzen 7.9.2007 Convex functions and sets Recall that a subset C R n is convex if {λx + (1 λ)y 0 λ 1} C for every x, y C and 0 λ 1. A function f :

More information

60 2 Convex sets. {x a T x b} {x ã T x b}

60 2 Convex sets. {x a T x b} {x ã T x b} 60 2 Convex sets Exercises Definition of convexity 21 Let C R n be a convex set, with x 1,, x k C, and let θ 1,, θ k R satisfy θ i 0, θ 1 + + θ k = 1 Show that θ 1x 1 + + θ k x k C (The definition of convexity

More information

Lecture 2 September 3

Lecture 2 September 3 EE 381V: Large Scale Optimization Fall 2012 Lecture 2 September 3 Lecturer: Caramanis & Sanghavi Scribe: Hongbo Si, Qiaoyang Ye 2.1 Overview of the last Lecture The focus of the last lecture was to give

More information

Convex Optimization. 2. Convex Sets. Prof. Ying Cui. Department of Electrical Engineering Shanghai Jiao Tong University. SJTU Ying Cui 1 / 33

Convex Optimization. 2. Convex Sets. Prof. Ying Cui. Department of Electrical Engineering Shanghai Jiao Tong University. SJTU Ying Cui 1 / 33 Convex Optimization 2. Convex Sets Prof. Ying Cui Department of Electrical Engineering Shanghai Jiao Tong University 2018 SJTU Ying Cui 1 / 33 Outline Affine and convex sets Some important examples Operations

More information

Convex Optimization. Convex Sets. ENSAE: Optimisation 1/24

Convex Optimization. Convex Sets. ENSAE: Optimisation 1/24 Convex Optimization Convex Sets ENSAE: Optimisation 1/24 Today affine and convex sets some important examples operations that preserve convexity generalized inequalities separating and supporting hyperplanes

More information

Lecture 19 Subgradient Methods. November 5, 2008

Lecture 19 Subgradient Methods. November 5, 2008 Subgradient Methods November 5, 2008 Outline Lecture 19 Subgradients and Level Sets Subgradient Method Convergence and Convergence Rate Convex Optimization 1 Subgradients and Level Sets A vector s is a

More information

CS522: Advanced Algorithms

CS522: Advanced Algorithms Lecture 1 CS5: Advanced Algorithms October 4, 004 Lecturer: Kamal Jain Notes: Chris Re 1.1 Plan for the week Figure 1.1: Plan for the week The underlined tools, weak duality theorem and complimentary slackness,

More information

Combinatorial Geometry & Topology arising in Game Theory and Optimization

Combinatorial Geometry & Topology arising in Game Theory and Optimization Combinatorial Geometry & Topology arising in Game Theory and Optimization Jesús A. De Loera University of California, Davis LAST EPISODE... We discuss the content of the course... Convex Sets A set is

More information

Shiqian Ma, MAT-258A: Numerical Optimization 1. Chapter 2. Convex Optimization

Shiqian Ma, MAT-258A: Numerical Optimization 1. Chapter 2. Convex Optimization Shiqian Ma, MAT-258A: Numerical Optimization 1 Chapter 2 Convex Optimization Shiqian Ma, MAT-258A: Numerical Optimization 2 2.1. Convex Optimization General optimization problem: min f 0 (x) s.t., f i

More information

MTAEA Convexity and Quasiconvexity

MTAEA Convexity and Quasiconvexity School of Economics, Australian National University February 19, 2010 Convex Combinations and Convex Sets. Definition. Given any finite collection of points x 1,..., x m R n, a point z R n is said to be

More information

Convex Optimization - Chapter 1-2. Xiangru Lian August 28, 2015

Convex Optimization - Chapter 1-2. Xiangru Lian August 28, 2015 Convex Optimization - Chapter 1-2 Xiangru Lian August 28, 2015 1 Mathematical optimization minimize f 0 (x) s.t. f j (x) 0, j=1,,m, (1) x S x. (x 1,,x n ). optimization variable. f 0. R n R. objective

More information

Convex Sets (cont.) Convex Functions

Convex Sets (cont.) Convex Functions Convex Sets (cont.) Convex Functions Optimization - 10725 Carlos Guestrin Carnegie Mellon University February 27 th, 2008 1 Definitions of convex sets Convex v. Non-convex sets Line segment definition:

More information

Lecture 6: Faces, Facets

Lecture 6: Faces, Facets IE 511: Integer Programming, Spring 2019 31 Jan, 2019 Lecturer: Karthik Chandrasekaran Lecture 6: Faces, Facets Scribe: Setareh Taki Disclaimer: These notes have not been subjected to the usual scrutiny

More information

Topological properties of convex sets

Topological properties of convex sets Division of the Humanities and Social Sciences Ec 181 KC Border Convex Analysis and Economic Theory Winter 2018 Topic 5: Topological properties of convex sets 5.1 Interior and closure of convex sets Let

More information

MA4254: Discrete Optimization. Defeng Sun. Department of Mathematics National University of Singapore Office: S Telephone:

MA4254: Discrete Optimization. Defeng Sun. Department of Mathematics National University of Singapore Office: S Telephone: MA4254: Discrete Optimization Defeng Sun Department of Mathematics National University of Singapore Office: S14-04-25 Telephone: 6516 3343 Aims/Objectives: Discrete optimization deals with problems of

More information

CS675: Convex and Combinatorial Optimization Spring 2018 Convex Sets. Instructor: Shaddin Dughmi

CS675: Convex and Combinatorial Optimization Spring 2018 Convex Sets. Instructor: Shaddin Dughmi CS675: Convex and Combinatorial Optimization Spring 2018 Convex Sets Instructor: Shaddin Dughmi Outline 1 Convex sets, Affine sets, and Cones 2 Examples of Convex Sets 3 Convexity-Preserving Operations

More information

Lecture 4: Convexity

Lecture 4: Convexity 10-725: Convex Optimization Fall 2013 Lecture 4: Convexity Lecturer: Barnabás Póczos Scribes: Jessica Chemali, David Fouhey, Yuxiong Wang Note: LaTeX template courtesy of UC Berkeley EECS dept. Disclaimer:

More information

Lecture 2: August 29, 2018

Lecture 2: August 29, 2018 10-725/36-725: Convex Optimization Fall 2018 Lecturer: Ryan Tibshirani Lecture 2: August 29, 2018 Scribes: Adam Harley Note: LaTeX template courtesy of UC Berkeley EECS dept. Disclaimer: These notes have

More information

Convex Optimization Lecture 2

Convex Optimization Lecture 2 Convex Optimization Lecture 2 Today: Convex Analysis Center-of-mass Algorithm 1 Convex Analysis Convex Sets Definition: A set C R n is convex if for all x, y C and all 0 λ 1, λx + (1 λ)y C Operations that

More information

2 Geometry Solutions

2 Geometry Solutions 2 Geometry Solutions jacques@ucsd.edu Here is give problems and solutions in increasing order of difficulty. 2.1 Easier problems Problem 1. What is the minimum number of hyperplanar slices to make a d-dimensional

More information

COM Optimization for Communications Summary: Convex Sets and Convex Functions

COM Optimization for Communications Summary: Convex Sets and Convex Functions 1 Convex Sets Affine Sets COM524500 Optimization for Communications Summary: Convex Sets and Convex Functions A set C R n is said to be affine if A point x 1, x 2 C = θx 1 + (1 θ)x 2 C, θ R (1) y = k θ

More information

Linear Programming in Small Dimensions

Linear Programming in Small Dimensions Linear Programming in Small Dimensions Lekcija 7 sergio.cabello@fmf.uni-lj.si FMF Univerza v Ljubljani Edited from slides by Antoine Vigneron Outline linear programming, motivation and definition one dimensional

More information

EE/ACM Applications of Convex Optimization in Signal Processing and Communications Lecture 6

EE/ACM Applications of Convex Optimization in Signal Processing and Communications Lecture 6 EE/ACM 150 - Applications of Convex Optimization in Signal Processing and Communications Lecture 6 Andre Tkacenko Signal Processing Research Group Jet Propulsion Laboratory April 19, 2012 Andre Tkacenko

More information

Lecture 19: Convex Non-Smooth Optimization. April 2, 2007

Lecture 19: Convex Non-Smooth Optimization. April 2, 2007 : Convex Non-Smooth Optimization April 2, 2007 Outline Lecture 19 Convex non-smooth problems Examples Subgradients and subdifferentials Subgradient properties Operations with subgradients and subdifferentials

More information

Open and Closed Sets

Open and Closed Sets Open and Closed Sets Definition: A subset S of a metric space (X, d) is open if it contains an open ball about each of its points i.e., if x S : ɛ > 0 : B(x, ɛ) S. (1) Theorem: (O1) and X are open sets.

More information

THREE LECTURES ON BASIC TOPOLOGY. 1. Basic notions.

THREE LECTURES ON BASIC TOPOLOGY. 1. Basic notions. THREE LECTURES ON BASIC TOPOLOGY PHILIP FOTH 1. Basic notions. Let X be a set. To make a topological space out of X, one must specify a collection T of subsets of X, which are said to be open subsets of

More information

Lecture 2: August 29, 2018

Lecture 2: August 29, 2018 10-725/36-725: Convex Optimization Fall 2018 Lecturer: Ryan Tibshirani Lecture 2: August 29, 2018 Scribes: Yingjing Lu, Adam Harley, Ruosong Wang Note: LaTeX template courtesy of UC Berkeley EECS dept.

More information

DM545 Linear and Integer Programming. Lecture 2. The Simplex Method. Marco Chiarandini

DM545 Linear and Integer Programming. Lecture 2. The Simplex Method. Marco Chiarandini DM545 Linear and Integer Programming Lecture 2 The Marco Chiarandini Department of Mathematics & Computer Science University of Southern Denmark Outline 1. 2. 3. 4. Standard Form Basic Feasible Solutions

More information

Intersection Cuts with Infinite Split Rank

Intersection Cuts with Infinite Split Rank Intersection Cuts with Infinite Split Rank Amitabh Basu 1,2, Gérard Cornuéjols 1,3,4 François Margot 1,5 April 2010; revised April 2011; revised October 2011 Abstract We consider mixed integer linear programs

More information

Convex sets and convex functions

Convex sets and convex functions Convex sets and convex functions Convex optimization problems Convex sets and their examples Separating and supporting hyperplanes Projections on convex sets Convex functions, conjugate functions ECE 602,

More information

Introductory Operations Research

Introductory Operations Research Introductory Operations Research Theory and Applications Bearbeitet von Harvir Singh Kasana, Krishna Dev Kumar 1. Auflage 2004. Buch. XI, 581 S. Hardcover ISBN 978 3 540 40138 4 Format (B x L): 15,5 x

More information

Convex sets and convex functions

Convex sets and convex functions Convex sets and convex functions Convex optimization problems Convex sets and their examples Separating and supporting hyperplanes Projections on convex sets Convex functions, conjugate functions ECE 602,

More information

Polar Duality and Farkas Lemma

Polar Duality and Farkas Lemma Lecture 3 Polar Duality and Farkas Lemma October 8th, 2004 Lecturer: Kamal Jain Notes: Daniel Lowd 3.1 Polytope = bounded polyhedron Last lecture, we were attempting to prove the Minkowsky-Weyl Theorem:

More information

Introduction to Modern Control Systems

Introduction to Modern Control Systems Introduction to Modern Control Systems Convex Optimization, Duality and Linear Matrix Inequalities Kostas Margellos University of Oxford AIMS CDT 2016-17 Introduction to Modern Control Systems November

More information

Lecture 2 Convex Sets

Lecture 2 Convex Sets Optimization Theory and Applications Lecture 2 Convex Sets Prof. Chun-Hung Liu Dept. of Electrical and Computer Engineering National Chiao Tung University Fall 2016 2016/9/29 Lecture 2: Convex Sets 1 Outline

More information

Simplex Algorithm in 1 Slide

Simplex Algorithm in 1 Slide Administrivia 1 Canonical form: Simplex Algorithm in 1 Slide If we do pivot in A r,s >0, where c s

More information

Point Cloud Simplification and Processing for Path-Planning. Master s Thesis in Engineering Mathematics and Computational Science DAVID ERIKSSON

Point Cloud Simplification and Processing for Path-Planning. Master s Thesis in Engineering Mathematics and Computational Science DAVID ERIKSSON Point Cloud Simplification and Processing for Path-Planning Master s Thesis in Engineering Mathematics and Computational Science DAVID ERIKSSON Department of Mathematical Sciences Chalmers University of

More information

CS 473: Algorithms. Ruta Mehta. Spring University of Illinois, Urbana-Champaign. Ruta (UIUC) CS473 1 Spring / 29

CS 473: Algorithms. Ruta Mehta. Spring University of Illinois, Urbana-Champaign. Ruta (UIUC) CS473 1 Spring / 29 CS 473: Algorithms Ruta Mehta University of Illinois, Urbana-Champaign Spring 2018 Ruta (UIUC) CS473 1 Spring 2018 1 / 29 CS 473: Algorithms, Spring 2018 Simplex and LP Duality Lecture 19 March 29, 2018

More information

CS599: Convex and Combinatorial Optimization Fall 2013 Lecture 4: Convex Sets. Instructor: Shaddin Dughmi

CS599: Convex and Combinatorial Optimization Fall 2013 Lecture 4: Convex Sets. Instructor: Shaddin Dughmi CS599: Convex and Combinatorial Optimization Fall 2013 Lecture 4: Convex Sets Instructor: Shaddin Dughmi Announcements New room: KAP 158 Today: Convex Sets Mostly from Boyd and Vandenberghe. Read all of

More information

Mathematical and Algorithmic Foundations Linear Programming and Matchings

Mathematical and Algorithmic Foundations Linear Programming and Matchings Adavnced Algorithms Lectures Mathematical and Algorithmic Foundations Linear Programming and Matchings Paul G. Spirakis Department of Computer Science University of Patras and Liverpool Paul G. Spirakis

More information

CMU-Q Lecture 9: Optimization II: Constrained,Unconstrained Optimization Convex optimization. Teacher: Gianni A. Di Caro

CMU-Q Lecture 9: Optimization II: Constrained,Unconstrained Optimization Convex optimization. Teacher: Gianni A. Di Caro CMU-Q 15-381 Lecture 9: Optimization II: Constrained,Unconstrained Optimization Convex optimization Teacher: Gianni A. Di Caro GLOBAL FUNCTION OPTIMIZATION Find the global maximum of the function f x (and

More information

EXTREME POINTS AND AFFINE EQUIVALENCE

EXTREME POINTS AND AFFINE EQUIVALENCE EXTREME POINTS AND AFFINE EQUIVALENCE The purpose of this note is to use the notions of extreme points and affine transformations which are studied in the file affine-convex.pdf to prove that certain standard

More information

MATH 890 HOMEWORK 2 DAVID MEREDITH

MATH 890 HOMEWORK 2 DAVID MEREDITH MATH 890 HOMEWORK 2 DAVID MEREDITH (1) Suppose P and Q are polyhedra. Then P Q is a polyhedron. Moreover if P and Q are polytopes then P Q is a polytope. The facets of P Q are either F Q where F is a facet

More information

A mini-introduction to convexity

A mini-introduction to convexity A mini-introduction to convexity Geir Dahl March 14, 2017 1 Introduction Convexity, or convex analysis, is an area of mathematics where one studies questions related to two basic objects, namely convex

More information

CS 372: Computational Geometry Lecture 10 Linear Programming in Fixed Dimension

CS 372: Computational Geometry Lecture 10 Linear Programming in Fixed Dimension CS 372: Computational Geometry Lecture 10 Linear Programming in Fixed Dimension Antoine Vigneron King Abdullah University of Science and Technology November 7, 2012 Antoine Vigneron (KAUST) CS 372 Lecture

More information

11 Linear Programming

11 Linear Programming 11 Linear Programming 11.1 Definition and Importance The final topic in this course is Linear Programming. We say that a problem is an instance of linear programming when it can be effectively expressed

More information

Lecture 15: The subspace topology, Closed sets

Lecture 15: The subspace topology, Closed sets Lecture 15: The subspace topology, Closed sets 1 The Subspace Topology Definition 1.1. Let (X, T) be a topological space with topology T. subset of X, the collection If Y is a T Y = {Y U U T} is a topology

More information

Lecture 3. Corner Polyhedron, Intersection Cuts, Maximal Lattice-Free Convex Sets. Tepper School of Business Carnegie Mellon University, Pittsburgh

Lecture 3. Corner Polyhedron, Intersection Cuts, Maximal Lattice-Free Convex Sets. Tepper School of Business Carnegie Mellon University, Pittsburgh Lecture 3 Corner Polyhedron, Intersection Cuts, Maximal Lattice-Free Convex Sets Gérard Cornuéjols Tepper School of Business Carnegie Mellon University, Pittsburgh January 2016 Mixed Integer Linear Programming

More information

Aspects of Convex, Nonconvex, and Geometric Optimization (Lecture 1) Suvrit Sra Massachusetts Institute of Technology

Aspects of Convex, Nonconvex, and Geometric Optimization (Lecture 1) Suvrit Sra Massachusetts Institute of Technology Aspects of Convex, Nonconvex, and Geometric Optimization (Lecture 1) Suvrit Sra Massachusetts Institute of Technology Hausdorff Institute for Mathematics (HIM) Trimester: Mathematics of Signal Processing

More information

Lecture 4: Rational IPs, Polyhedron, Decomposition Theorem

Lecture 4: Rational IPs, Polyhedron, Decomposition Theorem IE 5: Integer Programming, Spring 29 24 Jan, 29 Lecture 4: Rational IPs, Polyhedron, Decomposition Theorem Lecturer: Karthik Chandrasekaran Scribe: Setareh Taki Disclaimer: These notes have not been subjected

More information

Dubna 2018: lines on cubic surfaces

Dubna 2018: lines on cubic surfaces Dubna 2018: lines on cubic surfaces Ivan Cheltsov 20th July 2018 Lecture 1: projective plane Complex plane Definition A line in C 2 is a subset that is given by ax + by + c = 0 for some complex numbers

More information

Section 5 Convex Optimisation 1. W. Dai (IC) EE4.66 Data Proc. Convex Optimisation page 5-1

Section 5 Convex Optimisation 1. W. Dai (IC) EE4.66 Data Proc. Convex Optimisation page 5-1 Section 5 Convex Optimisation 1 W. Dai (IC) EE4.66 Data Proc. Convex Optimisation 1 2018 page 5-1 Convex Combination Denition 5.1 A convex combination is a linear combination of points where all coecients

More information

Mathematical Programming and Research Methods (Part II)

Mathematical Programming and Research Methods (Part II) Mathematical Programming and Research Methods (Part II) 4. Convexity and Optimization Massimiliano Pontil (based on previous lecture by Andreas Argyriou) 1 Today s Plan Convex sets and functions Types

More information

LP Geometry: outline. A general LP. minimize x c T x s.t. a T i. x b i, i 2 M 1 a T i x = b i, i 2 M 3 x j 0, j 2 N 1. where

LP Geometry: outline. A general LP. minimize x c T x s.t. a T i. x b i, i 2 M 1 a T i x = b i, i 2 M 3 x j 0, j 2 N 1. where LP Geometry: outline I Polyhedra I Extreme points, vertices, basic feasible solutions I Degeneracy I Existence of extreme points I Optimality of extreme points IOE 610: LP II, Fall 2013 Geometry of Linear

More information

1 Linear Programming. 1.1 Optimizion problems and convex polytopes 1 LINEAR PROGRAMMING

1 Linear Programming. 1.1 Optimizion problems and convex polytopes 1 LINEAR PROGRAMMING 1 LINEAR PROGRAMMING 1 Linear Programming Now, we will talk a little bit about Linear Programming. We say that a problem is an instance of linear programming when it can be effectively expressed in the

More information

Convexity. 1 X i is convex. = b is a hyperplane in R n, and is denoted H(p, b) i.e.,

Convexity. 1 X i is convex. = b is a hyperplane in R n, and is denoted H(p, b) i.e., Convexity We ll assume throughout, without always saying so, that we re in the finite-dimensional Euclidean vector space R n, although sometimes, for statements that hold in any vector space, we ll say

More information

Lecture 5: Properties of convex sets

Lecture 5: Properties of convex sets Lecture 5: Properties of convex sets Rajat Mittal IIT Kanpur This week we will see properties of convex sets. These properties make convex sets special and are the reason why convex optimization problems

More information

AMS : Combinatorial Optimization Homework Problems - Week V

AMS : Combinatorial Optimization Homework Problems - Week V AMS 553.766: Combinatorial Optimization Homework Problems - Week V For the following problems, A R m n will be m n matrices, and b R m. An affine subspace is the set of solutions to a a system of linear

More information

Lecture: Convex Sets

Lecture: Convex Sets /24 Lecture: Convex Sets http://bicmr.pku.edu.cn/~wenzw/opt-27-fall.html Acknowledgement: this slides is based on Prof. Lieven Vandenberghe s lecture notes Introduction 2/24 affine and convex sets some

More information

Walheer Barnabé. Topics in Mathematics Practical Session 2 - Topology & Convex

Walheer Barnabé. Topics in Mathematics Practical Session 2 - Topology & Convex Topics in Mathematics Practical Session 2 - Topology & Convex Sets Outline (i) Set membership and set operations (ii) Closed and open balls/sets (iii) Points (iv) Sets (v) Convex Sets Set Membership and

More information

In this chapter we introduce some of the basic concepts that will be useful for the study of integer programming problems.

In this chapter we introduce some of the basic concepts that will be useful for the study of integer programming problems. 2 Basics In this chapter we introduce some of the basic concepts that will be useful for the study of integer programming problems. 2.1 Notation Let A R m n be a matrix with row index set M = {1,...,m}

More information

Linear programming and duality theory

Linear programming and duality theory Linear programming and duality theory Complements of Operations Research Giovanni Righini Linear Programming (LP) A linear program is defined by linear constraints, a linear objective function. Its variables

More information

Polytopes Course Notes

Polytopes Course Notes Polytopes Course Notes Carl W. Lee Department of Mathematics University of Kentucky Lexington, KY 40506 lee@ms.uky.edu Fall 2013 i Contents 1 Polytopes 1 1.1 Convex Combinations and V-Polytopes.....................

More information

Graph Connectivity in Sparse Subspace Clustering

Graph Connectivity in Sparse Subspace Clustering www.nicta.com.au From imagination to impact Graph Connectivity in Sparse Subspace Clustering Behrooz Nasihatkon 24 March 2011 Outline 1 Subspace Clustering 2 Sparse Subspace Clustering 3 Graph Connectivity

More information

Topology 550A Homework 3, Week 3 (Corrections: February 22, 2012)

Topology 550A Homework 3, Week 3 (Corrections: February 22, 2012) Topology 550A Homework 3, Week 3 (Corrections: February 22, 2012) Michael Tagare De Guzman January 31, 2012 4A. The Sorgenfrey Line The following material concerns the Sorgenfrey line, E, introduced in

More information

College of Computer & Information Science Fall 2007 Northeastern University 14 September 2007

College of Computer & Information Science Fall 2007 Northeastern University 14 September 2007 College of Computer & Information Science Fall 2007 Northeastern University 14 September 2007 CS G399: Algorithmic Power Tools I Scribe: Eric Robinson Lecture Outline: Linear Programming: Vertex Definitions

More information

Interval-Vector Polytopes

Interval-Vector Polytopes Interval-Vector Polytopes Jessica De Silva Gabriel Dorfsman-Hopkins California State University, Stanislaus Dartmouth College Joseph Pruitt California State University, Long Beach July 28, 2012 Abstract

More information

Three Dimensional Geometry. Linear Programming

Three Dimensional Geometry. Linear Programming Three Dimensional Geometry Linear Programming A plane is determined uniquely if any one of the following is known: The normal to the plane and its distance from the origin is given, i.e. equation of a

More information

Chapter 8. Voronoi Diagrams. 8.1 Post Oce Problem

Chapter 8. Voronoi Diagrams. 8.1 Post Oce Problem Chapter 8 Voronoi Diagrams 8.1 Post Oce Problem Suppose there are n post oces p 1,... p n in a city. Someone who is located at a position q within the city would like to know which post oce is closest

More information

Convexity Theory and Gradient Methods

Convexity Theory and Gradient Methods Convexity Theory and Gradient Methods Angelia Nedić angelia@illinois.edu ISE Department and Coordinated Science Laboratory University of Illinois at Urbana-Champaign Outline Convex Functions Optimality

More information

Lecture 2: August 31

Lecture 2: August 31 10-725/36-725: Convex Optimization Fall 2016 Lecture 2: August 31 Lecturer: Lecturer: Ryan Tibshirani Scribes: Scribes: Lidan Mu, Simon Du, Binxuan Huang 2.1 Review A convex optimization problem is of

More information

Applied Lagrange Duality for Constrained Optimization

Applied Lagrange Duality for Constrained Optimization Applied Lagrange Duality for Constrained Optimization Robert M. Freund February 10, 2004 c 2004 Massachusetts Institute of Technology. 1 1 Overview The Practical Importance of Duality Review of Convexity

More information

L-CONVEX-CONCAVE SETS IN REAL PROJECTIVE SPACE AND L-DUALITY

L-CONVEX-CONCAVE SETS IN REAL PROJECTIVE SPACE AND L-DUALITY MOSCOW MATHEMATICAL JOURNAL Volume 3, Number 3, July September 2003, Pages 1013 1037 L-CONVEX-CONCAVE SETS IN REAL PROJECTIVE SPACE AND L-DUALITY A. KHOVANSKII AND D. NOVIKOV Dedicated to Vladimir Igorevich

More information

IE 5531: Engineering Optimization I

IE 5531: Engineering Optimization I IE 5531: Engineering Optimization I Lecture 3: Linear Programming, Continued Prof. John Gunnar Carlsson September 15, 2010 Prof. John Gunnar Carlsson IE 5531: Engineering Optimization I September 15, 2010

More information

LECTURE 7 LECTURE OUTLINE. Review of hyperplane separation Nonvertical hyperplanes Convex conjugate functions Conjugacy theorem Examples

LECTURE 7 LECTURE OUTLINE. Review of hyperplane separation Nonvertical hyperplanes Convex conjugate functions Conjugacy theorem Examples LECTURE 7 LECTURE OUTLINE Review of hyperplane separation Nonvertical hyperplanes Convex conjugate functions Conjugacy theorem Examples Reading: Section 1.5, 1.6 All figures are courtesy of Athena Scientific,

More information

Search and Intersection. O Rourke, Chapter 7 de Berg et al., Chapter 11

Search and Intersection. O Rourke, Chapter 7 de Berg et al., Chapter 11 Search and Intersection O Rourke, Chapter 7 de Berg et al., Chapter 11 Announcements Assignment 3 web-page has been updated: Additional extra credit Hints for managing a dynamic half-edge representation

More information

AM 221: Advanced Optimization Spring 2016

AM 221: Advanced Optimization Spring 2016 AM 221: Advanced Optimization Spring 2016 Prof. Yaron Singer Lecture 2 Wednesday, January 27th 1 Overview In our previous lecture we discussed several applications of optimization, introduced basic terminology,

More information

ORIE 6300 Mathematical Programming I September 2, Lecture 3

ORIE 6300 Mathematical Programming I September 2, Lecture 3 ORIE 6300 Mathematical Programming I September 2, 2014 Lecturer: David P. Williamson Lecture 3 Scribe: Divya Singhvi Last time we discussed how to take dual of an LP in two different ways. Today we will

More information