VC To Maxcut Reduction
VC To Maxcut Reduction
1 qstart u1 1 …. a cell ….
….
Input u-variables of ψ Observe: ψ(u) = 1 iff N(u) = 1
Recap: Cook-Levin Theorem
Let L ∈ NP. We intend to come up with a polynomial
time computable function f: x ϕx s.t.,
x∈L ϕx ∈ SAT
ψx is a poly(|x|)-size circuit
Recap: Cook-Levin Theorem
Let L ∈ NP. We intend to come up with a polynomial
time computable function f: x ϕx s.t.,
x∈L ϕx ∈ SAT
Max-Cut (NP-hard)
Example 1: Independent Set
INDSET := {(G, k): G has independent set of size k}
Ci
Ci
C1 Cm
Graph G on 7m vertices
Example 1: Independent Set
Reduction: Let ϕ be a 3CNF with m clauses and n
variables. Assume, every clause has exactly 3 literals.
Ci
C1 Cm
x1 ∨ x2 ∨ x3 x1 + (1- x2) + x3 ≥ 1
Example 5: Max Cut
MaxCut : Given a graph find a cut with the max size.
A cut of G = (V, E) is a tuple (U, V\U), U ⊆ V. Size of a
cut (U, V\U) is the number of edges from U to V\U.
w
u u
degH(u) – 1 edges
between u and w
H G
= 2.|EU(H)| - |U|
Example 5: Max Cut
Claim: |MaxCut(G)| = 2.|E(H)| - |MinVCover(H)|
Proof: Let V(H) = V. Then V(G) = V + w.
Suppose (U, V\U + w) is a cut in G.
ϕ(x1,…,xn)
SAT is downward self-reducible
Proof. (decision search) Let L = SAT, and A be a
poly-time algorithm to decide if ϕ(x1,…,xn) is satisfiable.
ϕ(x1,…,xn) A(ϕ) = Y
SAT is downward self-reducible
Proof. (decision search) Let L = SAT, and A be a
poly-time algorithm to decide if ϕ(x1,…,xn) is satisfiable.
ϕ(x1,…,xn) A(ϕ) = Y
ϕ(0,…,xn)
SAT is downward self-reducible
Proof. (decision search) Let L = SAT, and A be a
poly-time algorithm to decide if ϕ(x1,…,xn) is satisfiable.
ϕ(x1,…,xn) A(ϕ) = Y
A( ϕ(0,..) ) = N ϕ(0,…,xn)
SAT is downward self-reducible
Proof. (decision search) Let L = SAT, and A be a
poly-time algorithm to decide if ϕ(x1,…,xn) is satisfiable.
ϕ(x1,…,xn) A(ϕ) = Y
ϕ(x1,…,xn) A(ϕ) = Y
ϕ(x1,…,xn) A(ϕ) = Y
ϕ(1,0,…,xn)
SAT is downward self-reducible
Proof. (decision search) Let L = SAT, and A be a
poly-time algorithm to decide if ϕ(x1,…,xn) is satisfiable.
ϕ(x1,…,xn) A(ϕ) = Y
A( ϕ(1,0,..) ) = Y ϕ(1,0,…,xn)
SAT is downward self-reducible
Proof. (decision search) Let L = SAT, and A be a
poly-time algorithm to decide if ϕ(x1,…,xn) is satisfiable.
ϕ(x1,…,xn) A(ϕ) = Y
A( ϕ(1,0,..) ) = Y ϕ(1,0,…,xn)
ϕ(1,0,0,…,xn)
SAT is downward self-reducible
Proof. (decision search) Let L = SAT, and A be a
poly-time algorithm to decide if ϕ(x1,…,xn) is satisfiable.
ϕ(x1,…,xn) A(ϕ) = Y
A( ϕ(1,0,..) ) = Y ϕ(1,0,…,xn)
A( ϕ(1,0,0...) ) = N ϕ(1,0,0,…,xn)
SAT is downward self-reducible
Proof. (decision search) Let L = SAT, and A be a
poly-time algorithm to decide if ϕ(x1,…,xn) is satisfiable.
ϕ(x1,…,xn) A(ϕ) = Y
A( ϕ(1,0,..) ) = Y ϕ(1,0,…,xn)
ϕ(x1,…,xn) A(ϕ) = Y
A( ϕ(1,0,..) ) = Y ϕ(1,0,…,xn)
ϕ(x1,…,xn) A(ϕ) = Y
A( ϕ(1,0,..) ) = Y ϕ(1,0,…,xn)
ϕ(x1,…,xn) A(ϕ) = Y
A( ϕ(1,0,..) ) = Y ϕ(1,0,…,xn)
SAT ≤p L L ≤p SAT
Decision ≡ Search for NPC problems
Proof. (decision search) Let L be NP-complete, and
B be a poly-time algorithm to decide if x∈L.
SAT ≤p L L ≤p SAT
x ϕx
Decision ≡ Search for NPC problems
Proof. (decision search) Let L be NP-complete, and
B be a poly-time algorithm to decide if x∈L.
SAT ≤p L L ≤p SAT
x ϕx
SAT ≤p L L ≤p SAT
x ϕx
SAT ≤p L L ≤p SAT
x ϕx
SAT ≤p L L ≤p SAT
ϕ f(ϕ) x ϕx
SAT ≤p L L ≤p SAT
ϕ f(ϕ) x ϕx
Probably not!
Decision versus Search
Is search equivalent to decision for every NP problem?
n
Let EE = ∪ DTIME (2c.2 ) and
c≥0
Doubly exponential
n analogues of P and NP
NEE = ∪ NTIME (2 )
c.2
c≥0
Decision versus Search
Is search equivalent to decision for every NP problem?