On the NP-Hardness of Bounded Distance Decoding of Reed-Solomon Codes

Size: px
Start display at page:

Download "On the NP-Hardness of Bounded Distance Decoding of Reed-Solomon Codes"

Transcription

1 On the NP-Hardness of Bounded Distance Decoding of Reed-Solomon Codes Venkata Gandikota Purdue Universit Badih Ghazi MIT Elena Grigorescu Purdue Universit Abstract Guruswami and Vard (IEEE Trans. Inf. Theor, 005) show that given a Reed-Solomon code over a finite field F, of length n and dimension t, and given a target vector v F n, it is NP-hard to decide if there is a codeword that disagrees with v on at most n t 1 coordinates. Understanding the complexit of this Bounded Distance Decoding problem as the amount of error in the target decreases is an important open problem in the stud of Reed-Solomon codes. In this work, we extend the result of Guruswami and Vard b proving that it is NP-hard to decide the existence of a codeword that disagrees with v on n t, and on n t 3 coordinates. No other NP-hardness results were known before for an amount of error < n t 1. The core of our proofs is showing the NP-hardness of a parameterized generalization of the Subset-Sum problem to higher degrees (called Moments Subset-Sum) that ma be of independent interest. I. INTRODUCTION A linear error-correcting code of length n and dimension t, over a finite field alphabet F, is a vector space C F n of dimension t. The Hamming distance between x, F n is δ(x, ) := {i [n] : x i i }, and the minimum distance of C is λ(c) := min x C δ(x, ). In the Bounded Distance Decoding problem with parameter d, we are given a code C F n and a target vector v F n, and we are asked to decide whether there exists a codeword c C such that the Hamming distance δ(v, c) e(d, λ(c)), where e(d, ) is an error-weight function of interest. This is a fundamental question in the stud of general error-correcting codes, and its complexit is not full understood even for wellstudied codes such as Reed-Solomon (RS) codes. More precisel, RS codes still exhibit a wide gap between the setting of small error-weight, where the problem is solvable in polnomial-time [Sud97], [GS99], and the setting of large error-weight, where the problem is known to be NP-hard [GV05]. In this work, we improve this gap b generalizing the decade-old NP-hardness results of [GV05] to smaller error parameters. A Reed-Solomon code of length n, dimension t, defined over a finite field F, and specified b an evaluation set D = {x 1, x,..., x n } F is the set RS D,t = { f(x 1 ),..., f(x n ) : x 1,..., x n D, f(x) F[x], deg(f(x)) t 1}. Its minimum distance is λ = n t + 1. We are interested in the Bounded Distance Decoding problem for RS codes with parameter d (denoted RS-BDD d ) corresponding to the error-weight function e(d, λ) = λ d 1 = n t d. When e n nt (i.e., the Johnson radius ), the list-decoding algorithms of [Sud97], [GS99] can solve RS-BDD nt t in polnomial time. At the other end of the spectrum, if e = n t one can easil interpolate a degree t 1 polnomial that agrees with the target on a set of t arbitrar entries. The famous result of [GV05] shows that right below this value, i.e., when e = n t 1, RS-BDD 1 is NP-hard. Their proof is via a reduction from the 3D-matching problem, and it does not impl an hardness results for smaller values of the error-weight parameter. In the range where e < n t 1, the onl known hardness result is due to [CW10] who show a reduction from the Discrete Log problem, when the evaluation set is D = F q, for e 3 (n t + 1). Note that the hardness of Discrete Log is a stronger complexit-theoretic assumption than P NP. In particular, the Discrete Log problem over finite fields is not believed to be NP-hard and [Sho97] gives a polnomial-time quantum algorithm solving it. In this work, we prove that for ever d {, 3}, the RS-BDD d problem is NP-hard. We note that, as is the case of [GV05], our reductions require that n be pollogarithmic in F. Our proof starts with the observation that an extension of the Subset-Sum problem up to d moments (called Moments Subset-Sum with parameter d) is polnomial-time reducible to RS-BDD d. The crux of our proof is showing the NP-hardness of the Moments Subset-Sum problem, formall defined next. Definition 1 (Moments Subset-Sum: MSS d ). Given a set A = {a 1, a,..., a n } F n, integer k, and m 1, m,..., m d F, decide if there exists a subset S A of size k, satisfing s S si = m i for all i [d]. Note that MSS 1 is the usual Subset-Sum problem, which is in fact used b [CM07] to show an alternate

2 proof of [GV05]. The NP-hardness of Subset-Sum can be shown b a well-known reduction from 3-SAT. Surprisingl, it turns out to be much more difficult to prove NP-hardness for MSS d for values of d. Intuitivel, this is because the reduction from 3-SAT to Subset-Sum encodes satisfiabilit of a 3-SAT formula in the decimal representation of the integers of the Subset- Sum instance, and it becomes more difficult to control the decimal representations when constraints involving squares and higher powers are introduced. In fact, the current barrier to extending our proof approach to show the NP-hardness of MSS d for larger values of d (and thereb obtain the NP-hardness of RS- BDD d for larger values of d) is the following intriguing algebraic question. Question 1. Given a finite field F, a, b F, and d N, does there exist t = t(d) and explicit x 1, x,..., x t, 1,,..., t F satisfing x 1 + x + t t...+x t = t and a i + x i j = b i + for ever i {,..., d}? 1 j=1 j=1 For d {, 3}, we are able to answer this question in the affirmative and to provide explicit constructions over domains that are either finite fields of large characteristic, the rational numbers or the ring of integers. These constructions form the starting point of our NP-hardness proofs. II. REDUCTION FROM MOMENTS SUBSET SUM We start b reformulating the RS-BDD problem as a polnomial reconstruction question as follows. Definition (RS-BDD d ). Given a set of n distinct points in F, D = {(x 1, 1 ), (x, ),..., (x n, n )}, and an integer t < n, decide if there exists a polnomial f(x) F[x] of degree at most t 1 passing through at least t + d points in D. Here, the set of evaluation points of the code is D = {x 1,... x n } and the target vector is = ( 1,..., n ) F n. Note that if a polnomial f(x) passes through at least t+d points in D, then the corresponding codeword f(x 1 ),..., f(x n ) is at a Hamming distance of at most e = n t d from. We will reduce from the following problem which can be easil seen to be equivalent to MSS d over large prime finite fields F using Newton s identities [Sta99]. We note that this connection has been previousl made (e.g. [LW08]). Definition 3 (Smmetric Subset-Sum (SSS d )). Given a set of n distinct elements of F, A = {a 1, a,..., a n }, 1 We note that the same question is also of interest when a, b, x 1, x,..., x t, 1,,..., t are rational numbers or integers. i j integer k, and B 1, B,... B d F, decide if there exists a subset S of A of size k, such that for ever i [d] the elementar smmetric sums of the elements of S = {s 1,..., s k } satisf E i (S) = 1 j s 1<j < <j i k j 1... s ji = B i. We defer the proof of the reduction from SSS d (and hence from MSS d ) to RS-BDD d to Lemma 6 in Appendix A. III. NP-HARDNESS OF MSS Theorem 4. MSS is NP-hard. Proof: We present the proof for the case where the domain is the ring of integers, and then observe that the proof easil extends to an sufficientl large prime field (see the end of the proof for the details). We give a polnomial-time reduction from the 1-in-3- SAT problem in which we are given a 3-SAT formula φ on n variables and m clauses and are asked to determine if there exists an assignment x {0, 1} n satisfing exactl one literal in each clause. It is known that this problem is NP-hard even for m = O(n) [Sch78]. We start b recalling the reduction from 1-in-3-SAT to Subset-Sum which will be used in our reduction to MSS. In that reduction, each variable (x i, x i ) is mapped to integers a i (corresponding to x i ) and b i (corresponding to x i ). The integers a i and b i and the target B are defined in terms of their length-(n + m) Σ-ar representation (for some sufficientl large even constant, sa Σ = 4) as follows: The Σ-ar representatios of a i and b i consist of parts: a variable region consisting of the leftmost n digits and a clause region consisting of the (remaining) rightmost m digits. In the variable region, a i and b i have a 1 at the ith digit and 0 s at the other digits. In the clause region, for ever j [m], a i (resp. b i ) has a 1 at the jth location if x i (resp. x i ) appears in clause j, and a 0 otherwise. The target B is set to the integer whose Σ-ar representation is the all 1 s. Those Σ-ar representations are illustrated in Figure 1. n Σ-ar digits variable region m Σ-ar digits clause region Target: B = Fig. 1. Σ-ar representations in the original reduction from 1-in-3- SAT to Subset-Sum.

