Tool: Linearity Testing and the Walsh-Hadamard Code

Size: px
Start display at page:

Download "Tool: Linearity Testing and the Walsh-Hadamard Code"

Transcription

1 11.5 NP PCP(poly(n), 1): PCPfromtheWalsh-Hadamardcode 215 compute this mapping. We call reductions with these properties Levin reductions (see the proof of Theorem 2.18). It is worthwhile to observe that the PCP reductions of this chapter also satisfy this property. For example, the proof of Theorem actually yields awaynotjusttomap,say,acnfformulaϕ into a graph G such that ϕ is satisfiable iff G has a large independent set, but actually shows how to efficiently map a satisfying assignment for ϕ into a large independent set in G and a not-too-small independent set in G into a satisfying assignment for ϕ. This will become clear from our proof of the PCP Theorem in Chapter NP PCP(poly(n), 1): PCPfromtheWalsh-Hadamardcode We now prove a weaker version of the PCP Theorem, showing that every NP statement has an exponentially-long proof that can be locally tested by only looking at a constant number of bits. In addition to giving a taste of how one proves PCP Theorems, techniques from this section will be used in the proof of the full-fledged PCP theorem in Chapter 22. Theorem (Exponential-sized PCP system for NP [ALM + 92]) NP PCP(poly(n), 1) We prove this theorem by designing an appropriate verifier for an NP-complete language. The verifier expects the proof to contain an encoded version of the usual certificate. The verifier checks such an encoded certificate by simple probabilistic tests Tool: Linearity Testing and the Walsh-Hadamard Code We use the Walsh-Hadamard code (see also Section , though the treatment here is selfcontained). It is a way to encode bit strings of length n by linear functions in n variables over GF(2). The encoding function WH : {0, 1} {0, 1} maps a string u {0, 1} n to the truth table of the function x u x, whereforx, y {0, 1} n we define x y = n i=1 x iy i (mod 2). Note that this is a very inefficient encoding method: an n-bit string u {0, 1} n is encoded using WH(u) =2 n bits. If f {0, 1} 2n is equal to WH(u) forsomeu then we say that f is a Walsh-Hadamard codeword. Such a string f {0, 1} 2n can also be viewed as a function from {0, 1} n to {0, 1}. Below, we repeatedly use the following fact (see Claim A.31): random subsum principle: If u v then for 1 /2 the choices of x, u x v x. The random subsum principle implies that the Walsh-Hadamard codeisanerrorcorrecting code with minimum distance 1 /2, bywhichwemeanthatforeveryu v {0, 1} n, the encodings WH(u) and WH(v) differ in at least half the bits. Now we talk about local tests for the Walsh-Hadamard code (i.e., tests making only O(1) queries). Local testing of Walsh-Hadamard code. Suppose we are given access to a function f : {0, 1} n {0, 1} and want to test whether or not f is actually a codeword of Walsh- Hadamard. Since the Walsh-Hadamard codewords are precisely the set of all linear functions from {0, 1} n to {0, 1}, wecantestf by checking that f(x + y) =f(x)+f(y) (3)

2 PCP Theorem and Hardness of Approximation: An introduction for all the 2 2n pairs x, y {0, 1} n (where + on the left side of (3) denotes vector addition over GF(2) n and on the right side denotes addition over GF(2)). This test works by definition, but it involves reading all 2 n values of f. Can we test f by reading only a constant number of its values? The natural test is to choose x, y at random and verify (3). Clearly, even such a local test accepts a linear function with probability 1. However, now we can no longer guarantee that every function that is not linear is rejected with high probability! For example, if f is very close to being a linear function, meaning that f is obtained by modifying a linear function on a very small fraction of its inputs, then such a local test will encounter the nonlinear part with very low probability, and thus not be able to distinguish f from a linear function. So we set our goal less ambitiously: a test that on one hand accepts every linear function,and on the other hand rejects with high probability every function that is far from linear. The natural test above suffices for this job. Definition Let ρ [0, 1]. We say that f,g : {0, 1} n {0, 1} are ρ-close if Pr x R {0,1} n[f(x) = g(x)] ρ. We say that f is ρ-close to a linear function if there exists a linear function g such that f and g are ρ-close. Theorem (Linearity Testing [BLR90]) Let f : {0, 1} n {0, 1} be such that Pr x,y R {0,1} n[f(x + y) =f(x)+f(y)] ρ for some ρ > 1 /2. Thenf is ρ-close to a linear function. We defer the proof of Theorem to Section 22.5 of Chapter 22. For every δ (0, 1 /2), we can obtain a linearity test that rejects with probability at least 1 /2 every function that is not (1 δ)-close to a linear function, by testing Condition (3) repeatedly O(1/δ) times with independent randomness. We call such a test a (1 δ)-linearity test. Local decoding of Walsh-Hadamard code. Suppose that for δ < 1 4 the function f : {0, 1} n {0, 1} is (1 δ)-close to some linear function f. Becauseeverytwolinearfunctions differ on half of their inputs, the function f is uniquely determined by f. Suppose we are given x {0, 1} n and random access to f. Can we obtain the value f(x) usingonlya constant number of queries? The naive answer is that since most x s satisfy f(x) = f(x), we should be able to learn f(x) with good probability by making only the single query x to f. The problem is that x could very well be one of the places where f and f differ. Fortunately, there is still a simple way to learn f(x) whilemakingonlytwoqueriestof: 1. Choose x R {0, 1} n. 2. Set x = x + x. 3. Let y = f(x )andy = f(x ). 4. Output y + y. Since both x and x are individually uniformly distributed (even though they are dependent), by the union bound with probability at least 1 2δ we have y = f(x )and y = f(x ). Yet by the linearity of f, f(x) = f(x + x )= f(x )+ f(x ), and hence with at least 1 2δ probability f(x) =y + y. (We use here the fact that over GF(2), a + b = a b.) This technique is called local decoding of the Walsh-Hadamard code since it allows to recover any bit of the correct codeword (the linear function f) fromacorrupted version (the function f) whilemakingonlyaconstantnumberofqueries. Itisalsoknown as self correction of the Walsh-Hadamard code.

