Notes on Minimum Cuts and Modular Functions

Size: px
Start display at page:

Download "Notes on Minimum Cuts and Modular Functions"

Transcription

1 Notes on Minimum Cuts and Modular Functions 1 Introduction The following are my notes on Cunningham s paper [1]. Given a submodular function f and a set S, submodular minimisation is the problem of finding A S for which f(a) is minimum. There exists continuous optimization algorithms such as ellipsoid algorithm and min-norm point algorithm for solving the minimisation problem, which are weakly polynomial (that is, the order depends on the minimum value of f(a) ) and are slow in practice. Cut functions are a special class of submodular functions which can be represented as a graph. The minimum st-cut algorithm on this graph gives the the minimum of the cut function. Formally, let S = {1, 2,..., n}. The graph consists of two special vertices {s, t}. Let us define a set function The submodular function is f(a) = u(δ(a)) where δ(a) denotes {(v i, v j ) E, such that v i A {s}, and v j / A {s}} (that is, the set of arcs coming out from the set {A {s}}. Property 1. Cut functions are submodular. Proof. Let S = {1, 2,..., N}. The graph consists of the vertex set V = {v 1,..., v N } {s, t} and the edge set defined over the vertex set. Consider any one vertex v x. Without loss of generality, let there be n outgoing edges e 1, e 2... e n from v x to v 1, v 2,..., v n. Using equation?? f vx (X) = f vx (X {v 1... v n }) = n j=1,j / X f vx (X) is clearly non-increasing with respect to X. The paper can be divided as considering three problems: 1. Graph Construction of a Cut Function e j (1) 2. Equivalence of min st-cut of a submodular function to minimising a modular function 3. Properties of matroid polyhedra We will consider only the first two parts here. 1

2 1.1 Graph Construction of a Cut Function Theorem 1. If a submodular function is know to be a cut function, then a graph can be constructed in polynomial (O( S 2 )) time. The statement implies that the minimum of the submodular function can then be obtained solving minimum st-cut on the graph for which strongly polynomial algorithms exist. Property 2. Cut functions have the following remarkable property. A, B, C S, Given f(a B C) = f(a B)+f(B C)+f(A C) f(a) f(b) f(c) f(φ) (2) Proof. Let us first consider the simplest case, where S = {a, b, c} and A = {a}, B = {b}, C = {c}. In this case, A, B, C form a partition of S. For cut functions, f(s) = f(φ) = 0. Also, we have f({a, b}) = e ac + e bc f({b, c}) = e ba + e ca f({c, a}) = e cb + e ab f({a}) = e ab + e ac Using equations 3, we can write the R.H.S as f({b}) = e ba + e bc f({c}) = e ca + e cb (3) f({a, b}) + f({b, c}) + f({c, a}) f({a}) f({b}) f({c}) + f(φ) = 0 (4) Since L.H.S also equals 0, the proof is complete. The same approach can be taken for the case S = {a, b, c, d} and A = {a}, B = {b}, C = {c}, so that A, B, C do not partition S. A more general case is one where A, B, C are sets of vertices. Given A S, f(a) can be obtained only by calling an oracle which returns the value. Equation 2 suggests that for a cut function, if one obtains the function value for all sets of cardinality 0, 1 and 2, then the full f specification is known using the inductive relation and no further oracle calls are required. In fact, exactly 1 + S + S C 2 oracle calls are necessary (that is, O( S 2 ). Given a cut function, [1] gives the algorithm for graph construction in O( S 2 ) time. Note that, the graph representation of a cut function is not unique and the construction specified here is a specific instance of such graphs. 2

3 1.1.1 Graph Construction We would like to construct a directed graph G = (V, E) such that every cut on the graph corresponds to a set and equals the value of the submodular function for that set. Let V = {s, t} {v 1, v,..., v n } where v i corresponds to i-th element of S ( S = n). s, t denote the source and sink terminals respectively. Let us denote any two vertices as v, w and the capacity of the edge v w as u vw. Elements of E are one of three types: 1. s v edges (source to vertex edge) Select an arbitrary vertex x in V. Assign u sx = f(φ) and u sv = 0 v S {x} The above ensures that u(δ({s})) = f(φ) 2. v w edges (vertex to vertex edge) u vw = u wv = 1 (f({v}) + f({w}) f({v, w}) f(φ)) 2 Since f is submodular, u vw is positive. The reason for selecting constant as 1/2 will come clear later. 3. v t edges (vertex to sink edge) u vt = f({v}) x S {v} u sx x S {v} By construction, the cut function equals f for A = 0, 1. We now show that the equality also holds for A = 2. Consider A = {v, w}. u vx u(δ({v, w} {s})) = u(δ({r, v})) + u(δ({r, w})) u vw u wv u(δ(r)) = f({v}) + f({w}) 2 1/2 (f({v}) + f({w}) f({v, w}) f(φ)) f(φ) = f({v, w}) Because f is a cut function here, it follows that it follows the relation 2. For any A such that A > 2, one can use the relation 2 to obtain the value from sets of cardinality 2 or smaller. Not clear how f(a) = u(δ((a {r}))) for all A. One way to think about submodular and cut functions is as follows: submodularity suggests that f values are not random, but obey the diminishing returns property. The property of being cut function suggests that there is redundancy in the values of f to the extent, that only polynomial number of entries are sufficient to determine the exponentially-sized f. As an aside, note that it is NP-hard to determine whether or not a given f is submodular, since we need to evaluate property of?? for all 2 S values of f. Theorem 2. Determining whether or not a submodular function is a cut function is NP-hard. 3

4 The proof of this statement proceeds by considering a cut function (and hence submodular). From this function, another function is derived by decrementing the value of one entry for a set A of cardinality greater than 2, the remaining entries being the same. By construction, this function is not cut function (the property 2 is violated for the changed entry), but it still is submodular (how?). To discover that the derived function is not cut function, there is no alternative but to check whether all entries for set of cardinality greater than 2, satisfy relation Min Cut Problem and Modular Function Minimisation over a Lattice [1] claims that the minimum cut problem is equivalent to minimising a modular function over a lattice (lattice referred to as ring in the paper). Recall that a modular function has the property: The above implies f(a B) + f(a B) = f(a) + f(b) (5) f(a) = f(φ) + i A(f({i}) f(φ)) (6) Let A = {a} and B = {b} in equation 5. This gives f({a, b}) + f(φ) = f({a} + f({b}) f({a, b}) = f(φ) + (f({a} f(φ)) + (f({b}) f(φ)) Using above, the modular value property can be proved inductively. Let b 0 = f(φ) and b i = f(i) f(φ). Modular function minimisation over 2 S is trivial: select A S such that {i S, b i < 0}. Modular function over a lattice (a subset of 2 S closed under union and intersection) is not trivial, but is easy as shown below. A family of subsets defined on a set S is another name for a collection of subsets of S - that is a subset of 2 S. When the meaning is clear from context, we will refer a family of subsets on S as just a family. Definition 1. A family F is said to be a lattice or a ring, if it is closed under union and intersection. Formally, A, B F = A B F and A B F (7) S: For instance, let S = {a, b, c, d}. The following are some lattices defined on 4

5 F = {φ, {a}, {b}, {a, b}} F = {φ, {a}, {c}, {a, c}} F = {φ, {a}, {b}, {c}, {a, b}, {a, c}, {b, c}, {a, b, c}} Definition 2. A closure of a graph G = (V, E) is a set A V, such that δ(a) = φ. In other words, the above definition says that a closure is a set A V, such that there is no edge from A to V A in G. Clearly A = φ and A = V are closures. The following propositions hold true: Proposition 1. The family of all closures of a directed graph G = (V, E) forms a proper ring family over S = V. Proof. For any A, B S, δ(a B) and δ(a B) is in δ(a) or δ(b). If A, B are closures, δ(a) = 0 and δ(b) = 0. Hence, δ(a B) = 0 and δ(a B) = 0. Thus, A B and A B are also closures. Also, φ and V are closures. So the ring family is proper. Proposition 2. Given a proper ring family F, a graph G can be constructed such that every element F F is a closure in G. The graph construction proceeds by taking a vertex for each element of set, that is, V = S. A directed edge is drawn for vertex i to vertex j, if occurrence of i in any set of F implies the occurrence of j in that set. Hence, (u, v) E if u F = v F. By construction, for every v F and for every w / F, (u, w) / E. Hence, F is a closure of G. Proposition 3. Each closure F in the above graph G belongs to F. The proof proceeds by showing that F is the intersection of sets which are guaranteed to be in F and hence F is in F. Formally, for u F and v / F, there should be a set F uv F such that u F uv and v / F uv (otherwise (u, v) E). Let F v = (F uv, u F ). Since F v is union of sets in F, F v is also inf. F = (F v, v / F ) and hence F is in F. (Note that F is not a proper subset of (F v, v / F ), since we take intersection over all elements not in F ). To construct the above graph, we need to make use of an oracle which answers for each i, j S, Does there exist some F F, such that i F and j / F?. If yes, we do not draw an arc between i and j, else we draw an arc. 5

6 1.2.1 Modular Minimisation over Lattice as Min Cut Modular Minimisation over Lattice as Min Cut Given a modular function defined on a ring family, we construct a graph such that modular function minimisation corresponds to the minimum weight closure problem on the graph. The idea is to take the directed graph G constructed above and assign weights to the nodes. First, find strongly connected components in G (corresponds to A i ) (O(n)). In the corresponding DAG, sort them topologically (O(n + m) = O(n 2 ). Find a path from source to sink in DAG. Assign weights to nodes inductively starting in reverse from sink. Min Weight Closure as Min Cut Due to the result of Picard, the minimum weight closure problem can be translated to a minimum st-cut problem on an appropriately constructed graph. Given a graph G on which min weight closure is to be found, we construct a graph G as follows. G and G have the same set of vertices. G has in addition the two terminal vertices {s, t} - source and sink respectively. If there is an edge in G, we draw the same edge in G with infinite capacity. For each v S, if b v < 0, we draw arc (s, v) with capacity b v. Else, if b v > 0, we draw arc (v, t) with capacity b v. A closure F in G induces a finite capacity st-cut in G. The cut consists of arcs leaving F {r}. The value of capacity is: {bv : v F, b v > 0} + { b v : v V F, b v < 0} = {b v : v F, b v > 0} {b v : v V F, b v < 0} = {b v : v F, b v > 0} {b v : v V F, b v < 0} + {b v : v F, b v < 0} {b v : v F, b v < 0} = {b v : v F } {b v : v V, b v < 0} Hence, the value of each finite capacity cut equals the closure weight plus a positive constant. Min cut on G will give the min weight closure on G with a constant added Min Cut as Modular Minimisation over Lattice Also, given an st-graph G, one can define a ring family F and a modular function defined over it such that the minimiser of the modular function also gives the minimiser of the st-cut problem. Given a graph G = (V, E), we consider S = V E. Let the family F be defined as {V E : {s} V V {t} and E γ(v )} where γ(v ) is the set of all edges with both endpoints in V. First we verify that F is a ring family. Let A, B F. First we show A B F. 6

7 A B = V A E A V B E B Clearly, {r} V A V B V {t} Also, γ(v A) γ(v B) γ(v A V B) Since E A E B γ(v A) γ(v B) = E A E B γ(v A V B) Now we show A B F. A B = (V A E A) (V B E B) = (V A V B) (E A E B) Clearly, {r} V A V B V {t} Also, γ(v A) γ(v B) = γ(v A V B)( draw and check ) Since E A E B γ(v A) γ(v B) = E A E B γ(v A V B) The set function value is defined as f(v E ) = u(δ(v) : v V ) u(e ). It is modular (sum of function of individual elements). For minimum value of f, we can assume E = γ(v ), since u(e) > 0 e E. For the minimiser A = V γ(v ) of F, f(a) = u(δ(v )). Hence, the minimiser of f gives the min cut minimiser exactly. References [1] William H Cunningham. Minimum cuts, modular functions, and matroid polyhedra. Networks, 15(2): ,

8 Matroid Intersection

8 Matroid Intersection 8 Matroid Intersection 8.1 Definition and examples 8.2 Matroid Intersection Algorithm 8.1 Definitions Given two matroids M 1 = (X, I 1 ) and M 2 = (X, I 2 ) on the same set X, their intersection is M 1

More information

Graphs and Network Flows IE411. Lecture 21. Dr. Ted Ralphs

Graphs and Network Flows IE411. Lecture 21. Dr. Ted Ralphs Graphs and Network Flows IE411 Lecture 21 Dr. Ted Ralphs IE411 Lecture 21 1 Combinatorial Optimization and Network Flows In general, most combinatorial optimization and integer programming problems are

More information

Lecture 2. 1 Introduction. 2 The Set Cover Problem. COMPSCI 632: Approximation Algorithms August 30, 2017

Lecture 2. 1 Introduction. 2 The Set Cover Problem. COMPSCI 632: Approximation Algorithms August 30, 2017 COMPSCI 632: Approximation Algorithms August 30, 2017 Lecturer: Debmalya Panigrahi Lecture 2 Scribe: Nat Kell 1 Introduction In this lecture, we examine a variety of problems for which we give greedy approximation

More information

CPSC 536N: Randomized Algorithms Term 2. Lecture 10

CPSC 536N: Randomized Algorithms Term 2. Lecture 10 CPSC 536N: Randomized Algorithms 011-1 Term Prof. Nick Harvey Lecture 10 University of British Columbia In the first lecture we discussed the Max Cut problem, which is NP-complete, and we presented a very

More information

6. Lecture notes on matroid intersection

6. Lecture notes on matroid intersection Massachusetts Institute of Technology 18.453: Combinatorial Optimization Michel X. Goemans May 2, 2017 6. Lecture notes on matroid intersection One nice feature about matroids is that a simple greedy algorithm

More information

Lecture Orientations, Directed Cuts and Submodular Flows

Lecture Orientations, Directed Cuts and Submodular Flows 18.997 Topics in Combinatorial Optimization April 15th, 2004 Lecture 18 Lecturer: Michel X. Goemans Scribe: Nick Harvey 18 Orientations, irected Cuts and Submodular Flows In this lecture, we will introduce

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

Adjacent: Two distinct vertices u, v are adjacent if there is an edge with ends u, v. In this case we let uv denote such an edge.

Adjacent: Two distinct vertices u, v are adjacent if there is an edge with ends u, v. In this case we let uv denote such an edge. 1 Graph Basics What is a graph? Graph: a graph G consists of a set of vertices, denoted V (G), a set of edges, denoted E(G), and a relation called incidence so that each edge is incident with either one

More information

Rigidity, connectivity and graph decompositions

Rigidity, connectivity and graph decompositions First Prev Next Last Rigidity, connectivity and graph decompositions Brigitte Servatius Herman Servatius Worcester Polytechnic Institute Page 1 of 100 First Prev Next Last Page 2 of 100 We say that a framework

More information

Solution for Homework set 3

Solution for Homework set 3 TTIC 300 and CMSC 37000 Algorithms Winter 07 Solution for Homework set 3 Question (0 points) We are given a directed graph G = (V, E), with two special vertices s and t, and non-negative integral capacities

More information

CS 598CSC: Approximation Algorithms Lecture date: March 2, 2011 Instructor: Chandra Chekuri

CS 598CSC: Approximation Algorithms Lecture date: March 2, 2011 Instructor: Chandra Chekuri CS 598CSC: Approximation Algorithms Lecture date: March, 011 Instructor: Chandra Chekuri Scribe: CC Local search is a powerful and widely used heuristic method (with various extensions). In this lecture

More information

Important separators and parameterized algorithms

Important separators and parameterized algorithms Important separators and parameterized algorithms Dániel Marx 1 1 Institute for Computer Science and Control, Hungarian Academy of Sciences (MTA SZTAKI) Budapest, Hungary School on Parameterized Algorithms

More information

5. Lecture notes on matroid intersection

5. Lecture notes on matroid intersection Massachusetts Institute of Technology Handout 14 18.433: Combinatorial Optimization April 1st, 2009 Michel X. Goemans 5. Lecture notes on matroid intersection One nice feature about matroids is that a

More information

Binary Relations McGraw-Hill Education

Binary Relations McGraw-Hill Education Binary Relations A binary relation R from a set A to a set B is a subset of A X B Example: Let A = {0,1,2} and B = {a,b} {(0, a), (0, b), (1,a), (2, b)} is a relation from A to B. We can also represent

More information

Finding Strongly Connected Components

Finding Strongly Connected Components Yufei Tao ITEE University of Queensland We just can t get enough of the beautiful algorithm of DFS! In this lecture, we will use it to solve a problem finding strongly connected components that seems to

More information

Lecture : Topological Space

Lecture : Topological Space Example of Lecture : Dr. Department of Mathematics Lovely Professional University Punjab, India October 18, 2014 Outline Example of 1 2 3 Example of 4 5 6 Example of I Topological spaces and continuous

More information

1 Connected components in undirected graphs

1 Connected components in undirected graphs Lecture 10 Connected components of undirected and directed graphs Scribe: Luke Johnston (2016) and Mary Wootters (2017) Date: October 25, 2017 Much of the following notes were taken from Tim Roughgarden

More information

1 Linear programming relaxation

1 Linear programming relaxation Cornell University, Fall 2010 CS 6820: Algorithms Lecture notes: Primal-dual min-cost bipartite matching August 27 30 1 Linear programming relaxation Recall that in the bipartite minimum-cost perfect matching

More information

CS261: A Second Course in Algorithms Lecture #16: The Traveling Salesman Problem

CS261: A Second Course in Algorithms Lecture #16: The Traveling Salesman Problem CS61: A Second Course in Algorithms Lecture #16: The Traveling Salesman Problem Tim Roughgarden February 5, 016 1 The Traveling Salesman Problem (TSP) In this lecture we study a famous computational problem,

More information

9.5 Equivalence Relations

9.5 Equivalence Relations 9.5 Equivalence Relations You know from your early study of fractions that each fraction has many equivalent forms. For example, 2, 2 4, 3 6, 2, 3 6, 5 30,... are all different ways to represent the same

More information

Introduction to Graph Theory

Introduction to Graph Theory Introduction to Graph Theory Tandy Warnow January 20, 2017 Graphs Tandy Warnow Graphs A graph G = (V, E) is an object that contains a vertex set V and an edge set E. We also write V (G) to denote the vertex

More information

Matching Algorithms. Proof. If a bipartite graph has a perfect matching, then it is easy to see that the right hand side is a necessary condition.

Matching Algorithms. Proof. If a bipartite graph has a perfect matching, then it is easy to see that the right hand side is a necessary condition. 18.433 Combinatorial Optimization Matching Algorithms September 9,14,16 Lecturer: Santosh Vempala Given a graph G = (V, E), a matching M is a set of edges with the property that no two of the edges have

More information

A GRAPH FROM THE VIEWPOINT OF ALGEBRAIC TOPOLOGY

A GRAPH FROM THE VIEWPOINT OF ALGEBRAIC TOPOLOGY A GRAPH FROM THE VIEWPOINT OF ALGEBRAIC TOPOLOGY KARL L. STRATOS Abstract. The conventional method of describing a graph as a pair (V, E), where V and E repectively denote the sets of vertices and edges,

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

Fundamental Properties of Graphs

Fundamental Properties of Graphs Chapter three In many real-life situations we need to know how robust a graph that represents a certain network is, how edges or vertices can be removed without completely destroying the overall connectivity,

More information

Maximum flows & Maximum Matchings

Maximum flows & Maximum Matchings Chapter 9 Maximum flows & Maximum Matchings This chapter analyzes flows and matchings. We will define flows and maximum flows and present an algorithm that solves the maximum flow problem. Then matchings

More information

Massachusetts Institute of Technology Department of Electrical Engineering and Computer Science Algorithms For Inference Fall 2014

Massachusetts Institute of Technology Department of Electrical Engineering and Computer Science Algorithms For Inference Fall 2014 Suggested Reading: Massachusetts Institute of Technology Department of Electrical Engineering and Computer Science 6.438 Algorithms For Inference Fall 2014 Probabilistic Modelling and Reasoning: The Junction

More information

On 2-Subcolourings of Chordal Graphs

On 2-Subcolourings of Chordal Graphs On 2-Subcolourings of Chordal Graphs Juraj Stacho School of Computing Science, Simon Fraser University 8888 University Drive, Burnaby, B.C., Canada V5A 1S6 jstacho@cs.sfu.ca Abstract. A 2-subcolouring

More information

Graph Theory. Part of Texas Counties.

Graph Theory. Part of Texas Counties. Graph Theory Part of Texas Counties. We would like to visit each of the above counties, crossing each county only once, starting from Harris county. Is this possible? This problem can be modeled as a graph.

More information

Planar Graphs. 1 Graphs and maps. 1.1 Planarity and duality

Planar Graphs. 1 Graphs and maps. 1.1 Planarity and duality Planar Graphs In the first half of this book, we consider mostly planar graphs and their geometric representations, mostly in the plane. We start with a survey of basic results on planar graphs. This chapter

More information

Lecture 17: Continuous Functions

Lecture 17: Continuous Functions Lecture 17: Continuous Functions 1 Continuous Functions Let (X, T X ) and (Y, T Y ) be topological spaces. Definition 1.1 (Continuous Function). A function f : X Y is said to be continuous if the inverse

More information

MA651 Topology. Lecture 4. Topological spaces 2

MA651 Topology. Lecture 4. Topological spaces 2 MA651 Topology. Lecture 4. Topological spaces 2 This text is based on the following books: Linear Algebra and Analysis by Marc Zamansky Topology by James Dugundgji Fundamental concepts of topology by Peter

More information

Lecture 22 Tuesday, April 10

Lecture 22 Tuesday, April 10 CIS 160 - Spring 2018 (instructor Val Tannen) Lecture 22 Tuesday, April 10 GRAPH THEORY Directed Graphs Directed graphs (a.k.a. digraphs) are an important mathematical modeling tool in Computer Science,

More information

Recognizing Interval Bigraphs by Forbidden Patterns

Recognizing Interval Bigraphs by Forbidden Patterns Recognizing Interval Bigraphs by Forbidden Patterns Arash Rafiey Simon Fraser University, Vancouver, Canada, and Indiana State University, IN, USA arashr@sfu.ca, arash.rafiey@indstate.edu Abstract Let

More information

Module 11. Directed Graphs. Contents

Module 11. Directed Graphs. Contents Module 11 Directed Graphs Contents 11.1 Basic concepts......................... 256 Underlying graph of a digraph................ 257 Out-degrees and in-degrees.................. 258 Isomorphism..........................

More information

arxiv: v1 [math.co] 3 Apr 2016

arxiv: v1 [math.co] 3 Apr 2016 A note on extremal results on directed acyclic graphs arxiv:1604.0061v1 [math.co] 3 Apr 016 A. Martínez-Pérez, L. Montejano and D. Oliveros April 5, 016 Abstract The family of Directed Acyclic Graphs as

More information

Theorem 2.9: nearest addition algorithm

Theorem 2.9: nearest addition algorithm There are severe limits on our ability to compute near-optimal tours It is NP-complete to decide whether a given undirected =(,)has a Hamiltonian cycle An approximation algorithm for the TSP can be used

More information

Section 3.1: Nonseparable Graphs Cut vertex of a connected graph G: A vertex x G such that G x is not connected. Theorem 3.1, p. 57: Every connected

Section 3.1: Nonseparable Graphs Cut vertex of a connected graph G: A vertex x G such that G x is not connected. Theorem 3.1, p. 57: Every connected Section 3.1: Nonseparable Graphs Cut vertex of a connected graph G: A vertex x G such that G x is not connected. Theorem 3.1, p. 57: Every connected graph G with at least 2 vertices contains at least 2

More information

3 No-Wait Job Shops with Variable Processing Times

3 No-Wait Job Shops with Variable Processing Times 3 No-Wait Job Shops with Variable Processing Times In this chapter we assume that, on top of the classical no-wait job shop setting, we are given a set of processing times for each operation. We may select

More information

CMPSCI 311: Introduction to Algorithms Practice Final Exam

CMPSCI 311: Introduction to Algorithms Practice Final Exam CMPSCI 311: Introduction to Algorithms Practice Final Exam Name: ID: Instructions: Answer the questions directly on the exam pages. Show all your work for each question. Providing more detail including

More information

Greedy Algorithms 1. For large values of d, brute force search is not feasible because there are 2 d

Greedy Algorithms 1. For large values of d, brute force search is not feasible because there are 2 d Greedy Algorithms 1 Simple Knapsack Problem Greedy Algorithms form an important class of algorithmic techniques. We illustrate the idea by applying it to a simplified version of the Knapsack Problem. Informally,

More information

K 4 C 5. Figure 4.5: Some well known family of graphs

K 4 C 5. Figure 4.5: Some well known family of graphs 08 CHAPTER. TOPICS IN CLASSICAL GRAPH THEORY K, K K K, K K, K K, K C C C C 6 6 P P P P P. Graph Operations Figure.: Some well known family of graphs A graph Y = (V,E ) is said to be a subgraph of a graph

More information

A graph is finite if its vertex set and edge set are finite. We call a graph with just one vertex trivial and all other graphs nontrivial.

A graph is finite if its vertex set and edge set are finite. We call a graph with just one vertex trivial and all other graphs nontrivial. 2301-670 Graph theory 1.1 What is a graph? 1 st semester 2550 1 1.1. What is a graph? 1.1.2. Definition. A graph G is a triple (V(G), E(G), ψ G ) consisting of V(G) of vertices, a set E(G), disjoint from

More information

Slides for Faculty Oxford University Press All rights reserved.

Slides for Faculty Oxford University Press All rights reserved. Oxford University Press 2013 Slides for Faculty Assistance Preliminaries Author: Vivek Kulkarni vivek_kulkarni@yahoo.com Outline Following topics are covered in the slides: Basic concepts, namely, symbols,

More information

Treewidth and graph minors

Treewidth and graph minors Treewidth and graph minors Lectures 9 and 10, December 29, 2011, January 5, 2012 We shall touch upon the theory of Graph Minors by Robertson and Seymour. This theory gives a very general condition under

More information

Math 443/543 Graph Theory Notes

Math 443/543 Graph Theory Notes Math 443/543 Graph Theory Notes David Glickenstein September 8, 2014 1 Introduction We will begin by considering several problems which may be solved using graphs, directed graphs (digraphs), and networks.

More information

BAR-MAGNET POLYHEDRA AND NS-ORIENTATIONS OF MAPS

BAR-MAGNET POLYHEDRA AND NS-ORIENTATIONS OF MAPS University of Ljubljana Institute of Mathematics, Physics and Mechanics Department of Mathematics Jadranska 19, 1111 Ljubljana, Slovenia Preprint series, Vol. 42 (2004), 940 BAR-MAGNET POLYHEDRA AND NS-ORIENTATIONS

More information

The External Network Problem

The External Network Problem The External Network Problem Jan van den Heuvel and Matthew Johnson CDAM Research Report LSE-CDAM-2004-15 December 2004 Abstract The connectivity of a communications network can often be enhanced if the

More information

NP and computational intractability. Kleinberg and Tardos, chapter 8

NP and computational intractability. Kleinberg and Tardos, chapter 8 NP and computational intractability Kleinberg and Tardos, chapter 8 1 Major Transition So far we have studied certain algorithmic patterns Greedy, Divide and conquer, Dynamic programming to develop efficient

More information

Power Set of a set and Relations

Power Set of a set and Relations Power Set of a set and Relations 1 Power Set (1) Definition: The power set of a set S, denoted P(S), is the set of all subsets of S. Examples Let A={a,b,c}, P(A)={,{a},{b},{c},{a,b},{b,c},{a,c},{a,b,c}}

More information

2 A topological interlude

2 A topological interlude 2 A topological interlude 2.1 Topological spaces Recall that a topological space is a set X with a topology: a collection T of subsets of X, known as open sets, such that and X are open, and finite intersections

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

1 Variations of the Traveling Salesman Problem

1 Variations of the Traveling Salesman Problem Stanford University CS26: Optimization Handout 3 Luca Trevisan January, 20 Lecture 3 In which we prove the equivalence of three versions of the Traveling Salesman Problem, we provide a 2-approximate algorithm,

More information

Important separators and parameterized algorithms

Important separators and parameterized algorithms Important separators and parameterized algorithms Dániel Marx 1 1 Institute for Computer Science and Control, Hungarian Academy of Sciences (MTA SZTAKI) Budapest, Hungary PCSS 2017 Vienna, Austria September

More information

arxiv: v2 [math.co] 13 Aug 2013

arxiv: v2 [math.co] 13 Aug 2013 Orthogonality and minimality in the homology of locally finite graphs Reinhard Diestel Julian Pott arxiv:1307.0728v2 [math.co] 13 Aug 2013 August 14, 2013 Abstract Given a finite set E, a subset D E (viewed

More information

HOMEWORK #4 SOLUTIONS - MATH (1) (a) Prove that the chromatic polynomial of any tree with s vertices is. k(k 1) s 1

HOMEWORK #4 SOLUTIONS - MATH (1) (a) Prove that the chromatic polynomial of any tree with s vertices is. k(k 1) s 1 HOMEWORK #4 SOLUTIONS - MATH 3260 ASSIGNED: MARCH 19, 2003 DUE: APRIL 4, 2003 AT 2:30PM (1) (a) Prove that the chromatic polynomial of any tree with s vertices is k(k 1) s 1 Solution: Pick any vertex of

More information

Matching and Planarity

Matching and Planarity Matching and Planarity Po-Shen Loh June 010 1 Warm-up 1. (Bondy 1.5.9.) There are n points in the plane such that every pair of points has distance 1. Show that there are at most n (unordered) pairs of

More information

4 Generating functions in two variables

4 Generating functions in two variables 4 Generating functions in two variables (Wilf, sections.5.6 and 3.4 3.7) Definition. Let a(n, m) (n, m 0) be a function of two integer variables. The 2-variable generating function of a(n, m) is F (x,

More information

Part II. Graph Theory. Year

Part II. Graph Theory. Year Part II Year 2017 2016 2015 2014 2013 2012 2011 2010 2009 2008 2007 2006 2005 2017 53 Paper 3, Section II 15H Define the Ramsey numbers R(s, t) for integers s, t 2. Show that R(s, t) exists for all s,

More information

CSC 505, Fall 2000: Week 12

CSC 505, Fall 2000: Week 12 CSC 505, Fall 000: Week Proving the N P-completeness of a decision problem A:. Prove that A is in N P give a simple guess and check algorithm (the certificate being guessed should be something requiring

More information

Lecture 19 Thursday, March 29. Examples of isomorphic, and non-isomorphic graphs will be given in class.

Lecture 19 Thursday, March 29. Examples of isomorphic, and non-isomorphic graphs will be given in class. CIS 160 - Spring 2018 (instructor Val Tannen) Lecture 19 Thursday, March 29 GRAPH THEORY Graph isomorphism Definition 19.1 Two graphs G 1 = (V 1, E 1 ) and G 2 = (V 2, E 2 ) are isomorphic, write G 1 G

More information

Paths, Flowers and Vertex Cover

Paths, Flowers and Vertex Cover Paths, Flowers and Vertex Cover Venkatesh Raman, M.S. Ramanujan, and Saket Saurabh Presenting: Hen Sender 1 Introduction 2 Abstract. It is well known that in a bipartite (and more generally in a Konig)

More information

Paths, Flowers and Vertex Cover

Paths, Flowers and Vertex Cover Paths, Flowers and Vertex Cover Venkatesh Raman M. S. Ramanujan Saket Saurabh Abstract It is well known that in a bipartite (and more generally in a König) graph, the size of the minimum vertex cover is

More information

Figure : Example Precedence Graph

Figure : Example Precedence Graph CS787: Advanced Algorithms Topic: Scheduling with Precedence Constraints Presenter(s): James Jolly, Pratima Kolan 17.5.1 Motivation 17.5.1.1 Objective Consider the problem of scheduling a collection of

More information

Math 485, Graph Theory: Homework #3

Math 485, Graph Theory: Homework #3 Math 485, Graph Theory: Homework #3 Stephen G Simpson Due Monday, October 26, 2009 The assignment consists of Exercises 2129, 2135, 2137, 2218, 238, 2310, 2313, 2314, 2315 in the West textbook, plus the

More information

[Ramalingam, 4(12): December 2017] ISSN DOI /zenodo Impact Factor

[Ramalingam, 4(12): December 2017] ISSN DOI /zenodo Impact Factor GLOBAL JOURNAL OF ENGINEERING SCIENCE AND RESEARCHES FORCING VERTEX TRIANGLE FREE DETOUR NUMBER OF A GRAPH S. Sethu Ramalingam * 1, I. Keerthi Asir 2 and S. Athisayanathan 3 *1,2 & 3 Department of Mathematics,

More information

Definition 1 (Hand-shake model). A hand shake model is an incidence geometry for which every line has exactly two points.

Definition 1 (Hand-shake model). A hand shake model is an incidence geometry for which every line has exactly two points. Math 3181 Dr. Franz Rothe Name: All3181\3181_spr13t1.tex 1 Solution of Test I Definition 1 (Hand-shake model). A hand shake model is an incidence geometry for which every line has exactly two points. Definition

More information

Lecture 20 : Trees DRAFT

Lecture 20 : Trees DRAFT CS/Math 240: Introduction to Discrete Mathematics 4/12/2011 Lecture 20 : Trees Instructor: Dieter van Melkebeek Scribe: Dalibor Zelený DRAFT Last time we discussed graphs. Today we continue this discussion,

More information

Massachusetts Institute of Technology Department of Electrical Engineering and Computer Science Algorithms For Inference Fall 2014

Massachusetts Institute of Technology Department of Electrical Engineering and Computer Science Algorithms For Inference Fall 2014 Massachusetts Institute of Technology Department of Electrical Engineering and Computer Science 6.438 Algorithms For Inference Fall 2014 Recitation-6: Hardness of Inference Contents 1 NP-Hardness Part-II

More information

On Covering a Graph Optimally with Induced Subgraphs

On Covering a Graph Optimally with Induced Subgraphs On Covering a Graph Optimally with Induced Subgraphs Shripad Thite April 1, 006 Abstract We consider the problem of covering a graph with a given number of induced subgraphs so that the maximum number

More information

On a n Ed g e Crossing P roblem

On a n Ed g e Crossing P roblem On a n Ed g e Crossing P roblem Peter Eades, Department of Computer Science University of Queensland St. Lucia, Queensland 4067 Brendan D. McKay, Department of Computer Science Australian National University

More information

Discrete Mathematics and Probability Theory Fall 2009 Satish Rao,David Tse Note 8

Discrete Mathematics and Probability Theory Fall 2009 Satish Rao,David Tse Note 8 CS 70 Discrete Mathematics and Probability Theory Fall 2009 Satish Rao,David Tse Note 8 An Introduction to Graphs Formulating a simple, precise specification of a computational problem is often a prerequisite

More information

Algebra of Sets. Aditya Ghosh. April 6, 2018 It is recommended that while reading it, sit with a pen and a paper.

Algebra of Sets. Aditya Ghosh. April 6, 2018 It is recommended that while reading it, sit with a pen and a paper. Algebra of Sets Aditya Ghosh April 6, 2018 It is recommended that while reading it, sit with a pen and a paper. 1 The Basics This article is only about the algebra of sets, and does not deal with the foundations

More information

T. Background material: Topology

T. Background material: Topology MATH41071/MATH61071 Algebraic topology Autumn Semester 2017 2018 T. Background material: Topology For convenience this is an overview of basic topological ideas which will be used in the course. This material

More information

Discrete mathematics

Discrete mathematics Discrete mathematics Petr Kovář petr.kovar@vsb.cz VŠB Technical University of Ostrava DiM 470-2301/02, Winter term 2018/2019 About this file This file is meant to be a guideline for the lecturer. Many

More information

8.1 Polynomial-Time Reductions

8.1 Polynomial-Time Reductions 8.1 Polynomial-Time Reductions Classify Problems According to Computational Requirements Q. Which problems will we be able to solve in practice? A working definition. Those with polynomial-time algorithms.

More information

9.1 Cook-Levin Theorem

9.1 Cook-Levin Theorem CS787: Advanced Algorithms Scribe: Shijin Kong and David Malec Lecturer: Shuchi Chawla Topic: NP-Completeness, Approximation Algorithms Date: 10/1/2007 As we ve already seen in the preceding lecture, two

More information

Geometric Steiner Trees

Geometric Steiner Trees Geometric Steiner Trees From the book: Optimal Interconnection Trees in the Plane By Marcus Brazil and Martin Zachariasen Part 2: Global properties of Euclidean Steiner Trees and GeoSteiner Marcus Brazil

More information

4. Definition: topological space, open set, topology, trivial topology, discrete topology.

4. Definition: topological space, open set, topology, trivial topology, discrete topology. Topology Summary Note to the reader. If a statement is marked with [Not proved in the lecture], then the statement was stated but not proved in the lecture. Of course, you don t need to know the proof.

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

CS599: Convex and Combinatorial Optimization Fall 2013 Lecture 14: Combinatorial Problems as Linear Programs I. Instructor: Shaddin Dughmi

CS599: Convex and Combinatorial Optimization Fall 2013 Lecture 14: Combinatorial Problems as Linear Programs I. Instructor: Shaddin Dughmi CS599: Convex and Combinatorial Optimization Fall 2013 Lecture 14: Combinatorial Problems as Linear Programs I Instructor: Shaddin Dughmi Announcements Posted solutions to HW1 Today: Combinatorial problems

More information

Shannon Switching Game

Shannon Switching Game EECS 495: Combinatorial Optimization Lecture 1 Shannon s Switching Game Shannon Switching Game In the Shannon switching game, two players, Join and Cut, alternate choosing edges on a graph G. Join s objective

More information

Face Width and Graph Embeddings of face-width 2 and 3

Face Width and Graph Embeddings of face-width 2 and 3 Face Width and Graph Embeddings of face-width 2 and 3 Instructor: Robin Thomas Scribe: Amanda Pascoe 3/12/07 and 3/14/07 1 Representativity Recall the following: Definition 2. Let Σ be a surface, G a graph,

More information

Solving Linear Recurrence Relations (8.2)

Solving Linear Recurrence Relations (8.2) EECS 203 Spring 2016 Lecture 18 Page 1 of 10 Review: Recurrence relations (Chapter 8) Last time we started in on recurrence relations. In computer science, one of the primary reasons we look at solving

More information

HW Graph Theory SOLUTIONS (hbovik)

HW Graph Theory SOLUTIONS (hbovik) Diestel 1.3: Let G be a graph containing a cycle C, and assume that G contains a path P of length at least k between two vertices of C. Show that G contains a cycle of length at least k. If C has length

More information

Graph Theory S 1 I 2 I 1 S 2 I 1 I 2

Graph Theory S 1 I 2 I 1 S 2 I 1 I 2 Graph Theory S I I S S I I S Graphs Definition A graph G is a pair consisting of a vertex set V (G), and an edge set E(G) ( ) V (G). x and y are the endpoints of edge e = {x, y}. They are called adjacent

More information

CS 341: Algorithms. Douglas R. Stinson. David R. Cheriton School of Computer Science University of Waterloo. February 26, 2019

CS 341: Algorithms. Douglas R. Stinson. David R. Cheriton School of Computer Science University of Waterloo. February 26, 2019 CS 341: Algorithms Douglas R. Stinson David R. Cheriton School of Computer Science University of Waterloo February 26, 2019 D.R. Stinson (SCS) CS 341 February 26, 2019 1 / 296 1 Course Information 2 Introduction

More information

1. Suppose you are given a magic black box that somehow answers the following decision problem in polynomial time:

1. Suppose you are given a magic black box that somehow answers the following decision problem in polynomial time: 1. Suppose you are given a magic black box that somehow answers the following decision problem in polynomial time: Input: A CNF formula ϕ with n variables x 1, x 2,..., x n. Output: True if there is an

More information

Final Test in MAT 410: Introduction to Topology Answers to the Test Questions

Final Test in MAT 410: Introduction to Topology Answers to the Test Questions Final Test in MAT 410: Introduction to Topology Answers to the Test Questions Stefan Kohl Question 1: Give the definition of a topological space. (3 credits) A topological space (X, τ) is a pair consisting

More information

GRAPHS, GRAPH MODELS, GRAPH TERMINOLOGY, AND SPECIAL TYPES OF GRAPHS

GRAPHS, GRAPH MODELS, GRAPH TERMINOLOGY, AND SPECIAL TYPES OF GRAPHS GRAPHS, GRAPH MODELS, GRAPH TERMINOLOGY, AND SPECIAL TYPES OF GRAPHS DR. ANDREW SCHWARTZ, PH.D. 10.1 Graphs and Graph Models (1) A graph G = (V, E) consists of V, a nonempty set of vertices (or nodes)

More information

Lecture 2 - Graph Theory Fundamentals - Reachability and Exploration 1

Lecture 2 - Graph Theory Fundamentals - Reachability and Exploration 1 CME 305: Discrete Mathematics and Algorithms Instructor: Professor Aaron Sidford (sidford@stanford.edu) January 11, 2018 Lecture 2 - Graph Theory Fundamentals - Reachability and Exploration 1 In this lecture

More information

Advanced Algorithms Class Notes for Monday, October 23, 2012 Min Ye, Mingfu Shao, and Bernard Moret

Advanced Algorithms Class Notes for Monday, October 23, 2012 Min Ye, Mingfu Shao, and Bernard Moret Advanced Algorithms Class Notes for Monday, October 23, 2012 Min Ye, Mingfu Shao, and Bernard Moret Greedy Algorithms (continued) The best known application where the greedy algorithm is optimal is surely

More information

Bipartite Roots of Graphs

Bipartite Roots of Graphs Bipartite Roots of Graphs Lap Chi Lau Department of Computer Science University of Toronto Graph H is a root of graph G if there exists a positive integer k such that x and y are adjacent in G if and only

More information

Graph Representations and Traversal

Graph Representations and Traversal COMPSCI 330: Design and Analysis of Algorithms 02/08/2017-02/20/2017 Graph Representations and Traversal Lecturer: Debmalya Panigrahi Scribe: Tianqi Song, Fred Zhang, Tianyu Wang 1 Overview This lecture

More information

Faster parameterized algorithms for Minimum Fill-In

Faster parameterized algorithms for Minimum Fill-In Faster parameterized algorithms for Minimum Fill-In Hans L. Bodlaender Pinar Heggernes Yngve Villanger Abstract We present two parameterized algorithms for the Minimum Fill-In problem, also known as Chordal

More information

CSE 331: Introduction to Algorithm Analysis and Design Graphs

CSE 331: Introduction to Algorithm Analysis and Design Graphs CSE 331: Introduction to Algorithm Analysis and Design Graphs 1 Graph Definitions Graph: A graph consists of a set of verticies V and a set of edges E such that: G = (V, E) V = {v 0, v 1,..., v n 1 } E

More information

The strong chromatic number of a graph

The strong chromatic number of a graph The strong chromatic number of a graph Noga Alon Abstract It is shown that there is an absolute constant c with the following property: For any two graphs G 1 = (V, E 1 ) and G 2 = (V, E 2 ) on the same

More information

Basic Graph Theory with Applications to Economics

Basic Graph Theory with Applications to Economics Basic Graph Theory with Applications to Economics Debasis Mishra February, 0 What is a Graph? Let N = {,..., n} be a finite set. Let E be a collection of ordered or unordered pairs of distinct elements

More information

Strongly connected: A directed graph is strongly connected if every pair of vertices are reachable from each other.

Strongly connected: A directed graph is strongly connected if every pair of vertices are reachable from each other. Directed Graph In a directed graph, each edge (u, v) has a direction u v. Thus (u, v) (v, u). Directed graph is useful to model many practical problems (such as one-way road in traffic network, and asymmetric

More information

Math 443/543 Graph Theory Notes 5: Planar graphs and coloring

Math 443/543 Graph Theory Notes 5: Planar graphs and coloring Math 443/543 Graph Theory Notes 5: Planar graphs and coloring David Glickenstein October 10, 2014 1 Planar graphs The Three Houses and Three Utilities Problem: Given three houses and three utilities, can

More information