3 This reduction to Subset-Sum can be seen to be complete and sound. We now use it to give a reduction to MSS. In this reduction, each variable (x i, x i ) is mapped to 6 integers a i,1, a i,, a (corresponding to x i ) and b i,1, b i,, b (corresponding to x i ). Let {a i, b i : i [n]} be the integers produced b the above reduction to Subset-Sum. We denote b a v i (resp. a c i ) the Σ-ar representation of the variable (resp. clause) region of a i. For an Σ-ar representation x of a natural number, let (x) Σ be the natural number whose Σ -representation is x. For example, if x is the Σ-ar number (10011), then (x) Σ = Σ 4 +Σ +1. Denote b 1 l the concatenation of l ones. Let ν and h be natural numbers to be specified later on. The integers a i,1, a i,, a, b i,1, b i,, b and the targets B 1 and B are defined as follows: a i,1 = Σ ν+m+h 1 (a v i ) Σ + h Σν (a c i ) Σ b i,1 = Σ ν+m+h 1 (b v i ) Σ + h Σν (b c i ) Σ a i, = a i,1 b i,1 4Σ Σi i and a = a i,. b i, = a i,1 b i,1 4Σ + Σi i and b = b i,. B 1 = Σ ν+m+h 1 (1 n ) Σ h + Σ ν (1 m ) Σ n B = a i,1 + a i, + a. Note that a i,1 (resp. a i, ) defined above can be seen as obtained b inserting h 1 consecutive 0 s in the variable region of the Σ-ar representation of a i (resp. b i ), and then inserting ν zeros at the right. Those Σ-ar representations are illustrated in Figure. Moreover, observe that a i,, a, b i,, b are defined above in such a wa that a i, + a = b i, + b = 0 and a i,1 + a i, + a = b i,1 + b i, + b. Note that this reduction runs in time polnomial in n, m, h and ν. We next prove the correctness of the reduction. a) Completeness: Assume that the starting 3-SAT formula has a satisfing 1-in-3-SAT assignment x. Consider the subset S = :x{a i,1, a i,, a } :xi=0{b i,1, b i,, b } of size k = 3n. We now check that the first moments of S equal B 1 and B. = a i,1 + a i, + a + b i,1 + b i, + b S : x i =1 = = + = Σ ν+m+h 1 ( a i,1 + : x i =0 b i,1 Σ ν+m+h 1 (a v i ) Σ h + Σ ν (a c i) Σ Σ ν+m+h 1 (b v i ) Σ h + Σ ν (b c i) Σ a v i + b v i ) Σ h + Σ ν ( a c i + b c i) Σ = Σ ν+m+h 1 (1 n ) Σ h + Σ ν (1 m ) Σ = B 1 Furthermore, = S + a i,1 + a i, + a b i,1 + b i, + b = a i,1 + a i, + a = B where we used the fact that a i,1 + a i, + a = b i,1 + b i, + b for ever i [n]. b) Soundness: Assume that S is a satisfing subset of the MSS instance. We will use S in order to construct a 1-in-3-SAT satisfing assignment to the starting 3-SAT instance φ. Let s first sketch the high-level intuition of the proof. First, we argue that S should contain the same number of positive and negative integers from the set {a 1,, b 1,, a 1,3, b 1,3 }. This is because these four integers have roughl the same absolute value, which turns out to be much larger than B 1 and than an other possible integer in S. Thus, unless S contains the same number of positive and negative elements from {a 1,, b 1,, a 1,3, b 1,3 }, the integers in S cannot add up to B 1. Then, we show using an inductive argument that for each i [n], S contains the same number of positive and negative elements from {a i,, b i,, a, b } (i.e., Lemma 1). We next prove that, in fact, the elements of S from the set n {a i,, b i,, a, b } exactl cancel each other out, i.e., the add up to 0. Hence, we obtain that the integers of S from n {a i,1, b i,1 } add up to B 1, at which point we can run the soundness analsis of the original reduction from 1-in-3-SAT to Subset Sum in order to construct an assignment satisfing exactl one litteral in each clause. We now give the formal proof, which starts with the following lemma whose proof appears in Appendix B. We assume henceforth that ν 10(m + nh) and h 10m. Lemma 1. For ever i [n], S {a i,, b i, } = S {a, b }. Lemma 1 implies that for ever i [n], = r i Σ i for some r i S {a i,,b i,,a,b } { 1, 0, 1}. The next lemma, whose proof appears in Appendix B, argues that in fact each r i equals 0. Lemma. For ever i [n], r i = 0. 3

4 nh Σ-ar digits m Σ-ar digits ν Σ-ar digits large components region variable region clause region shift region 1st moment: B 1 = Fig.. Σ-ar representations in the reduction from 1-in-3-SAT to MSS. In this figure, h = 3. The large components region onl contains zeros in {a i,1, b i,1 : i [n]} but contains non-zeros in { a i,, b i, : i [n]}. Lemma implies that = 0 S n {ai,,bi,,a,b} and hence that = B 1. We can S n {ai,1,bi,1} now carr out the soundness analsis of the original reduction from 1-in-3-SAT to Subset Sum in order to construct an assignmnent that satisfies exactl one litteral in each clause of the given 3-SAT formula. This concludes the soundness analsis of our reduction. To sum up, setting h = 10m, ν = 10(m + nh) and Σ to be a sufficientl large even constant (sa 4) ields a polnomial-time reduction from 1-in-3-SAT to MSS. Hence, MSS is NP-hard. We now extend the proof to an sufficientl large prime field. Let p cn be a prime number with c some absolute constant. This ensures that the magnitudes of all integers appearing in the above proof are < p/. Performing the above computations modulo p, we can carr out all the arguments as in the case of the integers, and hence the proof holds over F p. IV. NP-HARDNESS OF MSS 3 Theorem 5. MSS 3 is NP-hard. Proof: We present the proof over the field of rational numbers, and then observe that the proof easil extends to an sufficientl large prime field (see the end of the proof for the details). We give a polnomial-time reduction from the 1- in-3-sat problem in which we are given a 3-SAT formula φ on n variables and m clauses and are asked to determine whether there exists an assignment x {0, 1} n that satisfies exactl one literal in each clause. It is known that this problem is NP-hard even for m = O(n) [Sch78]. Recall the known reduction from 1-in-3-SAT to Subset-Sum that is described at the beginning of the proof of Theorem 4. Let a i and b i be the positive integers corresponding to variable (x i, x i ) and let B be the target positive integer in that reduction. As before the Σ-ar representations of the a i s, the b i s and B are illustrated in Figure 1. We now use this reduction to reduce 1-in-3-SAT to MSS 3. In the new reduction, each variable (x i, x i ) is mapped to 6 rational numbers a i,1, a i,, a (corresponding to x i ) and b i,1, b i,, b (corresponding to x i ). The smbols a v i, a c i and (x) Σ are defined as in the proof of Theroem 4. Let ν and h be natural numbers to be specified later on. The rational numbers a i,1, a i,, a, b i,1, b i,, b and the targets B 1, B and B 3 are defined as follows: a i,1 = Σ ν+m+h 1 (a v i ) Σ h + Σν (a c i ) Σ b i,1 = Σ ν+m+h 1 (b v i ) Σ h + Σν (b c i ) Σ Define β i := Σ i, γ i := a i,1 b i,1 β i and α i := a 3 i,1 b 3 i,1 6β iγ i. a i, = α i + γi βi... βi. a = α i γi + βi b i, = α i + γi + βi b = α i γi B 1 = Σ ν+m+h 1 (1 n ) Σ h + Σ ν (1 m ) Σ + n a i, + a. B = B 3 = n n a i,1 + a. a 3 i,1 + a 3 i, + a 3. Note that a i,1 and b i,1 are positive integers defined as in the proof of Theroem 4 and, in particular, their Σ-ar representations are identical to those illustrated in Figure for the reduction from 1-in-3-SAT to MSS. Note that this reduction runs in time polnomial in n, m, h and ν. We next prove the correctness of the reduction. c) Completeness: The completeness analsis uses the next proposition whose proof appears in Appendix C. Proposition 1. For ever i [n], the quantities a i,, a, b i,, b defined above satisf a i, + a = b i, + b a i,1 + a = b i,1 + b i, + b a 3 i,1 + a 3 i, + a 3 = b 3 i,1 + b 3 i, + b 3 Assume that the starting 3 SAT formula has a satisfing 1-in-3-SAT assignment x. Consider the subset S = :x{a i,1, a i,, a } :xi=0{b i,1, b i,, b } of size k = 3n. In Appendix C, we use Proposition 1 to check that the first 3 moments of S equal B 1, B and B 3 respectivel. 4