3 11.5 NP PCP(poly(n), 1): PCPfromtheWalsh-Hadamardcode Proof of Theorem We will show a (poly(n), 1)-verifier proof system for a particular NP-complete language L. The result that NP PCP(poly(n), 1) follows since every NP language is reducible to L. TheNP-complete language L we use is QUADEQ, thelanguageofsystemsofquadratic equations over GF(2) = {0, 1} that are satisfiable. Example The following is an instance of QUADEQ over the variables u 1,...,u 5 : u 1 u 2 + u 3 u 4 + u 1 u 5 =1 u 2 u 3 + u 1 u 4 =0 u 1 u 4 + u 3 u 5 + u 3 u 4 =1 This instance is satisfiable since the all-1 assignment satisfies all the equations. QUADEQ is NP-complete, as can be checked by reducing from the NP-complete language CKT-SAT of satisfiable Boolean circuits (see Section 6.1.2). The idea istohavea variable represent the value of each wire in the circuit (including the input wires) and to express AND and OR using the equivalent quadratic polynomial: x y =1iff (1 x)(1 y) =0, and so on. Details are left as Exercise Since u i =(u i ) 2 in GF(2), we can assume the equations do not contain terms of the form u i (i.e., all terms are of degree exactly two). Hence m quadratic equations over the variables u 1,...,u n can be described by an m n 2 matrix A and an m-dimensional vector b (both over GF(2)). Indeed, the problem QUADEQ can be phrased as the task, given such A, b, offindingann 2 -dimensional vector U satisfying (1) AU = b and (2) U is the tensor product u u of some n-dimensional vector u. 4 WH(u) WH(uOu) x Figure 11.2 The PCP proof that a set of quadratic equations is satisfiable consists of WH(u) andwh(u u) forsomevectoru. Theverifierfirstchecksthattheproofiscloseto having this form, and then uses the local decoder of the Walsh-Hadamard code to ensure that u is a solution for the quadratic equation instance. In the figure above the dotted areas represent corrupted coordinates. The PCP verifier. We now describe the PCP system for QUADEQ. Let A, b be an instance of QUADEQ and suppose that A, b is satisfiable by an assignment u {0, 1} n. The verifier V gets access to a proof π {0, 1} 2n +2 n2, which we interpret as a pair of functions f : {0, 1} n {0, 1} and g : {0, 1} n2 {0, 1}. In the correct PCP proof π for A, b, thefunctionf will be the Walsh-Hadamard encoding for u and the function g will be the Walsh-Hadamard encoding for u u. Thatis, wewilldesignthepcp verifier V in a way ensuring that it accepts proofs of this form with probability one, hence satisfying the completeness condition. The analysis repeatedly uses the random subsum principle. Step 1: Check that f, g are linear functions. As already noted, this isn t something that the verifier can check per se using local tests. Instead, the verifier performs a linearity test on both f,g, andrejectstheproofatonceifeithertestfails. Thus, if either of f,g is not close to a linear function, then V rejects with high probability. Therefore for the rest of the procedure we can assume that there exist two 4 If x, y are two n-dimensional vectors then their tensor product, denotedx y, isthen 2 -dimensional vector (or n n matrix) whose i, j th entry is x i y j (identifying [n 2 ]with[n] [n] insomecanonicalway). See also Section

4 PCP Theorem and Hardness of Approximation: An introduction linear functions f : {0, 1} n {0, 1} and g : {0, 1} n2 {0, 1} such that f is close to f, and g is close to g. (Note:inacorrectproof,thetestssucceedwithprobability 1 and f = f and g = g.) In fact, we will assume that for Steps 2 and 3, the verifier can query f, g at any desired point. The reason is that local decoding allows the verifier to recoveranydesiredvalueof f, g with good probability, and Steps 2 and 3 will only use a small (less than 20) number of queries to f, g. Thuswithhighprobability(say> 0.9) local decoding will succeed on all these queries. notation: To simplify notation and in the rest of the procedure we use f,g for f, g respectively. (This is OK since as argued above, V can query f, g at will.) In particular we assume both f and g are linear, and thus they must encode some strings u {0, 1} n and w {0, 1} n2.inotherwords,f,g are the functions given by f(r) =u r and g(z) =w z. Step 2: Verify that g encodes u u, where u {0, 1} n is the string encoded by f. The verifier does the following test ten times using independent random bits: Choose r, r independently at random from {0, 1} n,andiff(r)f(r ) g(r r )thenhaltandreject. In a correct proof, w = u u, so f(r)f(r )= u i r i u j r j = u i u j r i r j =(u u) (r r ), i [n] j [n] i,j [n] which in the correct proof is equal to g(r r ). Thus Step 2 never rejects a correct proof. Suppose now that, unlike the case of the correct proof, w u u. Weclaimthatineach of the ten trials V will halt and reject with probability at least 1 4.(Thustheprobabilityof rejecting in at least one trial is at least 1 (3/4) 10 > 0.9.) Indeed, let W be an n n matrix with the same entries as w, letu be the n n matrix such that U i,j = u i u j and think of r as a row vector and r as a column vector. In this notation, g(r r )=w (r r )= w i,j r i r j = rw r i,j [n] n n f(r)f(r )=(u r)(u r )=( u i r i )( u j r j)= u i u j r i r j = rur i=1 j=1 i,j [n] And V rejects if rw r rur. The random subsum principle implies that if W U then at least 1 /2 of all r satisfy rw ru. Applyingtherandomsubsumprincipleforeach such r, weconcludethatatleast 1 /2 the r satisfy rw r rur.weconcludethatthetrial rejects for at least 1/4 ofallpairsr, r. Step 3: Verify that f encodes a satisfying assignment. Using all that has been verified about f,g in the previous two steps, it is easy to check that any particular equation, say the kth equation of the input, is satisfied by u, namely, A k,(i,j) u i u j = b k. (4) i,j Denoting by z the n 2 dimensional vector (A k,(i,j) ) (where i, j vary over [1..n]), we see that the left hand side is nothing but g(z). Since the verifier knows A k,(i,j) and b k,itsimply queries g at z and checks that g(z) =b k. The drawback of the above idea is that in order to check that u satisfies the entire system, the verifier needs to make a query to g for each k =1, 2,...,m,whereasthenumber of queries is required to be independent of m. Luckily, we can use the random subsum principle again! The verifier takes a random subset of the equations and computes their sum mod 2. (In other words, for k =1, 2,...,m multiply the equation in (4) by a random bit and take the sum.) This sum is a new quadratic equation, and therandomsubsum principle implies that if u does not satisfy even one equation in the original system, then with probability at least 1/2 itwillnotsatisfythisnewequation. Theverifierchecksthat u satisfies this new equation.

5 Chapter notes and history 219 Overall, we get a verifier V such that (1) if A, b is satisfiable then V accepts the correct proof with probability 1 and (2) if A, b is not satisfiable then V accepts every proof with probability at most 0.8. The probability of accepting a proof for a false statement can be reduced to 1 /2 by simple repetition, completing the proof of Theorem Chapter notes and history The notion of approximation algorithms predates the discovery of NP-completeness; for instance Graham s 1966 paper [Gra66] alreadygivesanapproximationalgorithmforaschedulingprob- lem that was later proven NP-complete. Shortly after the discovery of NP-completeness, Johnson [Joh74] formalized the issue of computing approximate solutions, gave some easy approximation algorithms (such as the 1/2-approximation for MAX-SAT) for a variety of problems and posed the question of whether better algorithms exist. Over the next 20 years,althoughafewresultswere proven regarding the hardness of computing approximate solutions (such as for general TSP in Sahni and Gonzalez [SG76]) and a few approximation algorithms were designed, it became increasingly obvious that we were lacking serious techniques for proving the hardness of approximation. One of the problems seemed to be that there were no obvious interreducibilies among problems that preserved approximability. The paper by Papadimitriou andyannakakis[py88] showedsuch interreducibilities among a large set of problems they called MAX-SNP, and showed further that MAX-3SAT is complete for this class. This made MAX-3SAT an attractive problem to study both from point of view of algorithm design and for proving hardness results. Soon after this work, seemingly unrelated developments occurred in study of interactive proofs, some of which we studied in Chapter 8. The most relevant for the topicofthischapterwasthe result of Babai, Fortnow and Lund [BFL90] thatmip = NEXP, whichwassoonmadetoapplyto NP in the paper of Babai, Fortnow, Levin, and Szegedy [BFLS91]. After this there were a sequence of swift developments. In 1991 came a stunning result by Feige, Goldwasser, Lovasz, Safra and Szegedy [FGL + 91] whichshowedthatifsat does not have subexponential time algorithms then the INDSET problem cannot be approximated within a factor 2 log1 ϵ n for any ϵ > 0. This was the first paper to connect hardness of approximation with PCP-like theorems, though at the time many researchers felt (especially because the result did not prove NP-completeness per se) that this was the wrong idea and the result would ultimately be reproven with no mention of interactive proofs. (Intriguingly, Dinur s gap amplification lemma brings us closer to that dream.) However, a year later Arora and Safra [AS92] furtherrefinedtheideasof[bfl90] (togetherwiththeideaofverifier composition) to prove that approximating INDSET is actually NP-complete. They also proved a surprising new characterization of NP in terms of PCP, namely,np = PCP(log n, log n). At that point it became clear that if the query parameter could be sublogarithmic, it might well be made a constant! The subsequent paper of Arora, Lund, Motwani, Sudan, and Szegedy [ALM + 92] took this next step (in the process introducing the constant-bit verifier of Section 11.5, as well as other ideas) to prove NP = PCP(log n, 1), which they showed also implied the NP-hardness of approximating MAX-3SAT. SincethenmanyotherPCP theorems have been proven, as surveyed in Chapter 22. (Note that in this chapter we derived the hardness result for INDSET from the result for MAX-3SAT, eventhoughhistoricallytheformerhappenedfirst.) The overall idea in the AS-ALMSS proof of the PCP Theorem (as indeed the one in the proof of MIP = NEXP) issimilartotheproofoftheorem InfactTheorem11.19 is the only part of the original proof that still survives in our writeup; therestoftheproofinchapter22isa more recent proof due to Dinur. However, in addition to using encodings based upon the Walsh- Hadamard code the AS-ALMSS proof also used encodings based upon low degree multivariate polynomials. These have associated procedures analogous to thelinearitytestandlocaldecoding, though the proofs of correctness are a fair bit harder. The proof also drew intuition from the topic of self-testing and self-correcting programs [BLR90, RS92]. The PCP Theorem led to a flurry of results about hardness of approximation. See Trevisan [Tre05]forarecentsurveyandArora-Lund[AL95] foranolderone. The PCP Theorem, as well as its cousin, MIP = NEXP, doesnotrelativize[frs88]. In this chapter we only talked about some very trivial approximation algorithms, which are unfortunately not very representative of the state of the art. See Hochbaum [Hoc97] andvazirani [Vaz01] for a good survey of the many ingenious approximation algorithms that have been developed.

6 Proofs of PCP Theorems and the Fourier Transform Technique 22.5 Tool: the Fourier transform technique Theorem is proved using Fourier analysis. The continuous Fourier transform is extremely useful in mathematics and engineering. Likewise, the discrete Fourier transform has found many uses in algorithms and complexity, in particular for constructing and analyzing PCP s. The Fourier transform technique for PCP s involves calculating the maximum acceptance probability of the verifier using Fourier analysis of the functions presented in the proof string. (See Note for a broader perspective of uses of discrete Fourier transforms in combinatorial and probabilistic arguments.) It is delicate enough to give tight inapproximability results for MAX-INDSET, MAX-3SAT, and many other problems. To introduce the technique we start with a simple example: analysis of the linearity test over GF(2) (i.e., proof of Theorem 11.21). We then introduce the Long Code and show how to test for membership in it. These ideas are then used to prove Håstad s 3-bit PCP Theorem Fourier transform over GF(2) n The Fourier transform over GF(2) n is a tool to study functions on the Boolean hypercube. In this chapter, it will be useful to use the set {+1, 1} = {±1} instead of {0, 1}. To transform {0, 1} to {±1}, weusethemappingb ( 1) b (i.e., 0 +1, 1 1). Thus we write the hypercube as {±1} n instead of the more usual {0, 1} n.notethismapsthexor operation (i.e., addition in GF(2)) into the multiplication operationoverr. The set of functions from {±1} n to R defines a 2 n -dimensional Hilbert space (i.e., a vector space with an associated inner product) as follows. Addition and multiplication by ascalararedefinedinthenaturalway:(f + g)(x) =f(x)+g(x) and(αf)(x) =αf(x) for every f,g : {±1} n R, α R. Wedefinetheinnerproductoftwofunctionsf,g, denoted f,g, tobee x {±1} n[f(x)g(x)]. (This is the expectation inner product.) The standard basis for this space is the set {e x } x {±1} n,wheree x (y) isequalto1ify = x, andequalto0otherwise.thisisanorthogonalbasis,andevery function f : {±1} n R can be represented in this basis as f = x a xe x.foreveryx {±1} n,thecoefficient a x is equal to f(x). The Fourier basis is an alternative orthonormal basis that contains, for every subset α [n], a function χ α where χ α (x) = i α x i. (We define χ to be the function that is 1 everywhere). This basis is actually the Walsh-Hadamard code (see Section ) in disguise: the basis vectors correspond to the linear functions over GF(2). To see this, note that every linear function of the form b a b (with a, b {0, 1} n )ismappedbyour transformation to the function taking x {±1} n to i s.t. a x i=1 i.tocheckthatthefourier basis is indeed an orthonormal basis for R 2n,notethattherandomsubsumprincipleimplies that for every α, β [n], χ α, χ β = δ α,β where δ α,β is equal to 1 iff α = β and equal to 0 otherwise. Remark Note that in the { 1, 1} view, the basis functions can be viewed as multilinear polynomials (i.e., multivariate polynomials whose degree in each variable is 1). Thus the fact that every real-valued function f :{ 1, 1} n has a Fourier expansion can also be phrased as Every such function can be represented by a multilinear polynomial. This is very much in the same spirit as the polynomial representations used in Chapters 8 and 11. Since the Fourier basis is an orthonormal basis, every function f : {±1} n R can be represented as f = α [n] ˆf α χ α.wecallˆf α the α th Fourier coefficient of f. Wewilloften use the following simple lemma: Lemma Every two functions f,g:{±1} n R satisfy 1. f,g = α ˆf α ĝ α. 2. (Parseval s Identity) f,f = α ˆf 2 α.