5 d) Soundness: Assume that S is a satisfing subset of the MSS 3 instance. We will use S in order to construct a 1-in-3-SAT satisfing assignment to the starting 3- SAT formula φ. Let s first sketch the high-level intuition of the proof. First, we prove using an inductive argument (i.e., Lemma 3) that, for each i [n], S should contain the same number of positive and negative rational numbers from the set {a i,, b i,, a, b }. This is because these four numbers have roughl the same absolute value, which turns out to be much larger than B 1 and than an other possible number in S. Thus, unless S contains the same number of positive and negative elements from {a i,, b i,, a, b }, the elements of S cannot add up to B 1. Next, we show using another inductive argument (i.e., Lemma 4) that, for ever i [n], S should contain exactl two elements from the set {a i,, b i,, a, b }. This is because otherwise, the sum of squares of the elements in S {a i,, b i,, a, b } would be ver far from a i, +a, which would impl that the sum of squares of the elements in S is ver far from B. We then show (in Lemma 5) that, in fact, the elements of S {a i,, b i,, a, b } exactl add up to α i ; namel, the β i and γ i terms cancel each other out. Hence, we obtain that the elements of S from n {a i,1, b i,1} add up to B 1 α i = Σ ν+m+h 1 (1 n ) Σ h+σ ν (1 m ) Σ, at which point we can run the soundness analsis of the original reduction from 1-in-3-SAT to Subset Sum in order to construct an assignment satisfing exactl one literal in each clause. We now give the formal proof which uses the following lemmas whose proofs appear in Appendix C. We set ν = 10(m + nh) and h = 10m. Lemma 3. i [n], S {a i,, b i,} = S {a, b }. Lemma 4. i [n], S {a i,, b i,, a, b } =. n Lemma 5. = α i. S n {a i,,b i,,a,b } Lemmas 3, 4 and 5 impl that S n {a i,1,b i,1} = Σ ν+m+h 1 (1 n ) Σ h + Σ ν (1 m ) Σ. We now carr out the soundness analsis of the original reduction from 1-in- 3-SAT to Subset Sum to construct an assignmnent that satisfies exactl one literal in each clause of the given 3-SAT formula. This concludes our soundness analsis. Thus, setting Σ to be a sufficientl large even constant (sa 4) ields a polnomial-time reduction from 1-in-3- SAT to MSS 3. Hence, MSS 3 is NP-hard. The proof also holds over the ring of integers b first multipling the numbers {a i,j, b i,j }, B 1, B, B 3 b the least common multiple of the denominators of {α i, γ i /, α i /}. This preserves the moment constraints since the are homogeneous equations. Let c = O(1) and p > cn3 be a prime number such that all integers appearing in this proof are < p/. The proof extends to F p b performing all computations modulo p. V. CONCLUSION In this work, we proved that RS-BDD and RS-BDD 3 are NP-hard. The main open problem raised b our work is to understand the limits of our approach. In particular, can one design explicit constructions satisfing the properties in Question 1, and use them to prove the NPhardness of RS-BDD d for larger values of d? Finall, we remark that a positive answer to Question 1 could ield to a better understanding of the structure of BCH codes over large fields, and to their the local testabilit properties (e.g., [GK1].) ACKNOWLEDGMENT The authors would like to thank Amir Abboud, Swastik Koppart, Madhu Sudan and Andrew Sutherland for ver helpful discussions and pointers. [CM07] REFERENCES Qi Cheng and Elizabeth Murra. On deciding deep holes of Reed-Solomon codes. In TAMC 007, Shanghai, China, pages , 007. [CW10] Qi Cheng and Daqing Wan. Complexit of decoding positive-rate primitive Reed-Solomon codes. IEEE Transactions on Information Theor, 56(10):517 5, 010. [GK1] Elena Grigorescu and Tali Kaufman. Explicit low-weight bases for BCH codes. IEEE Transactions on Information Theor, 58(1):78 81, 01. [GS99] Venkatesan Guruswami and Madhu Sudan. Improved decoding of reed-solomon and algebraic-geometr codes. IEEE Transactions on Information Theor, 45(6): , [GV05] Venkatesan Guruswami and Alexander Vard. Maximumlikelihood decoding of Reed-Solomon codes is NP-hard. IEEE Transactions on Information Theor, 51(7):49 56, 005. [LW08] Jiou Li and Daqing Wan. On the subset sum problem over finite fields. Finite Fields and Their Applications, 14(4):911 99, 008. [Sch78] [Sho97] [Sta99] [Sud97] Thomas J Schaefer. The complexit of satisfiabilit problems. In Proceedings of the tenth annual ACM smposium on Theor of computing, pages ACM, Peter W Shor. Polnomial-time algorithms for prime factorization and discrete logarithms on a quantum computer. SIAM Journal on Computing, 6(5): , R P Stanle. Enumerative Combinatorics, vol.. Cambridge Universit Press, Madhu Sudan. Decoding of Reed Solomon codes beond the error-correction bound. J. Complexit, 13(1): ,

6 A. Proofs from Section II APPENDIX Lemma 6. SSS d is polnomial-time reducible to RS- BDD d. Proof: Henceforth, let q := F. Given an instance A, k, B 1, B,..., B d of SSS d, we construct an instance D, t of RS-BDD d such that there exists a polnomial f(x) F q [X] of degree at most t 1 which agrees with at least t + d points of D if and onl if there is a solution to the given instance of SSS d. Here, A = {a 1, a,..., a n } is a set of distinct, nonzero elements of F q, B 1, B,..., B d F q and k Z. Let t = k d + 1. Define the degree d polnomial p(x) := x d B 1 x d ( 1) d 1 B d 1 x. For each a i of A, define an element of F q as i = p(a i ) The set D is then given b D = {(a 1 i, i ) for all a i A} {(0, ( 1) d B d )}. Note that D, t is an instance of RS-BDD d which can be constructed in polnomial time given the instance A, k, B 1,..., B d of SSS d. Let S be the solution to SSS d. We now show that there exists a polnomial of degree at most k d which agrees with D in at least k + 1 points. Define the following degree k polnomial, g(x) := (x a i ) = c 0 + c 1 x + + c k 1 x k 1 + x k a i S The coefficients of this polnomial are the smmetric sums of the roots of g(x). Therefore, c k d = ( 1) d B d,..., c k = B, and c k 1 = B 1. Now define, f(x) = (x k g(1/x) x d p(1/x))/x d = c 0 x k d + c 1 x k d c k d and note that f(x) has degree k d = t 1. Also, the constant term of this polnomial is c k d = ( 1) d B d. Hence, f(0) = ( 1) d B d and since g(a i ) = 0, for all a i S, it follows that f(a 1 i ) = p(a i ) = i for all a i S. Therefore, f(x) agrees with k + 1 = t + d points in D. Conversel, we now show that if there is a polnomial f(x) of degree at most t 1 which agrees with t + d points in D, then there is a solution to SSS d. We first observe that if a degree t 1 polnomial passes through t + d points of D, then it has to pass through (0, ( 1) d B d ). To show this, assume f(x) agrees with t + d points of the form (a 1 i, i ) D. Let g(x) be a t + d 1 degree polnomial defined as, g(x) = x t 1 (f(1/x) + p(x)) Therefore, if f(x) = c 0 + c 1 x + + c t 1 x t 1, g(x) can be written as g(x) = x t+d 1 + B 1 x t+d + + ( 1) d 1 B d 1 x t + c 0 x t 1 + c 1 x t + + c t 1 Since, we know that f(a 1 i ) = i = p(a i ) for t + d points, we have b defintion that g(a i ) = 0 for these t + d a is. This is a contradiction since g(x) has degree at most t+d 1 and it cannot have t+d roots. Therefore, f(0) = c 0 = ( 1) d B d. Also, g(x) has t + d 1 = k roots which have their first d smmetric sums equal to B 1, B,..., B d respectivel. Hence, there exists a solution to the given instance of SSS d. B. Proofs from Section III We now prove Lemma 1. To do so, we need the following lemma whose proof is deferred to the end of the section. Lemma 7. Let j 1 be an integer and assume that S {a j,, b j, } = S {a j,3, b j,3 }. Furthermore, assume that if j, then S {a i,, b i, } = S {a, b } for all i < j. Then, we have the following two inequalities: (i) Ω(Σν n ). (ii) S {a j,,b j,,a j,3,b j,3} S {a j,,b j,,a j,3,b j,3} S\{a j,,b j,,a j,3,b j,3} We are now read to prove Lemma 1. ΣΩ(min(ν,h)). Proof of Lemma 1: We proceed b induction on i [n]. At the jth step of the induction (with j ), we assume that S {a i,, b i, } = S {a, b } for all i < j and we need to show that S {a j,, b j, } = S {a j,3, b j,3 }. Assume for the sake of contradiction that S {a j,, b j, } S {a j,3, b j,3 }. Then, Lemma 7 and the fact that for an a, b R, a b max( a, b ) min( a, b ) impl that S = + S {a j,,b j,,a j,3,b j,3} S\{a j,,b j,,a j,3,b j,3} S {a j,,b j,,a j,3,b j,3} S\{a j,,b j,,a j,3,b j,3} 6

7 1 (1 Σ ) Ω(min(ν,h)) = Ω(Σ ν n ) S {a j,,b j,,a j,3,b j,3} On the other hand, we have that B 1 = B 1 Σ nh+m+ν. Hence, we get a contradiction since ν 10(m + nh). The base case of the induction corresponds to setting j = 1 and it follows along the same lines as above except that we invoke Lemma 7 with j = 1. This concludes the proof of Lemma 1. We now prove Lemma. Proof of Lemma : To see this, assume for the sake of contradiction that there exists i [n] s.t. r i { 1, 1} and let i [n] be the smallest such i. Since the Σ-ar representations of each of B 1 and {a i,1, b i,1 : i [n]} have zeros in the rightmost ν digits, the first moment constraint = B 1 is equivalent S to l i=i +1 c i Σ i + r i Σ i = 0 for some l N and c i { 1, 0, 1, } for all i {i + 1,..., l}. Dividing l b Σ i, we get that c i Σ i i = r i. Since Σ is i=i +1 assumed to be an even integer and since r i { 1, 1}, the left-hand side is an even integer whereas the righthand side is an odd integer; a contradiction. The onl remaining part is to prove Lemma 7. Proof of Lemma 7: We first derive in the next proposition some inequalities that are satisfied b the integers {a i,1, a i,, a, b i,1, b i,, b : i [n]} and that will be used to prove Lemma 7. Proposition. Let j [n]. 1) a j,1 b j,1 Σ ν. ) If ν 10(m + nh), then i [n] : a j, a i,1 Σ Ω(ν) and a j, b i,1 3) If h 10m and j < n, then Σ Ω(ν) i {j + 1,..., n} : a j, a i, ΣΩ(h) and a j, b i, ΣΩ(h) The same inequalities also hold if we replace a j, b b j,. Proof of Proposition : The first part of the proposition follows from the assumption (which can be made without loss of generalit) that for each j [n], there exists a SAT clause that contains exactl one of x j and x j. We next prove the second part of the proposition. Fix j, i [n]. Without loss of generalit, assume that a j,1 > b j,1. Then, the first part of the proposition ields that a j,1 b j,1 Σ ν. Then, we have that a j, = a j,1 b j,1 Σj = (a j,1 b j,1 )(a j,1 + b j,1 ) Σν Σ ν Σj Σ ν 3n Σj On the other hand, we have that a i,1 Σ ν+m+nh and b i,1 Σ ν+m+nh. Using the assumption that ν 10(m + nh), we conclude that aj, a i,1 Σ Ω(ν) and a j, b i,1 Σ Ω(ν). We now prove the third part of the proposition. Fix j < n and i {j+1,..., n}. Without loss of generalit, assume that a j,1 > b j,1 and a i,1 > b i,1. Then, we have that a j, = (a j,1 b j,1 )(a j,1 + b j,1 ) Σν Σ (n j)h+m+ν Σ ν+(n j)h+m j On the other hand, we have that Therefore, a i, = (a i,1 b i,1 )(a i,1 + b i,1 ) 4Σ i Σj Σj Σi Σν+m Σ (n i)h+m+ν+1 4Σ i = Σ ν+m+(n i)h i+1 a j, a i, 1 Σ(i j)h m+(i j) 1 1 Σh m = Σ Ω(h) where the last equalit above follows from the assumption that h 10m. The proof that a j, b i, Σ Ω(h) follows along the same lines. Observe that for an j 1, if S {a j,, b j, } S {a j,3, b j,3 }, then S {a j,, b j,, a j,3, b j,3 } is one of the following possible sets: {a j, }, {b j, }, {a j,3 }, {b j,3 }, {a j,, b j,, a j,3 }, {a j,, b j,, b j,3 }, {a j,, a j,3, b j,3 }, {b j,, a j,3, b j,3 } 7

8 In each of these cases, the following inequalit is satisfied min( a j,, b j, ) Σ j (1) S {a j,,b j,,a j,3,b j,3} We now prove the first part of Lemma 7. Since S {a j,, b j, } = S {a j,3, b j,3 } and assuming that a j,1 > b j,1 without loss of generalit, Eq. (1) gives that (a j,1 b j,1)(a j,1 + b j,1) S {a j,,b j,,a j,3,b j,3} 3Σj Σν Σ ν+m+(n j)h 3Σj = Ω(Σ ν n ) We now prove the second part of Lemma 7, which we first show for the case where j and S {a i,, b i, } = S {a, b } for all i < j. These equalities impl that Σ O(n) and hence min( a j,, b j, ) Σ ν 3n Σ Ω(ν) S j 1 {ai,,bi,,a,b} S j 1 {ai,,bi,,a,b} () Using Equation (1) and Proposition, we then have that min( a j,, b j, ) Σ j S {a j,,b j,,a j,3,b j,3} Θ(n) 1 Θ(n) 1 ( Θ(n) j=1 min( a j,, b j, ) Σ j Σ Ω(ν) S n {ai,1,bi,1} + Σ Ω(h) S n i=j+1 {ai,,bi,,a,b} + Σ Ω(ν) S j 1 {ai,,bi,,a,b} ) Σ j Σ Ω(min(ν,h)) S\{a j,,b j,,a j,3,b j,3} where the last inequalit above follows from the triangle inequalit. The proof for the case where j = 1 follows along the same lines as above except that the quantit is replaced b 0 and Equation () is not S j 1 {ai,,bi,,a,b} needed. C. Proofs from Section IV Proof of Proposition 1: For the first identit, we have that a i, + a = α i = b i, + b. For the second identit, we have that a i,1 + a (b i,1 + b i, + b ) = a i,1 b i,1 + (a i, b i,)(a i, + b i,) + (a b )(a + b ) = a i,1 b i,1 β i (α i + γ i ) + β i (α i γ i ) = a i,1 b i,1 β i γ i = 0 For the third identit, we have that a 3 i,1 + a 3 i, + a 3 (b 3 i,1 + b 3 i, + b 3 ) i,1 + (a i, b i,)(a i, + a i,b i, + b i,) + (a b )(a + a b + b ) i,1 β i (a i, + a i,b i, + b i,) + β i (a + a b + b ) i,1 β i ((a i, a )(a i, + a ) + a i,b i, a b + (b i, b )(b i, + b ) i,1 β i ((γ i β i )α i + a i,b i, a b + (γ i + β i )α i ) i,1 4α i β i γ i β i (a i,b i, a b ) i,1 6α i β i γ i = 0 where the penultimate equalit uses the fact that a i,b i, a b = α i γ i. We now use Proposition 1 in order to check that the first 3 moments of S are equal to B 1, B and ) 8

9 B 3 respectivel, and thereb finish the completeness analsis of Theorem 5. = a i,1 + a i, + a S + = + = b i,1 + b i, + b a i,1 + a i, + a + a i,1 + + a i, + a = + + a i, + a = Σ ν+m+h 1 ( + Σ ν ( b i,1 b i,1 b i, + b Σ ν+m+h 1 (a v i ) Σ h + Σ ν (a c i) Σ Σ ν+m+h 1 (b v i ) Σ h + Σ ν (b c i) Σ a c i + + a i, + a a v i + b c i) Σ = Σ ν+m+h 1 (1 n ) Σ h + Σ ν (1 m ) Σ + a i, + a = B 1 Furthermore, = Finall, S 3 = S + = = B + a i,1 + a b i,1 + b i, + b a i,1 + a a 3 i,1 + a 3 i, + a 3 b 3 i,1 + b 3 i, + b 3 b v i ) Σ h = = B 3 a 3 i,1 + a 3 i, + a 3 We now turn to the proofs of Lemmas 3, 4 and 5. We will use the following proposition whose proof is similar to that of Proposition (because of the fact that a i,l = Θ( a i,l ) and b i,l = Θ( b i,l ) for ever i [n] and l [3]). Proposition 3. Let j [n]. 1) a j,1 b j,1 Σ ν. ) If ν 10(m + nh), then a j, i [n] : a Σ Ω(ν) and a j, i,1 b i,1 3) If h 10m and j < n, then i {j + 1,..., n} : a j, a i, ΣΩ(h) Σ Ω(ν) 4) If ν 10(m + nh), j, i < j and S {a i,, b i,, a, b } =, then a j,/σ Ω(ν) is at least a S {a i,,b i,,a,b } The same inequalities also hold if we replace a j, b one of {b j,, a j,3, b j,3} or if we replace a i, b one of {b i,, a, b } Proof of Lemma 3: Follows along the same lines as the proof of Lemma 1 but using Proposition 3 instead of Proposition. The proof of Lemma 4 uses the following lemma. Lemma 8. Let j 1 be an integer. Furthermore, assume that if j, then S {a i,, b i,, a, b } = for all i < j. Then, min {a j,,b j,,a j,3,b j,3 } is lower bounded b: ( n (i) Σ Ω(min(ν,h)) a i,1 + n i=j+1 j 1 (a a ) + S {a i,,b i,,a,b } (ii) Σ( Ω(min(ν,h)) + S n i=j+1 {a i,,b i,,a,b } S n {a i,1,b i,1} ) ) 9