7 22.5 Tool: the Fourier transform technique 411 Proof: The second property follows from the first. To prove the first we expand f,g = α ˆf α χ α, β ĝ β χ β = α,β ˆf α ĝ β χ α, χ β = α,β ˆf α ĝ β δ α,β = α ˆf α ĝ α Example Some examples for the Fourier transform of particular functions: 1. The majority function on 3 variables (i.e., the function MAJ(u 1,u 2,u 3 ) that outputs +1 if and only if at least two of its inputs are +1, and 1 otherwise) can be expressed as 1 /2u /2u /2u 3 1 /2u 1 u 2 u 3. Thus, it has four Fourier coefficients equal to 1 /2 and the rest are equal to zero. 2. If f(u 1,u 2,...,u n )=u i (i.e., f is a coordinate function, aconceptwewill see again in context of long codes) then f = χ {i} and so ˆf {i} =1and ˆf α =0 for α {i}. 3. If f is a random Boolean function on n bits, then each ˆf α is a random variable that is a sum of 2 n binomial variables (equally likely to be 1, 1) and hence looks like a normally distributed variable with standard deviation 2 n/2 and mean 0. Thus with high probability, all 2 n Fourier coefficients have values in [ poly(n), poly(n) ]. 2 n/2 2 n/ The connection to PCPs: High level view In the PCP context we are interested in Boolean-valued functions, i.e., those from GF (2) n to GF (2). Under our transformation they turn into functions from {±1} n to {±1}. Thus, we say that f : {±1} n R is Boolean if f(x) {±1} for every x {±1} n. Note that if f is Boolean then f,f = E x [f(x) 2 ]=1. On a high level, we use the Fourier transform in the soundness proofs for PCP s to show that if the verifier accepts a proof π with high probability then π is close to being wellformed (where the precise meaning of close-to and well-formed is context dependent). Usually we relate the acceptance probability of the verifier to an expectation of the form f,g = E x [f(x)g(x)], where f and g are Boolean functions arising from the proof. We then use techniques similar to those used to prove Lemma to relate this acceptance probability to the Fourier coefficients of f,g, allowing us to argue that if the verifier s test accepts with high probability, then f and g have few relatively large Fourier coefficients. This will provide us with some nontrivial useful information aboutf and g, since in a generic or random function, all the Fourier coefficient are small and roughly equal Analysis of the linearity test over GF (2) We will now prove Theorem 11.21, thus completing the proof of the PCP Theorem. Recall that the linearity test is provided a function f :GF(2) n GF(2) and has to determine whether f has significant agreement with a linear function. To do this itpicksx, y GF(2) n randomly and accepts iff f(x + y) =f(x)+f(y). Now we rephrase this test using {±1} instead of GF(2), so linear functions turn into Fourier basis functions. For every two vectors x, y {±1} n,wedenotebyxy their componentwise multiplication. That is, xy =(x 1 y 1,...,x n y n ). Note that for every basis function χ α (xy) =χ α (x)χ α (y). For two Boolean functions f,g, theirinnerproduct f,g is equal to the fraction of inputs on which they agree minus the fraction of inputs on which they disagree. It follows

Lecture 8 (Notes) 1. The book Computational Complexity: A Modern Approach by Sanjeev Arora and Boaz Barak;

Lecture 8 (Notes) 1. The book Computational Complexity: A Modern Approach by Sanjeev Arora and Boaz Barak; Topics in Theoretical Computer Science April 18, 2016 Lecturer: Ola Svensson Lecture 8 (Notes) Scribes: Ola Svensson Disclaimer: These notes were written for the lecturer only and may contain inconsistent

More information

DRAFT. PCP and Hardness of Approximation. Chapter 19

DRAFT. PCP and Hardness of Approximation. Chapter 19 Chapter 19 PCP and Hardness of Approximation...most problem reductions do not create or preserve such gaps...to create such a gap in the generic reduction (cf. Cook)...also seems doubtful. The intuitive

More information

PCP Theorem and Hardness of Approximation

PCP Theorem and Hardness of Approximation PCP Theorem and Hardness of Approximation An Introduction Lee Carraher and Ryan McGovern Department of Computer Science University of Cincinnati October 27, 2003 Introduction Assuming NP P, there are many

More information

Advanced Algorithms (XIII) Yijia Chen Fudan University

Advanced Algorithms (XIII) Yijia Chen Fudan University Advanced Algorithms (XIII) Yijia Chen Fudan University The PCP Theorem Theorem NP = PCP(log n, 1). Motivation Approximate solutions Definition (Approximation of MAX-3SAT) For every 3CNF formula ϕ, the

More information

[PCP Theorem is] the most important result in complexity theory since Cook s Theorem. Ingo Wegener, 2005

[PCP Theorem is] the most important result in complexity theory since Cook s Theorem. Ingo Wegener, 2005 PCP Theorem [PCP Theorem is] the most important result in complexity theory since Cook s Theorem. Ingo Wegener, 2005 Computational Complexity, by Fu Yuxi PCP Theorem 1 / 88 S. Arora, C. Lund, R. Motwani,

More information

Lecture 3: Boolean Functions and the Walsh Hadamard Code 1

Lecture 3: Boolean Functions and the Walsh Hadamard Code 1 CS-E4550 Advanced Combinatorics in Computer Science Autumn 2016: Selected Topics in Complexity Theory Lecture 3: Boolean Functions and the Walsh Hadamard Code 1 1. Introduction The present lecture develops

More information

Complexity Theory. Jörg Kreiker. Summer term Chair for Theoretical Computer Science Prof. Esparza TU München

Complexity Theory. Jörg Kreiker. Summer term Chair for Theoretical Computer Science Prof. Esparza TU München Complexity Theory Jörg Kreiker Chair for Theoretical Computer Science Prof. Esparza TU München Summer term 2010 Lecture 19 Hardness of Approximation 3 Recap Recap: optimization many decision problems we

More information

Lecture 22. m n c (k) i,j x i x j = c (k) k=1

Lecture 22. m n c (k) i,j x i x j = c (k) k=1 Notes on Complexity Theory Last updated: June, 2014 Jonathan Katz Lecture 22 1 N P PCP(poly, 1) We show here a probabilistically checkable proof for N P in which the verifier reads only a constant number

More information

Lecture 10: Hardness of approximating clique, FGLSS graph

Lecture 10: Hardness of approximating clique, FGLSS graph CSE 533: The PCP Theorem and Hardness of Approximation (Autumn 2005) Lecture 10: Hardness of approximating clique, FGLSS graph Nov. 2, 2005 Lecturer: Venkat Guruswami and Ryan O Donnell Scribe: Ioannis

More information

Lecture 16 November 6th, 2012 (Prasad Raghavendra)

Lecture 16 November 6th, 2012 (Prasad Raghavendra) 6.841: Advanced Complexity Theory Fall 2012 Lecture 16 November 6th, 2012 (Prasad Raghavendra) Prof. Dana Moshkovitz Scribe: Geng Huang 1 Overview In this lecture, we will begin to talk about the PCP Theorem

More information

B(w, z, v 1, v 2, v 3, A(v 1 ), A(v 2 ), A(v 3 )).

B(w, z, v 1, v 2, v 3, A(v 1 ), A(v 2 ), A(v 3 )). Lecture 13 PCP Continued Last time we began the proof of the theorem that PCP(poly, poly) = NEXP. May 13, 2004 Lecturer: Paul Beame Notes: Tian Sang We showed that IMPLICIT-3SAT is NEXP-complete where

More information

Almost transparent short proofs for NP R

Almost transparent short proofs for NP R Brandenburgische Technische Universität, Cottbus, Germany From Dynamics to Complexity: A conference celebrating the work of Mike Shub Toronto, May 10, 2012 Supported by DFG under GZ:ME 1424/7-1 Outline

More information

Lecture 8: Linearity and Assignment Testing

Lecture 8: Linearity and Assignment Testing CE 533: The PCP Theorem and Hardness of Approximation (Autumn 2005) Lecture 8: Linearity and Assignment Testing 26 October 2005 Lecturer: Venkat Guruswami cribe: Paul Pham & Venkat Guruswami 1 Recap In

More information

PCP Theorem And Hardness Of Approximation For MAX-SATISFY Over Finite Fields

PCP Theorem And Hardness Of Approximation For MAX-SATISFY Over Finite Fields MM Research Preprints KLMM, AMSS, Academia Sinica Vol. 7, 1 15, July, 008 1 PCP Theorem And Hardness Of Approximation For MAX-SATISFY Over Finite Fields Shangwei Zhao Key Laboratory of Mathematics Mechanization

More information

6.841/18.405J: Advanced Complexity Wednesday, April 2, Lecture Lecture 14

6.841/18.405J: Advanced Complexity Wednesday, April 2, Lecture Lecture 14 6.841/18.405J: Advanced Complexity Wednesday, April 2, 2003 Lecture Lecture 14 Instructor: Madhu Sudan In this lecture we cover IP = PSPACE Interactive proof for straightline programs. Straightline program

More information

2 Completing the Hardness of approximation of Set Cover

2 Completing the Hardness of approximation of Set Cover CSE 533: The PCP Theorem and Hardness of Approximation (Autumn 2005) Lecture 15: Set Cover hardness and testing Long Codes Nov. 21, 2005 Lecturer: Venkat Guruswami Scribe: Atri Rudra 1 Recap We will first

More information

Notes for Lecture 2. Statement of the PCP Theorem and Constraint Satisfaction

Notes for Lecture 2. Statement of the PCP Theorem and Constraint Satisfaction U.C. Berkeley Handout N2 CS294: PCP and Hardness of Approximation January 23, 2006 Professor Luca Trevisan Scribe: Luca Trevisan Notes for Lecture 2 These notes are based on my survey paper [5]. L.T. Statement

More information

Dinur s Proof of the PCP Theorem

Dinur s Proof of the PCP Theorem Dinur s Proof of the PCP Theorem Zampetakis Manolis School of Electrical and Computer Engineering National Technical University of Athens December 22, 2014 Table of contents 1 Introduction 2 PCP Theorem

More information

Lecture 6. k+1 n, wherein n =, is defined for a given

Lecture 6. k+1 n, wherein n =, is defined for a given (67611) Advanced Topics in Complexity: PCP Theory November 24, 2004 Lecturer: Irit Dinur Lecture 6 Scribe: Sharon Peri Abstract In this lecture we continue our discussion of locally testable and locally

More information

On the efficient approximability of constraint satisfaction problems

On the efficient approximability of constraint satisfaction problems On the efficient approximability of constraint satisfaction problems July 13, 2007 My world Max-CSP Efficient computation. P Polynomial time BPP Probabilistic Polynomial time (still efficient) NP Non-deterministic

More information

Lecture 19: Interactive Proofs and the PCP Theorem

Lecture 19: Interactive Proofs and the PCP Theorem Lecture 19: Interactive Proofs and the PCP Theorem Valentine Kabanets November 29, 2016 1 Interactive Proofs In this model, we have an all-powerful Prover (with unlimited computational prover) and a polytime

More information

Introduction Long transparent proofs The real PCP theorem. Real Number PCPs. Klaus Meer. Brandenburg University of Technology, Cottbus, Germany

Introduction Long transparent proofs The real PCP theorem. Real Number PCPs. Klaus Meer. Brandenburg University of Technology, Cottbus, Germany Santaló s Summer School, Part 3, July, 2012 joint work with Martijn Baartse (work supported by DFG, GZ:ME 1424/7-1) Outline 1 Introduction 2 Long transparent proofs for NP R 3 The real PCP theorem First

More information

1 Randomized Computation

1 Randomized Computation CS 6743 Lecture 17 1 Fall 2007 1 Randomized Computation Why is randomness useful? Imagine you have a stack of bank notes, with very few counterfeit ones. You want to choose a genuine bank note to pay at

More information

Sublinear Algorithms Lecture 3

Sublinear Algorithms Lecture 3 Sublinear Algorithms Lecture 3 Sofya Raskhodnikova Penn State University Thanks to Madhav Jha (Penn State) for help with creating these slides. Tentative Plan Lecture. Background. Testing properties of

More information

Lecture 15: A Brief Look at PCP

Lecture 15: A Brief Look at PCP IAS/PCMI Summer Session 2000 Clay Mathematics Undergraduate Program Basic Course on Computational Complexity Lecture 15: A Brief Look at PCP David Mix Barrington and Alexis Maciel August 4, 2000 1. Overview

More information

Complexity Classes V. More PCPs. Eric Rachlin

Complexity Classes V. More PCPs. Eric Rachlin Complexity Classes V More PCPs Eric Rachlin 1 Recall from last time Nondeterminism is equivalent to having access to a certificate. If a valid certificate exists, the machine accepts. We see that problems

More information

Two Query PCP with Sub-Constant Error

Two Query PCP with Sub-Constant Error Electronic Colloquium on Computational Complexity, Report No 71 (2008) Two Query PCP with Sub-Constant Error Dana Moshkovitz Ran Raz July 28, 2008 Abstract We show that the N P-Complete language 3SAT has

More information

1 Probabilistically checkable proofs

1 Probabilistically checkable proofs CSC 5170: Theory of Computational Complexity Lecture 12 The Chinese University of Hong Kong 12 April 2010 Interactive proofs were introduced as a generalization of the classical notion of a proof in the

More information

Approximating MAX-E3LIN is NP-Hard

Approximating MAX-E3LIN is NP-Hard Approximating MAX-E3LIN is NP-Hard Evan Chen May 4, 2016 This lecture focuses on the MAX-E3LIN problem. We prove that approximating it is NP-hard by a reduction from LABEL-COVER. 1 Introducing MAX-E3LIN

More information

20.1 2SAT. CS125 Lecture 20 Fall 2016

20.1 2SAT. CS125 Lecture 20 Fall 2016 CS125 Lecture 20 Fall 2016 20.1 2SAT We show yet another possible way to solve the 2SAT problem. Recall that the input to 2SAT is a logical expression that is the conunction (AND) of a set of clauses,

More information

Building Assignment Testers DRAFT

Building Assignment Testers DRAFT Building Assignment Testers DRAFT Andrew Drucker University of California, San Diego Abstract In this expository paper, we show how to construct Assignment Testers using the Hadamard and quadratic encodings.

More information

Towards the Sliding Scale Conjecture (Old & New PCP constructions)

Towards the Sliding Scale Conjecture (Old & New PCP constructions) Towards the Sliding Scale Conjecture (Old & New PCP constructions) Prahladh Harsha TIFR [Based on joint works with Irit Dinur & Guy Kindler] Outline Intro, Background & Context Goals and questions in this

More information

2 Evidence that Graph Isomorphism is not NP-complete

2 Evidence that Graph Isomorphism is not NP-complete Topics in Theoretical Computer Science April 11, 2016 Lecturer: Ola Svensson Lecture 7 (Notes) Scribes: Ola Svensson Disclaimer: These notes were written for the lecturer only and may contain inconsistent

More information

Complexity Classes IV

Complexity Classes IV Complexity Classes IV NP Optimization Problems and Probabilistically Checkable Proofs Eric Rachlin 1 Decision vs. Optimization Most complexity classes are defined in terms of Yes/No questions. In the case

More information

P versus NP over Various Structures

P versus NP over Various Structures 26th ESSLLI Summer School 2014, Tübingen, August 2014 PART 5: Probabilistically Checkable Proofs jointly with J.A. Makowsky Outline for today 1 Introduction 2 Verifiers and real PCP classes 3 The classical

More information

Hardness of Approximation

Hardness of Approximation CSE 594: Combinatorial and Graph Algorithms Lecturer: Hung Q. Ngo SUNY at Buffalo, Fall 2006 Last update: November 25, 2006 Hardness of Approximation 1 Overview To date, thousands of natural optimization