10 Proof of Lemma 8: Similar to that of Lemma 7 but uses Proposition 3 instead of Proposition. Proof of Lemma 4: We proceed b induction on i [n]. At the jth step of the induction (with j ), we assume that S {a i,, b i,, a, b } = for all i < j and we need to show that S {a j,, b j,, a j,3, b j,3} =. Assume for the sake of contradiction that S {a j,, b j,, a j,3, b j,3}. We have that B S j {a i,,b i,,a,b } where q 1 := (a j, +a j,3) and j 1 ( q := n S {a i,,b i,,a,b } a i,1 n i=j+1 (a = q 1 q S {a j,,b j,,a j,3,b j,3} a i, a ) ) Then, Lemma 8 and the fact that for an a, b R, a b max( a, b ) min( a, b ) impl that B j, + a + (a ( j 1 S j {a i,,b i,,a,b } a n Ω( a i,1 + j,3) n i=j+1 min q 1 q ) S {a j,,b j,,a j,3,b j,3} (a S {a i,,b i,,a,b } {a j,,b j,,a j,3,b j,3 } ) ) 1 min Σ Ω(min(ν,h)) {a j,,b j,,a j,3,b j,3 } = Ω( min {a j,,b j,,a j,3,b j,3 } ) Lemma 8 impl that B = + S j {a i,,b i,,a,b } S n i=j+1 {a i,,b i,,a,b } S n {a i,1,b i,1} 1 min Σ Ω(min(ν,h)) {a j,,b j,,a j,3,b j,3 } which ields a contradiction. Proof of Lemma 5: Lemmas 3 and 4 impl that for ever i [n], = α i +r i Σ i S {a i,,b i,,a,b } for some r i { 1, 0, 1}. The next lemma argues that, in fact, all r i s are equal to 0. Lemma 9. For ever i [n], r i = 0. Proof of Lemma 9: To see this, assume for the sake of contradiction that there exists i [n] s.t. r i { 1, 1} and let i [n] be the smallest such i. Note that the first moment constraint = S B 1 is equivalent to S n {a i,1,b i,1} + n r i Σ i = Σ ν+m+h 1 (1 n ) Σ h + Σ ν (1 m ) Σ. Since the Σ- ar representations of each of the positive integers Σ ν+m+h 1 (1 n ) Σ h + Σ ν (1 m ) Σ and {a i,1, b i,1 : i [n]} have zeros in the rightmost ν digits, this constraint l is also equivalent to c i Σ i + r i Σ i = 0 for some i=i +1 l N and c i { 1, 0, 1, } for all i {i + 1,..., l}. l Dividing b Σ i, we get that c i Σ i i = r i. i=i +1 Since Σ is assumed to be an even integer and since r i { 1, 1}, the left-hand side is an even integer whereas the right-hand side is an odd integer; a contradiction. This completes the proof of Lemma 5. On the other hand, the fact that = B and S 10

On the NP-Hardness of Bounded Distance Decoding of Reed-Solomon Codes

On the NP-Hardness of Bounded Distance Decoding of Reed-Solomon Codes On the NP-Hardness of Bounded Distance Decoding of Reed-Solomon Codes Venkata Gandikota Purdue University vgandiko@purdue.edu Badih Ghazi MIT badih@mit.edu Elena Grigorescu Purdue University elena-g@purdue.edu

More information

Approximation of Continuous Functions

Approximation of Continuous Functions Approximation of Continuous Functions Francis J. Narcowich October 2014 1 Modulus of Continuit Recall that ever function continuous on a closed interval < a x b < is uniforml continuous: For ever ɛ > 0,

More information

Computing Error Distance of Reed-Solomon Codes

Computing Error Distance of Reed-Solomon Codes Computing Error Distance of Reed-Solomon Codes Guizhen Zhu Institute For Advanced Study Tsinghua University, Beijing, 100084, PR China Email:zhugz08@mailstsinghuaeducn Daqing Wan Department of Mathematics

More information

The Maze Generation Problem is NP-complete

The Maze Generation Problem is NP-complete The Mae Generation Problem is NP-complete Mario Alviano Department of Mathematics, Universit of Calabria, 87030 Rende (CS), Ital alviano@mat.unical.it Abstract. The Mae Generation problem has been presented

More information

Minimal reductions of monomial ideals

Minimal reductions of monomial ideals ISSN: 1401-5617 Minimal reductions of monomial ideals Veronica Crispin Quiñonez Research Reports in Mathematics Number 10, 2004 Department of Mathematics Stocholm Universit Electronic versions of this

More information

Provable intractability. NP-completeness. Decision problems. P problems. Algorithms. Two causes of intractability:

Provable intractability. NP-completeness. Decision problems. P problems. Algorithms. Two causes of intractability: Provable intractabilit -completeness Selected from Computer and Intractabilit b MR Gare and DS Johnson (979) Two causes of intractabilit: The problem is so difficult that an exponential amount of time

More information

Chapter 6 Reed-Solomon Codes. 6.1 Finite Field Algebra 6.2 Reed-Solomon Codes 6.3 Syndrome Based Decoding 6.4 Curve-Fitting Based Decoding

Chapter 6 Reed-Solomon Codes. 6.1 Finite Field Algebra 6.2 Reed-Solomon Codes 6.3 Syndrome Based Decoding 6.4 Curve-Fitting Based Decoding Chapter 6 Reed-Solomon Codes 6. Finite Field Algebra 6. Reed-Solomon Codes 6.3 Syndrome Based Decoding 6.4 Curve-Fitting Based Decoding 6. Finite Field Algebra Nonbinary codes: message and codeword symbols

More information

Notes 10: List Decoding Reed-Solomon Codes and Concatenated codes

Notes 10: List Decoding Reed-Solomon Codes and Concatenated codes Introduction to Coding Theory CMU: Spring 010 Notes 10: List Decoding Reed-Solomon Codes and Concatenated codes April 010 Lecturer: Venkatesan Guruswami Scribe: Venkat Guruswami & Ali Kemal Sinop DRAFT

More information

Lecture Introduction. 2 Linear codes. CS CTT Current Topics in Theoretical CS Oct 4, 2012

Lecture Introduction. 2 Linear codes. CS CTT Current Topics in Theoretical CS Oct 4, 2012 CS 59000 CTT Current Topics in Theoretical CS Oct 4, 01 Lecturer: Elena Grigorescu Lecture 14 Scribe: Selvakumaran Vadivelmurugan 1 Introduction We introduced error-correcting codes and linear codes in

More information

New algebraic decoding method for the (41, 21,9) quadratic residue code

New algebraic decoding method for the (41, 21,9) quadratic residue code New algebraic decoding method for the (41, 21,9) quadratic residue code Mohammed M. Al-Ashker a, Ramez Al.Shorbassi b a Department of Mathematics Islamic University of Gaza, Palestine b Ministry of education,

More information

Solutions to Assignment 1

Solutions to Assignment 1 Solutions to Assignment 1 Question 1. [Exercises 1.1, # 6] Use the division algorithm to prove that every odd integer is either of the form 4k + 1 or of the form 4k + 3 for some integer k. For each positive

More information

A Combinatorial Bound on the List Size

A Combinatorial Bound on the List Size 1 A Combinatorial Bound on the List Size Yuval Cassuto and Jehoshua Bruck California Institute of Technology Electrical Engineering Department MC 136-93 Pasadena, CA 9115, U.S.A. E-mail: {ycassuto,bruck}@paradise.caltech.edu

More information

Complexity of Decoding Positive-Rate Reed-Solomon Codes

Complexity of Decoding Positive-Rate Reed-Solomon Codes Complexity of Decoding Positive-Rate Reed-Solomon Codes Qi Ceng 1 and Daqing Wan 1 Scool of Computer Science Te University of Oklaoma Norman, OK73019 Email: qceng@cs.ou.edu Department of Matematics University

More information

Lecture 19 : Reed-Muller, Concatenation Codes & Decoding problem

Lecture 19 : Reed-Muller, Concatenation Codes & Decoding problem IITM-CS6845: Theory Toolkit February 08, 2012 Lecture 19 : Reed-Muller, Concatenation Codes & Decoding problem Lecturer: Jayalal Sarma Scribe: Dinesh K Theme: Error correcting codes In the previous lecture,

More information

EQUIVALENT FORMULATIONS OF HYPERCONTRACTIVITY USING INFORMATION MEASURES

EQUIVALENT FORMULATIONS OF HYPERCONTRACTIVITY USING INFORMATION MEASURES 1 EQUIVALENT FORMULATIONS OF HYPERCONTRACTIVITY USING INFORMATION MEASURES CHANDRA NAIR 1 1 Dept. of Information Engineering, The Chinese Universit of Hong Kong Abstract We derive alternate characterizations

More information

4. Product measure spaces and the Lebesgue integral in R n.

4. Product measure spaces and the Lebesgue integral in R n. 4 M. M. PELOSO 4. Product measure spaces and the Lebesgue integral in R n. Our current goal is to define the Lebesgue measure on the higher-dimensional eucledean space R n, and to reduce the computations

More information

Section 3.1. ; X = (0, 1]. (i) f : R R R, f (x, y) = x y

Section 3.1. ; X = (0, 1]. (i) f : R R R, f (x, y) = x y Paul J. Bruillard MATH 0.970 Problem Set 6 An Introduction to Abstract Mathematics R. Bond and W. Keane Section 3.1: 3b,c,e,i, 4bd, 6, 9, 15, 16, 18c,e, 19a, 0, 1b Section 3.: 1f,i, e, 6, 1e,f,h, 13e,

More information

INTRODUCTION TO DIOPHANTINE EQUATIONS

INTRODUCTION TO DIOPHANTINE EQUATIONS INTRODUCTION TO DIOPHANTINE EQUATIONS In the earl 20th centur, Thue made an important breakthrough in the stud of diophantine equations. His proof is one of the first eamples of the polnomial method. His

More information

arxiv: v2 [cs.ds] 17 Sep 2017

arxiv: v2 [cs.ds] 17 Sep 2017 Two-Dimensional Indirect Binary Search for the Positive One-In-Three Satisfiability Problem arxiv:1708.08377v [cs.ds] 17 Sep 017 Shunichi Matsubara Aoyama Gakuin University, 5-10-1, Fuchinobe, Chuo-ku,

More information

A. Derivation of regularized ERM duality

A. Derivation of regularized ERM duality A. Derivation of regularized ERM dualit For completeness, in this section we derive the dual 5 to the problem of computing proximal operator for the ERM objective 3. We can rewrite the primal problem as

More information

Lecture 12: November 6, 2017

Lecture 12: November 6, 2017 Information and Coding Theory Autumn 017 Lecturer: Madhur Tulsiani Lecture 1: November 6, 017 Recall: We were looking at codes of the form C : F k p F n p, where p is prime, k is the message length, and

More information

Lecture 19: Elias-Bassalygo Bound

Lecture 19: Elias-Bassalygo Bound Error Correcting Codes: Combinatorics, Algorithms and Applications (Fall 2007) Lecturer: Atri Rudra Lecture 19: Elias-Bassalygo Bound October 10, 2007 Scribe: Michael Pfetsch & Atri Rudra In the last lecture,

More information

4 Inverse function theorem

4 Inverse function theorem Tel Aviv Universit, 2013/14 Analsis-III,IV 53 4 Inverse function theorem 4a What is the problem................ 53 4b Simple observations before the theorem..... 54 4c The theorem.....................

More information

2.5 CONTINUITY. a x. Notice that Definition l implicitly requires three things if f is continuous at a:

2.5 CONTINUITY. a x. Notice that Definition l implicitly requires three things if f is continuous at a: SECTION.5 CONTINUITY 9.5 CONTINUITY We noticed in Section.3 that the it of a function as approaches a can often be found simpl b calculating the value of the function at a. Functions with this propert

More information

Introduction to Arithmetic Geometry Fall 2013 Lecture #5 09/19/2013

Introduction to Arithmetic Geometry Fall 2013 Lecture #5 09/19/2013 18.782 Introduction to Arithmetic Geometry Fall 2013 Lecture #5 09/19/2013 5.1 The field of p-adic numbers Definition 5.1. The field of p-adic numbers Q p is the fraction field of Z p. As a fraction field,

More information

Reed-Solomon Error-correcting Codes

Reed-Solomon Error-correcting Codes The Deep Hole Problem Matt Keti (Advisor: Professor Daqing Wan) Department of Mathematics University of California, Irvine November 8, 2012 Humble Beginnings Preview of Topics 1 Humble Beginnings Problems

More information

On a Balanced Property of Compositions

On a Balanced Property of Compositions On a Balanced Property of Compositions Miklós Bóna Department of Mathematics University of Florida Gainesville FL 32611-8105 USA Submitted: October 2, 2006; Accepted: January 24, 2007; Published: March

More information

Affine Hybrid Systems

Affine Hybrid Systems Affine Hbrid Sstems Aaron D Ames and Shankar Sastr Universit of California, Berkele CA 9472, USA {adames,sastr}@eecsberkeleedu Abstract Affine hbrid sstems are hbrid sstems in which the discrete domains

More information

Toda s Theorem: PH P #P

Toda s Theorem: PH P #P CS254: Computational Compleit Theor Prof. Luca Trevisan Final Project Ananth Raghunathan 1 Introduction Toda s Theorem: PH P #P The class NP captures the difficult of finding certificates. However, in

More information

You don't have to be a mathematician to have a feel for numbers. John Forbes Nash, Jr.

You don't have to be a mathematician to have a feel for numbers. John Forbes Nash, Jr. Course Title: Real Analsis Course Code: MTH3 Course instructor: Dr. Atiq ur Rehman Class: MSc-II Course URL: www.mathcit.org/atiq/fa5-mth3 You don't have to be a mathematician to have a feel for numbers.

More information

8. Limit Laws. lim(f g)(x) = lim f(x) lim g(x), (x) = lim x a f(x) g lim x a g(x)

8. Limit Laws. lim(f g)(x) = lim f(x) lim g(x), (x) = lim x a f(x) g lim x a g(x) 8. Limit Laws 8.1. Basic Limit Laws. If f and g are two functions and we know the it of each of them at a given point a, then we can easily compute the it at a of their sum, difference, product, constant

More information

Two NP-hard Interchangeable Terminal Problems*

Two NP-hard Interchangeable Terminal Problems* o NP-hard Interchangeable erminal Problems* Sartaj Sahni and San-Yuan Wu Universit of Minnesota ABSRAC o subproblems that arise hen routing channels ith interchangeable terminals are shon to be NP-hard

More information

Chapter 6 Lagrange Codes

Chapter 6 Lagrange Codes Chapter 6 Lagrange Codes 6. Introduction Joseph Louis Lagrange was a famous eighteenth century Italian mathematician [] credited with minimum degree polynomial interpolation amongst his many other achievements.

More information

Arrangements, matroids and codes

Arrangements, matroids and codes Arrangements, matroids and codes first lecture Ruud Pellikaan joint work with Relinde Jurrius ACAGM summer school Leuven Belgium, 18 July 2011 References 2/43 1. Codes, arrangements and matroids by Relinde

More information

Glossary. Also available at BigIdeasMath.com: multi-language glossary vocabulary flash cards. An equation that contains an absolute value expression

Glossary. Also available at BigIdeasMath.com: multi-language glossary vocabulary flash cards. An equation that contains an absolute value expression Glossar This student friendl glossar is designed to be a reference for ke vocabular, properties, and mathematical terms. Several of the entries include a short eample to aid our understanding of important

More information

New Algebraic Decoding of (17,9,5) Quadratic Residue Code by using Inverse Free Berlekamp-Massey Algorithm (IFBM)

New Algebraic Decoding of (17,9,5) Quadratic Residue Code by using Inverse Free Berlekamp-Massey Algorithm (IFBM) International Journal of Computational Intelligence Research (IJCIR). ISSN: 097-87 Volume, Number 8 (207), pp. 205 2027 Research India Publications http://www.ripublication.com/ijcir.htm New Algebraic

More information

Notes for the Hong Kong Lectures on Algorithmic Coding Theory. Luca Trevisan. January 7, 2007

Notes for the Hong Kong Lectures on Algorithmic Coding Theory. Luca Trevisan. January 7, 2007 Notes for the Hong Kong Lectures on Algorithmic Coding Theory Luca Trevisan January 7, 2007 These notes are excerpted from the paper Some Applications of Coding Theory in Computational Complexity [Tre04].

More information

Hardness of the Covering Radius Problem on Lattices

Hardness of the Covering Radius Problem on Lattices Hardness of the Covering Radius Problem on Lattices Ishay Haviv Oded Regev June 6, 2006 Abstract We provide the first hardness result for the Covering Radius Problem on lattices (CRP). Namely, we show

More information

On Range and Reflecting Functions About the Line y = mx

On Range and Reflecting Functions About the Line y = mx On Range and Reflecting Functions About the Line = m Scott J. Beslin Brian K. Heck Jerem J. Becnel Dept.of Mathematics and Dept. of Mathematics and Dept. of Mathematics and Computer Science Computer Science

More information

A Questionable Distance-Regular Graph

A Questionable Distance-Regular Graph A Questionable Distance-Regular Graph Rebecca Ross Abstract In this paper, we introduce distance-regular graphs and develop the intersection algebra for these graphs which is based upon its intersection

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

Linear Algebra March 16, 2019

Linear Algebra March 16, 2019 Linear Algebra March 16, 2019 2 Contents 0.1 Notation................................ 4 1 Systems of linear equations, and matrices 5 1.1 Systems of linear equations..................... 5 1.2 Augmented

More information

Ordinal One-Switch Utility Functions

Ordinal One-Switch Utility Functions Ordinal One-Switch Utilit Functions Ali E. Abbas Universit of Southern California, Los Angeles, California 90089, aliabbas@usc.edu David E. Bell Harvard Business School, Boston, Massachusetts 0163, dbell@hbs.edu

More information

Solutions of Exam Coding Theory (2MMC30), 23 June (1.a) Consider the 4 4 matrices as words in F 16

Solutions of Exam Coding Theory (2MMC30), 23 June (1.a) Consider the 4 4 matrices as words in F 16 Solutions of Exam Coding Theory (2MMC30), 23 June 2016 (1.a) Consider the 4 4 matrices as words in F 16 2, the binary vector space of dimension 16. C is the code of all binary 4 4 matrices such that the

More information

CHAPTER 10 Shape Preserving Properties of B-splines

CHAPTER 10 Shape Preserving Properties of B-splines CHAPTER 10 Shape Preserving Properties of B-splines In earlier chapters we have seen a number of examples of the close relationship between a spline function and its B-spline coefficients This is especially

More information

x c x c This suggests the following definition.

x c x c This suggests the following definition. 110 Chapter 1 / Limits and Continuit 1.5 CONTINUITY A thrown baseball cannot vanish at some point and reappear someplace else to continue its motion. Thus, we perceive the path of the ball as an unbroken

More information

A.5. Complex Numbers AP-12. The Development of the Real Numbers

A.5. Complex Numbers AP-12. The Development of the Real Numbers AP- A.5 Comple Numbers Comple numbers are epressions of the form a + ib, where a and b are real numbers and i is a smbol for -. Unfortunatel, the words real and imaginar have connotations that somehow

More information

Lecture Introduction. 2 Formal Definition. CS CTT Current Topics in Theoretical CS Oct 30, 2012

Lecture Introduction. 2 Formal Definition. CS CTT Current Topics in Theoretical CS Oct 30, 2012 CS 59000 CTT Current Topics in Theoretical CS Oct 30, 0 Lecturer: Elena Grigorescu Lecture 9 Scribe: Vivek Patel Introduction In this lecture we study locally decodable codes. Locally decodable codes are

More information

Chapter 6* The PPSZ Algorithm

Chapter 6* The PPSZ Algorithm Chapter 6* The PPSZ Algorithm In this chapter we present an improvement of the pp algorithm. As pp is called after its inventors, Paturi, Pudlak, and Zane [PPZ99], the improved version, pps, is called

More information

Standard forms for writing numbers

Standard forms for writing numbers Standard forms for writing numbers In order to relate the abstract mathematical descriptions of familiar number systems to the everyday descriptions of numbers by decimal expansions and similar means,

More information

MA123, Chapter 1: Equations, functions and graphs (pp. 1-15)

MA123, Chapter 1: Equations, functions and graphs (pp. 1-15) MA123, Chapter 1: Equations, functions and graphs (pp. 1-15) Date: Chapter Goals: Identif solutions to an equation. Solve an equation for one variable in terms of another. What is a function? Understand

More information

Orthogonal Arrays & Codes

Orthogonal Arrays & Codes Orthogonal Arrays & Codes Orthogonal Arrays - Redux An orthogonal array of strength t, a t-(v,k,λ)-oa, is a λv t x k array of v symbols, such that in any t columns of the array every one of the possible

More information

PARTIAL SEMIGROUPS AND PRIMALITY INDICATORS IN THE FRACTAL GENERATION OF BINOMIAL COEFFICIENTS TO A PRIME SQUARE MODULUS

PARTIAL SEMIGROUPS AND PRIMALITY INDICATORS IN THE FRACTAL GENERATION OF BINOMIAL COEFFICIENTS TO A PRIME SQUARE MODULUS PARTIAL SEMIGROUPS AND PRIMALITY INDICATORS IN THE FRACTAL GENERATION OF BINOMIAL COEFFICIENTS TO A PRIME SQUARE MODULUS D. DOAN, B. KIVUNGE 2, J.J. POOLE 3, J.D.H SMITH 4, T. SYKES, AND M. TEPLITSKIY

More information

An Interpolation Algorithm for List Decoding of Reed-Solomon Codes

An Interpolation Algorithm for List Decoding of Reed-Solomon Codes An Interpolation Algorithm for List Decoding of Reed-Solomon Codes Kwankyu Lee Department of Mathematics San Diego State University San Diego, USA Email: kwankyu@sogangackr Michael E O Sullivan Department

More information

Permanent is hard to compute even on a good day

Permanent is hard to compute even on a good day Permanent is hard to compute even on a good day Yuval Filmus September 11, 2012 Abstract We give an exposition of Cai, Pavan and Sivakumar s result on the hardness of permanent. They show that assuming

More information

Subfield value sets over finite fields

Subfield value sets over finite fields Subfield value sets over finite fields Wun-Seng Chou Institute of Mathematics Academia Sinica, and/or Department of Mathematical Sciences National Chengchi Universit Taipei, Taiwan, ROC Email: macws@mathsinicaedutw

More information

On the List and Bounded Distance Decodability of Reed-Solomon Codes

On the List and Bounded Distance Decodability of Reed-Solomon Codes On the List and Bounded Distance Decodability of Reed-Solomon Codes Qi Cheng School of Computer Science The University of Oklahoma Norman, OK 73019, USA qcheng@cs.ou.edu Daqing Wan University of California

More information

Solutions to Practice Final

Solutions to Practice Final s to Practice Final 1. (a) What is φ(0 100 ) where φ is Euler s φ-function? (b) Find an integer x such that 140x 1 (mod 01). Hint: gcd(140, 01) = 7. (a) φ(0 100 ) = φ(4 100 5 100 ) = φ( 00 5 100 ) = (

More information

10.2 The Unit Circle: Cosine and Sine

10.2 The Unit Circle: Cosine and Sine 0. The Unit Circle: Cosine and Sine 77 0. The Unit Circle: Cosine and Sine In Section 0.., we introduced circular motion and derived a formula which describes the linear velocit of an object moving on

More information

RMT 2013 Power Round Solutions February 2, 2013

RMT 2013 Power Round Solutions February 2, 2013 RMT 013 Power Round Solutions February, 013 1. (a) (i) {0, 5, 7, 10, 11, 1, 14} {n N 0 : n 15}. (ii) Yes, 5, 7, 11, 16 can be generated by a set of fewer than 4 elements. Specifically, it is generated

More information

The Tensor Product of Two Codes is Not Necessarily Robustly Testable

The Tensor Product of Two Codes is Not Necessarily Robustly Testable The Tensor Product of Two Codes is Not Necessarily Robustly Testable Paul Valiant Massachusetts Institute of Technology pvaliant@mit.edu Abstract. There has been significant interest lately in the task

More information

8.1 Exponents and Roots

8.1 Exponents and Roots Section 8. Eponents and Roots 75 8. Eponents and Roots Before defining the net famil of functions, the eponential functions, we will need to discuss eponent notation in detail. As we shall see, eponents

More information

Notes on Convexity. Roy Radner Stern School, NYU. September 11, 2006

Notes on Convexity. Roy Radner Stern School, NYU. September 11, 2006 Notes on Convexit Ro Radner Stern School, NYU September, 2006 Abstract These notes are intended to complement the material in an intermediate microeconomic theor course. In particular, the provide a rigorous

More information

Generalized Reed-Solomon Codes

Generalized Reed-Solomon Codes Chapter 5 Generalized Reed-Solomon Codes In 1960, I.S. Reed and G. Solomon introduced a family of error-correcting codes that are douly lessed. The codes and their generalizations are useful in practice,

More information

CLASSIFICATION OF TORIC MANIFOLDS OVER AN n-cube WITH ONE VERTEX CUT

CLASSIFICATION OF TORIC MANIFOLDS OVER AN n-cube WITH ONE VERTEX CUT CLASSIFICATION OF TORIC MANIFOLDS OVER AN n-cube WITH ONE VERTEX CUT SHO HASUI, HIDEYA KUWATA, MIKIYA MASUDA, AND SEONJEONG PARK Abstract We say that a complete nonsingular toric variety (called a toric

More information

1.3 LIMITS AT INFINITY; END BEHAVIOR OF A FUNCTION

1.3 LIMITS AT INFINITY; END BEHAVIOR OF A FUNCTION . Limits at Infinit; End Behavior of a Function 89. LIMITS AT INFINITY; END BEHAVIOR OF A FUNCTION Up to now we have been concerned with its that describe the behavior of a function f) as approaches some

More information

COUNTING NUMERICAL SEMIGROUPS BY GENUS AND SOME CASES OF A QUESTION OF WILF

COUNTING NUMERICAL SEMIGROUPS BY GENUS AND SOME CASES OF A QUESTION OF WILF COUNTING NUMERICAL SEMIGROUPS BY GENUS AND SOME CASES OF A QUESTION OF WILF NATHAN KAPLAN Abstract. The genus of a numerical semigroup is the size of its complement. In this paper we will prove some results

More information

math0320 FALL interactmath sections developmental mathematics sullivan 1e

math0320 FALL interactmath sections developmental mathematics sullivan 1e Eam final eam review 180 plus 234 TSI questions for intermediate algebra m032000 013014 NEW Name www.alvarezmathhelp.com math0320 FALL 201 1400 interactmath sections developmental mathematics sullivan

More information

locally maximal solutions for random CSPs 109 Why almost all satisfiable k-cnf formulas are easy

locally maximal solutions for random CSPs 109 Why almost all satisfiable k-cnf formulas are easy locall maximal solutions for random CSPs 109 Wh almost all satisfiable k-cnf formulas are eas 2007 Conference on Analsis of Algorithms, AofA 07 DMTCS proc. AH, 2007, 109 120 Expected number of locall maximal

More information

Complexity of Decoding Positive-Rate Primitive Reed-Solomon Codes

Complexity of Decoding Positive-Rate Primitive Reed-Solomon Codes 1 Complexity of Decoding Positive-Rate Primitive Reed-Solomon Codes Qi Ceng and Daqing Wan Abstract It as been proved tat te maximum likeliood decoding problem of Reed-Solomon codes is NP-ard. However,

More information

Chapter 8. P-adic numbers. 8.1 Absolute values

Chapter 8. P-adic numbers. 8.1 Absolute values Chapter 8 P-adic numbers Literature: N. Koblitz, p-adic Numbers, p-adic Analysis, and Zeta-Functions, 2nd edition, Graduate Texts in Mathematics 58, Springer Verlag 1984, corrected 2nd printing 1996, Chap.

More information

SMT 2013 Power Round Solutions February 2, 2013

SMT 2013 Power Round Solutions February 2, 2013 Introduction This Power Round is an exploration of numerical semigroups, mathematical structures which appear very naturally out of answers to simple questions. For example, suppose McDonald s sells Chicken

More information

Marcinkiewicz Interpolation Theorem by Daniel Baczkowski

Marcinkiewicz Interpolation Theorem by Daniel Baczkowski 1 Introduction Marcinkiewicz Interpolation Theorem b Daniel Baczkowski Let (, µ be a measure space. Let M denote the collection of all extended real valued µ-measurable functions on. Also, let M denote

More information

Lecture 28: Generalized Minimum Distance Decoding

Lecture 28: Generalized Minimum Distance Decoding Error Correcting Codes: Combinatorics, Algorithms and Applications (Fall 007) Lecture 8: Generalized Minimum Distance Decoding November 5, 007 Lecturer: Atri Rudra Scribe: Sandipan Kundu & Atri Rudra 1

More information

Representation of Functions by Power Series. Geometric Power Series

Representation of Functions by Power Series. Geometric Power Series 60_0909.qd //0 :09 PM Page 669 SECTION 9.9 Representation of Functions b Power Series 669 The Granger Collection Section 9.9 JOSEPH FOURIER (768 80) Some of the earl work in representing functions b power

More information

Modular Counting of Rational Points over Finite Fields

Modular Counting of Rational Points over Finite Fields Modular Counting of Rational Points over Finite Fields Daqing Wan Department of Mathematics University of California Irvine, CA 92697-3875 dwan@math.uci.edu Abstract Let F q be the finite field of q elements,

More information

Error-Correcting Codes

Error-Correcting Codes Error-Correcting Codes HMC Algebraic Geometry Final Project Dmitri Skjorshammer December 14, 2010 1 Introduction Transmission of information takes place over noisy signals. This is the case in satellite

More information

Quantitative stability of the Brunn-Minkowski inequality for sets of equal volume

Quantitative stability of the Brunn-Minkowski inequality for sets of equal volume Quantitative stabilit of the Brunn-Minkowski inequalit for sets of equal volume Alessio Figalli and David Jerison Abstract We prove a quantitative stabilit result for the Brunn-Minkowski inequalit on sets

More information

K. Johnson Department of Mathematics, Dalhousie University, Halifax, Nova Scotia, Canada D. Patterson

K. Johnson Department of Mathematics, Dalhousie University, Halifax, Nova Scotia, Canada D. Patterson #A21 INTEGERS 11 (2011) PROJECTIVE P -ORDERINGS AND HOMOGENEOUS INTEGER-VALUED POLYNOMIALS K. Johnson Department of Mathematics, Dalhousie University, Halifax, Nova Scotia, Canada johnson@mathstat.dal.ca

More information

Analytic Number Theory Solutions

Analytic Number Theory Solutions Analytic Number Theory Solutions Sean Li Cornell University sxl6@cornell.edu Jan. 03 Introduction This document is a work-in-progress solution manual for Tom Apostol s Introduction to Analytic Number Theory.

More information

Introduction to Association Schemes

Introduction to Association Schemes Introduction to Association Schemes Akihiro Munemasa Tohoku University June 5 6, 24 Algebraic Combinatorics Summer School, Sendai Assumed results (i) Vandermonde determinant: a a m =. a m a m m i

More information

CHAPTER 8: EXPLORING R

CHAPTER 8: EXPLORING R CHAPTER 8: EXPLORING R LECTURE NOTES FOR MATH 378 (CSUSM, SPRING 2009). WAYNE AITKEN In the previous chapter we discussed the need for a complete ordered field. The field Q is not complete, so we constructed

More information

Soft-decision Decoding of Chinese Remainder Codes

Soft-decision Decoding of Chinese Remainder Codes Soft-decision Decoding of Chinese Remainder Codes Venkatesan Guruswami Amit Sahai Ý Madhu Sudan Þ Abstract Given Ò relatively prime integers Ô Ô Ò and an integer Ò, the Chinese Remainder Code, ÊÌ É ÔÔÒ,

More information

Week 3 September 5-7.

Week 3 September 5-7. MA322 Weekl topics and quiz preparations Week 3 September 5-7. Topics These are alread partl covered in lectures. We collect the details for convenience.. Solutions of homogeneous equations AX =. 2. Using

More information

Error Correcting Codes: Combinatorics, Algorithms and Applications Spring Homework Due Monday March 23, 2009 in class

Error Correcting Codes: Combinatorics, Algorithms and Applications Spring Homework Due Monday March 23, 2009 in class Error Correcting Codes: Combinatorics, Algorithms and Applications Spring 2009 Homework Due Monday March 23, 2009 in class You can collaborate in groups of up to 3. However, the write-ups must be done

More information

Linear programming: Theory

Linear programming: Theory Division of the Humanities and Social Sciences Ec 181 KC Border Convex Analsis and Economic Theor Winter 2018 Topic 28: Linear programming: Theor 28.1 The saddlepoint theorem for linear programming The

More information

PICONE S IDENTITY FOR A SYSTEM OF FIRST-ORDER NONLINEAR PARTIAL DIFFERENTIAL EQUATIONS

PICONE S IDENTITY FOR A SYSTEM OF FIRST-ORDER NONLINEAR PARTIAL DIFFERENTIAL EQUATIONS Electronic Journal of Differential Equations, Vol. 2013 (2013), No. 143, pp. 1 7. ISSN: 1072-6691. URL: http://ejde.math.txstate.edu or http://ejde.math.unt.edu ftp ejde.math.txstate.edu PICONE S IDENTITY

More information

Lecture 7. The Cluster Expansion Lemma

Lecture 7. The Cluster Expansion Lemma Stanford Universit Spring 206 Math 233: Non-constructive methods in combinatorics Instructor: Jan Vondrák Lecture date: Apr 3, 206 Scribe: Erik Bates Lecture 7. The Cluster Expansion Lemma We have seen

More information

Lecture 12: Reed-Solomon Codes

Lecture 12: Reed-Solomon Codes Error Correcting Codes: Combinatorics, Algorithms and Applications (Fall 007) Lecture 1: Reed-Solomon Codes September 8, 007 Lecturer: Atri Rudra Scribe: Michel Kulhandjian Last lecture we saw the proof

More information

Lecture 03: Polynomial Based Codes

Lecture 03: Polynomial Based Codes Lecture 03: Polynomial Based Codes Error-Correcting Codes (Spring 016) Rutgers University Swastik Kopparty Scribes: Ross Berkowitz & Amey Bhangale 1 Reed-Solomon Codes Reed Solomon codes are large alphabet

More information

On representable graphs

On representable graphs On representable graphs Sergey Kitaev and Artem Pyatkin 3rd November 2005 Abstract A graph G = (V, E) is representable if there exists a word W over the alphabet V such that letters x and y alternate in

More information

Locally Dense Codes. Daniele Micciancio. August 26, 2013

Locally Dense Codes. Daniele Micciancio. August 26, 2013 Electronic Colloquium on Computational Complexity, Report No. 115 (2013) Locally Dense Codes Daniele Micciancio August 26, 2013 Abstract The Minimum Distance Problem (MDP), i.e., the computational task

More information

Proof: Let the check matrix be

Proof: Let the check matrix be Review/Outline Recall: Looking for good codes High info rate vs. high min distance Want simple description, too Linear, even cyclic, plausible Gilbert-Varshamov bound for linear codes Check matrix criterion

More information

On Irreducible Polynomial Remainder Codes

On Irreducible Polynomial Remainder Codes 2011 IEEE International Symposium on Information Theory Proceedings On Irreducible Polynomial Remainder Codes Jiun-Hung Yu and Hans-Andrea Loeliger Department of Information Technology and Electrical Engineering

More information

Math 120 HW 9 Solutions

Math 120 HW 9 Solutions Math 120 HW 9 Solutions June 8, 2018 Question 1 Write down a ring homomorphism (no proof required) f from R = Z[ 11] = {a + b 11 a, b Z} to S = Z/35Z. The main difficulty is to find an element x Z/35Z

More information

5.0 BCH and Reed-Solomon Codes 5.1 Introduction

5.0 BCH and Reed-Solomon Codes 5.1 Introduction 5.0 BCH and Reed-Solomon Codes 5.1 Introduction A. Hocquenghem (1959), Codes correcteur d erreurs; Bose and Ray-Chaudhuri (1960), Error Correcting Binary Group Codes; First general family of algebraic

More information

MY PUTNAM PROBLEMS. log(1 + x) dx = π2

MY PUTNAM PROBLEMS. log(1 + x) dx = π2 MY PUTNAM PROBLEMS These are the problems I proposed when I was on the Putnam Problem Committee for the 984 86 Putnam Exams. Problems intended to be A or B (and therefore relatively easy) are marked accordingly.

More information

Design and Analysis of Algorithms

Design and Analysis of Algorithms CSE 101, Winter 2018 Design and Analsis of Algorithms Lecture 15: NP-Completeness Class URL: http://vlsicad.ucsd.edu/courses/cse101-w18/ From Application to Algorithm Design Find all maimal regularl-spaced,

More information

Algebra Review 2. 1 Fields. A field is an extension of the concept of a group.

Algebra Review 2. 1 Fields. A field is an extension of the concept of a group. Algebra Review 2 1 Fields A field is an extension of the concept of a group. Definition 1. A field (F, +,, 0 F, 1 F ) is a set F together with two binary operations (+, ) on F such that the following conditions

More information

: Error Correcting Codes. October 2017 Lecture 1

: Error Correcting Codes. October 2017 Lecture 1 03683072: Error Correcting Codes. October 2017 Lecture 1 First Definitions and Basic Codes Amnon Ta-Shma and Dean Doron 1 Error Correcting Codes Basics Definition 1. An (n, K, d) q code is a subset of

More information