More information

2 Natural Proofs: a barrier for proving circuit lower bounds

2 Natural Proofs: a barrier for proving circuit lower bounds Topics in Theoretical Computer Science April 4, 2016 Lecturer: Ola Svensson Lecture 6 (Notes) Scribes: Ola Svensson Disclaimer: These notes were written for the lecturer only and may contain inconsistent

More information

HARDNESS AMPLIFICATION VIA SPACE-EFFICIENT DIRECT PRODUCTS

HARDNESS AMPLIFICATION VIA SPACE-EFFICIENT DIRECT PRODUCTS HARDNESS AMPLIFICATION VIA SPACE-EFFICIENT DIRECT PRODUCTS Venkatesan Guruswami and Valentine Kabanets Abstract. We prove a version of the derandomized Direct Product lemma for deterministic space-bounded

More information

Lecture 18: PCP Theorem and Hardness of Approximation I

Lecture 18: PCP Theorem and Hardness of Approximation I Lecture 18: and Hardness of Approximation I Arijit Bishnu 26.04.2010 Outline 1 Introduction to Approximation Algorithm 2 Outline 1 Introduction to Approximation Algorithm 2 Approximation Algorithm Approximation

More information

Lecture 18: Inapproximability of MAX-3-SAT

Lecture 18: Inapproximability of MAX-3-SAT CS 880: Advanced Complexity Theory 3/7/2008 Lecture 18: Inapproximability of MAX-3-SAT Instructor: Dieter van Melkebeek Scribe: Jeff Kinne In this lecture we prove a tight inapproximability result for

More information

NP-Complete problems

NP-Complete problems NP-Complete problems NP-complete problems (NPC): A subset of NP. If any NP-complete problem can be solved in polynomial time, then every problem in NP has a polynomial time solution. NP-complete languages

More information

1 Distributional problems

1 Distributional problems CSCI 5170: Computational Complexity Lecture 6 The Chinese University of Hong Kong, Spring 2016 23 February 2016 The theory of NP-completeness has been applied to explain why brute-force search is essentially

More information

Lecture 26. Daniel Apon

Lecture 26. Daniel Apon Lecture 26 Daniel Apon 1 From IPPSPACE to NPPCP(log, 1): NEXP has multi-prover interactive protocols If you ve read the notes on the history of the PCP theorem referenced in Lecture 19 [3], you will already

More information

Lecture 23: Alternation vs. Counting

Lecture 23: Alternation vs. Counting CS 710: Complexity Theory 4/13/010 Lecture 3: Alternation vs. Counting Instructor: Dieter van Melkebeek Scribe: Jeff Kinne & Mushfeq Khan We introduced counting complexity classes in the previous lecture

More information

Tutorial: Locally decodable codes. UT Austin

Tutorial: Locally decodable codes. UT Austin Tutorial: Locally decodable codes Anna Gál UT Austin Locally decodable codes Error correcting codes with extra property: Recover (any) one message bit, by reading only a small number of codeword bits.

More information

Improved Hardness of Approximating Chromatic Number

Improved Hardness of Approximating Chromatic Number Improved Hardness of Approximating Chromatic Number Sangxia Huang KTH Royal Institute of Technology Stockholm, Sweden sangxia@csc.kth.se April 13, 2013 Abstract We prove that for sufficiently large K,

More information

Lecture 17 November 8, 2012

Lecture 17 November 8, 2012 6.841: Advanced Complexity Theory Fall 2012 Prof. Dana Moshkovitz Lecture 17 November 8, 2012 Scribe: Mark Bun 1 Overview In the previous lecture, we saw an overview of probabilistically checkable proofs,

More information

FOURIER ANALYSIS OF BOOLEAN FUNCTIONS

FOURIER ANALYSIS OF BOOLEAN FUNCTIONS FOURIER ANALYSIS OF BOOLEAN FUNCTIONS SAM SPIRO Abstract. This paper introduces the technique of Fourier analysis applied to Boolean functions. We use this technique to illustrate proofs of both Arrow

More information

Lecture 7: Passive Learning

Lecture 7: Passive Learning CS 880: Advanced Complexity Theory 2/8/2008 Lecture 7: Passive Learning Instructor: Dieter van Melkebeek Scribe: Tom Watson In the previous lectures, we studied harmonic analysis as a tool for analyzing

More information

Lecture 29: Computational Learning Theory

Lecture 29: Computational Learning Theory CS 710: Complexity Theory 5/4/2010 Lecture 29: Computational Learning Theory Instructor: Dieter van Melkebeek Scribe: Dmitri Svetlov and Jake Rosin Today we will provide a brief introduction to computational

More information

Where do pseudo-random generators come from?

Where do pseudo-random generators come from? Computer Science 2426F Fall, 2018 St. George Campus University of Toronto Notes #6 (for Lecture 9) Where do pseudo-random generators come from? Later we will define One-way Functions: functions that are

More information

Questions Pool. Amnon Ta-Shma and Dean Doron. January 2, Make sure you know how to solve. Do not submit.

Questions Pool. Amnon Ta-Shma and Dean Doron. January 2, Make sure you know how to solve. Do not submit. Questions Pool Amnon Ta-Shma and Dean Doron January 2, 2017 General guidelines The questions fall into several categories: (Know). (Mandatory). (Bonus). Make sure you know how to solve. Do not submit.

More information

CSC 5170: Theory of Computational Complexity Lecture 9 The Chinese University of Hong Kong 15 March 2010

CSC 5170: Theory of Computational Complexity Lecture 9 The Chinese University of Hong Kong 15 March 2010 CSC 5170: Theory of Computational Complexity Lecture 9 The Chinese University of Hong Kong 15 March 2010 We now embark on a study of computational classes that are more general than NP. As these classes

More information

Probabilistically Checkable Proofs. 1 Introduction to Probabilistically Checkable Proofs

Probabilistically Checkable Proofs. 1 Introduction to Probabilistically Checkable Proofs Course Proofs and Computers, JASS 06 Probabilistically Checkable Proofs Lukas Bulwahn May 21, 2006 1 Introduction to Probabilistically Checkable Proofs 1.1 History of Inapproximability Results Before introducing

More information

Essential facts about NP-completeness:

Essential facts about NP-completeness: CMPSCI611: NP Completeness Lecture 17 Essential facts about NP-completeness: Any NP-complete problem can be solved by a simple, but exponentially slow algorithm. We don t have polynomial-time solutions

More information

Today. Few Comments. PCP Theorem, Simple proof due to Irit Dinur [ECCC, TR05-046]! Based on some ideas promoted in [Dinur- Reingold 04].

Today. Few Comments. PCP Theorem, Simple proof due to Irit Dinur [ECCC, TR05-046]! Based on some ideas promoted in [Dinur- Reingold 04]. Today Few Comments PCP Theorem, Simple proof due to Irit Dinur [ECCC, TR05-046]! Based on some ideas promoted in [Dinur- Reingold 04]. Remarkably simple novel proof. Leads to new quantitative results too!

More information

CS151 Complexity Theory. Lecture 15 May 22, 2017

CS151 Complexity Theory. Lecture 15 May 22, 2017 CS151 Complexity Theory Lecture 15 New topic(s) Optimization problems, Approximation Algorithms, and Probabilistically Checkable Proofs Optimization Problems many hard problems (especially NP-hard) are

More information

1 The Low-Degree Testing Assumption

1 The Low-Degree Testing Assumption Advanced Complexity Theory Spring 2016 Lecture 17: PCP with Polylogarithmic Queries and Sum Check Prof. Dana Moshkovitz Scribes: Dana Moshkovitz & Michael Forbes Scribe Date: Fall 2010 In this lecture

More information

: On the P vs. BPP problem. 30/12/2016 Lecture 12

: On the P vs. BPP problem. 30/12/2016 Lecture 12 03684155: On the P vs. BPP problem. 30/12/2016 Lecture 12 Time Hierarchy Theorems Amnon Ta-Shma and Dean Doron 1 Diagonalization arguments Throughout this lecture, for a TM M, we denote M t to be the machine

More information

Lecture 21: P vs BPP 2

Lecture 21: P vs BPP 2 Advanced Complexity Theory Spring 206 Prof. Dana Moshkovitz Lecture 2: P vs BPP 2 Overview In the previous lecture, we began our discussion of pseudorandomness. We presented the Blum- Micali definition

More information

Keywords. Approximation Complexity Theory: historical remarks. What s PCP?

Keywords. Approximation Complexity Theory: historical remarks. What s PCP? Keywords The following terms should be well-known to you. 1. P, NP, NP-hard, NP-complete. 2. (polynomial-time) reduction. 3. Cook-Levin theorem. 4. NPO problems. Instances. Solutions. For a long time it

More information

Tolerant Versus Intolerant Testing for Boolean Properties

Tolerant Versus Intolerant Testing for Boolean Properties Tolerant Versus Intolerant Testing for Boolean Properties Eldar Fischer Faculty of Computer Science Technion Israel Institute of Technology Technion City, Haifa 32000, Israel. eldar@cs.technion.ac.il Lance

More information

Postprint.

Postprint. http://www.diva-portal.org Postprint This is the accepted version of a paper presented at 16th International Workshop on Approximation Algorithms for Combinatorial Optimization Problems, APPROX 2013 and

More information

Computational Complexity: Problem Set 4

Computational Complexity: Problem Set 4 Computational Complexity: Problem Set 4 Due: Friday January 8, 16, at 3:59 AoE. Submit your solutions as a PDF le by e-mail to jakobn at kth dot se with the subject line Problem set 4: your full name.

More information

Basic Probabilistic Checking 3

Basic Probabilistic Checking 3 CS294: Probabilistically Checkable and Interactive Proofs February 21, 2017 Basic Probabilistic Checking 3 Instructor: Alessandro Chiesa & Igor Shinkar Scribe: Izaak Meckler Today we prove the following

More information

Randomness and non-uniformity

Randomness and non-uniformity Randomness and non-uniformity JASS 2006 Course 1: Proofs and Computers Felix Weninger TU München April 2006 Outline Randomized computation 1 Randomized computation 2 Computation with advice Non-uniform

More information

Lecture Notes on Linearity (Group Homomorphism) Testing

Lecture Notes on Linearity (Group Homomorphism) Testing Lecture Notes on Linearity (Group Homomorphism) Testing Oded Goldreich April 5, 2016 Summary: These notes present a linearity tester that, on input a description of two groups G,H and oracle access to

More information

DRAFT. Complexity of counting. Chapter 8

DRAFT. Complexity of counting. Chapter 8 Chapter 8 Complexity of counting It is an empirical fact that for many combinatorial problems the detection of the existence of a solution is easy, yet no computationally efficient method is known for

More information

Learning and Fourier Analysis

Learning and Fourier Analysis Learning and Fourier Analysis Grigory Yaroslavtsev http://grigory.us CIS 625: Computational Learning Theory Fourier Analysis and Learning Powerful tool for PAC-style learning under uniform distribution

More information

Compute the Fourier transform on the first register to get x {0,1} n x 0.

Compute the Fourier transform on the first register to get x {0,1} n x 0. CS 94 Recursive Fourier Sampling, Simon s Algorithm /5/009 Spring 009 Lecture 3 1 Review Recall that we can write any classical circuit x f(x) as a reversible circuit R f. We can view R f as a unitary

More information

Lecture 5: Derandomization (Part II)

Lecture 5: Derandomization (Part II) CS369E: Expanders May 1, 005 Lecture 5: Derandomization (Part II) Lecturer: Prahladh Harsha Scribe: Adam Barth Today we will use expanders to derandomize the algorithm for linearity test. Before presenting

More information

Lecture 3 (Notes) 1. The book Computational Complexity: A Modern Approach by Sanjeev Arora and Boaz Barak;

Lecture 3 (Notes) 1. The book Computational Complexity: A Modern Approach by Sanjeev Arora and Boaz Barak; Topics in Theoretical Computer Science March 7, 2016 Lecturer: Ola Svensson Lecture 3 (Notes) Scribes: Ola Svensson Disclaimer: These notes were written for the lecturer only and may contain inconsistent

More information

Testing Low-Degree Polynomials over GF (2)

Testing Low-Degree Polynomials over GF (2) Testing Low-Degree Polynomials over GF (2) Noga Alon Tali Kaufman Michael Krivelevich Simon Litsyn Dana Ron July 9, 2003 Abstract We describe an efficient randomized algorithm to test if a given binary

More information

Lecture 12: Interactive Proofs

Lecture 12: Interactive Proofs princeton university cos 522: computational complexity Lecture 12: Interactive Proofs Lecturer: Sanjeev Arora Scribe:Carl Kingsford Recall the certificate definition of NP. We can think of this characterization

More information

Three Query Locally Decodable Codes with Higher Correctness Require Exponential Length

Three Query Locally Decodable Codes with Higher Correctness Require Exponential Length Three Query Locally Decodable Codes with Higher Correctness Require Exponential Length Anna Gál UT Austin panni@cs.utexas.edu Andrew Mills UT Austin amills@cs.utexas.edu March 8, 20 Abstract Locally decodable

More information

Lecture 4: LMN Learning (Part 2)

Lecture 4: LMN Learning (Part 2) CS 294-114 Fine-Grained Compleity and Algorithms Sept 8, 2015 Lecture 4: LMN Learning (Part 2) Instructor: Russell Impagliazzo Scribe: Preetum Nakkiran 1 Overview Continuing from last lecture, we will

More information

Lecture 5: February 16, 2012

Lecture 5: February 16, 2012 COMS 6253: Advanced Computational Learning Theory Lecturer: Rocco Servedio Lecture 5: February 16, 2012 Spring 2012 Scribe: Igor Carboni Oliveira 1 Last time and today Previously: Finished first unit on

More information

Limits to Approximability: When Algorithms Won't Help You. Note: Contents of today s lecture won t be on the exam

Limits to Approximability: When Algorithms Won't Help You. Note: Contents of today s lecture won t be on the exam Limits to Approximability: When Algorithms Won't Help You Note: Contents of today s lecture won t be on the exam Outline Limits to Approximability: basic results Detour: Provers, verifiers, and NP Graph

More information

PCPs and Inapproximability Gap-producing and Gap-Preserving Reductions. My T. Thai

PCPs and Inapproximability Gap-producing and Gap-Preserving Reductions. My T. Thai PCPs and Inapproximability Gap-producing and Gap-Preserving Reductions My T. Thai 1 1 Hardness of Approximation Consider a maximization problem Π such as MAX-E3SAT. To show that it is NP-hard to approximation

More information

Tolerant Versus Intolerant Testing for Boolean Properties

Tolerant Versus Intolerant Testing for Boolean Properties Electronic Colloquium on Computational Complexity, Report No. 105 (2004) Tolerant Versus Intolerant Testing for Boolean Properties Eldar Fischer Lance Fortnow November 18, 2004 Abstract A property tester

More information

Notes on Complexity Theory Last updated: December, Lecture 2

Notes on Complexity Theory Last updated: December, Lecture 2 Notes on Complexity Theory Last updated: December, 2011 Jonathan Katz Lecture 2 1 Review The running time of a Turing machine M on input x is the number of steps M takes before it halts. Machine M is said

More information

Quasi-Random PCP and Hardness of 2-Catalog Segmentation

Quasi-Random PCP and Hardness of 2-Catalog Segmentation Quasi-Random PCP and Hardness of 2-Catalog Segmentation Rishi Saket Carnegie Mellon University rsaket@cs.cmu.edu ABSTRACT. We study the problem of 2-Catalog Segmentation which is one of the several variants

More information

Local list-decoding and testing of random linear codes from high-error

Local list-decoding and testing of random linear codes from high-error Local list-decoding and testing of random linear codes from high-error Swastik Kopparty Shubhangi Saraf February 4, 01 Abstract In this paper, we give efficient algorithms for list-decoding and testing

More information

Lec. 11: Håstad s 3-bit PCP

Lec. 11: Håstad s 3-bit PCP Limits of Approximation Algorithms 15 April, 2010 (TIFR) Lec. 11: Håstad s 3-bit PCP Lecturer: Prahladh Harsha cribe: Bodhayan Roy & Prahladh Harsha In last lecture, we proved the hardness of label cover

More information

Composition of low-error 2-query PCPs using decodable PCPs

Composition of low-error 2-query PCPs using decodable PCPs Composition of low-error 2-query PCPs using decodable PCPs Irit Dinur Prahladh Harsha August 5, 2009 Abstract The main result of this paper is a generic composition theorem for low error two-query probabilistically

More information

6.045: Automata, Computability, and Complexity (GITCS) Class 17 Nancy Lynch

6.045: Automata, Computability, and Complexity (GITCS) Class 17 Nancy Lynch 6.045: Automata, Computability, and Complexity (GITCS) Class 17 Nancy Lynch Today Probabilistic Turing Machines and Probabilistic Time Complexity Classes Now add a new capability to standard TMs: random

More information

NP-hardness of coloring 2-colorable hypergraph with poly-logarithmically many colors

NP-hardness of coloring 2-colorable hypergraph with poly-logarithmically many colors Electronic Colloquium on Computational Complexity, Report No. 73 (2018) NP-hardness of coloring 2-colorable with poly-logarithmically many colors Amey Bhangale April 21, 2018 Abstract We give very short

More information

Probabilistically checkable proofs

Probabilistically checkable proofs Probabilistically checkable proofs Madhu Sudan MIT CSAIL, 32 Vassar Street, Cambridge, MA 02139, USA ABSTRACT Can a proof be checked without reading it? That certainly seems impossible, no matter how much

More information

1 AC 0 and Håstad Switching Lemma

1 AC 0 and Håstad Switching Lemma princeton university cos 522: computational complexity Lecture 19: Circuit complexity Lecturer: Sanjeev Arora Scribe:Tony Wirth Complexity theory s Waterloo As we saw in an earlier lecture, if PH Σ P 2

More information

ITCS:CCT09 : Computational Complexity Theory Apr 8, Lecture 7

ITCS:CCT09 : Computational Complexity Theory Apr 8, Lecture 7 ITCS:CCT09 : Computational Complexity Theory Apr 8, 2009 Lecturer: Jayalal Sarma M.N. Lecture 7 Scribe: Shiteng Chen In this lecture, we will discuss one of the basic concepts in complexity theory; namely

More information

Show that the following problems are NP-complete

Show that the following problems are NP-complete Show that the following problems are NP-complete April 7, 2018 Below is a list of 30 exercises in which you are asked to prove that some problem is NP-complete. The goal is to better understand the theory

More information

Notes on Complexity Theory Last updated: November, Lecture 10

Notes on Complexity Theory Last updated: November, Lecture 10 Notes on Complexity Theory Last updated: November, 2015 Lecture 10 Notes by Jonathan Katz, lightly edited by Dov Gordon. 1 Randomized Time Complexity 1.1 How Large is BPP? We know that P ZPP = RP corp

More information

1 Agenda. 2 History. 3 Probabilistically Checkable Proofs (PCPs). Lecture Notes Definitions. PCPs. Approximation Algorithms.

1 Agenda. 2 History. 3 Probabilistically Checkable Proofs (PCPs). Lecture Notes Definitions. PCPs. Approximation Algorithms. CS 221: Computational Complexity Prof. Salil Vadhan Lecture Notes 20 April 12, 2010 Scribe: Jonathan Pines 1 Agenda. PCPs. Approximation Algorithms. PCPs = Inapproximability. 2 History. First, some history

More information

CS286.2 Lecture 8: A variant of QPCP for multiplayer entangled games

CS286.2 Lecture 8: A variant of QPCP for multiplayer entangled games CS286.2 Lecture 8: A variant of QPCP for multiplayer entangled games Scribe: Zeyu Guo In the first lecture, we saw three equivalent variants of the classical PCP theorems in terms of CSP, proof checking,

More information

Great Theoretical Ideas in Computer Science

Great Theoretical Ideas in Computer Science 15-251 Great Theoretical Ideas in Computer Science Lecture 28: A Computational Lens on Proofs December 6th, 2016 Evolution of proof First there was GORM GORM = Good Old Regular Mathematics Pythagoras s

More information

Non-Approximability Results (2 nd part) 1/19

Non-Approximability Results (2 nd part) 1/19 Non-Approximability Results (2 nd part) 1/19 Summary - The PCP theorem - Application: Non-approximability of MAXIMUM 3-SAT 2/19 Non deterministic TM - A TM where it is possible to associate more than one

More information

Computational Complexity: A Modern Approach. Draft of a book: Dated January 2007 Comments welcome!

Computational Complexity: A Modern Approach. Draft of a book: Dated January 2007 Comments welcome! i Computational Complexity: A Modern Approach Draft of a book: Dated January 2007 Comments welcome! Sanjeev Arora and Boaz Barak Princeton University complexitybook@gmail.com Not to be reproduced or distributed

More information

CPSC 536N: Randomized Algorithms Term 2. Lecture 9

CPSC 536N: Randomized Algorithms Term 2. Lecture 9 CPSC 536N: Randomized Algorithms 2011-12 Term 2 Prof. Nick Harvey Lecture 9 University of British Columbia 1 Polynomial Identity Testing In the first lecture we discussed the problem of testing equality

More information

PCP Soundness amplification Meeting 2 ITCS, Tsinghua Univesity, Spring April 2009

PCP Soundness amplification Meeting 2 ITCS, Tsinghua Univesity, Spring April 2009 PCP Soundness amplification Meeting 2 ITCS, Tsinghua Univesity, Spring 2009 29 April 2009 Speaker: Andrej Bogdanov Notes by: Andrej Bogdanov Recall the definition of probabilistically checkable proofs

More information