This paper was converted on www.awesomepapers.org from LaTeX by an anonymous user.
Want to know more? Visit the Converter page.

Incomplete sets in 𝐏{\mathbf{P}} for logspace reduction

Reiner Czerwinski
TU Berlin (Alumnus)
reiner.czerwinski@posteo.de
Abstract

In this article, we investigate the behaviour of TMs with time limit and tape space limit. This problem is in 𝐏{\mathbf{P}} when the time limit is unary coded. When both limits go to infinity, it is undecidable which limit is exceeded first. Thus logspace incomplete sets can be constructed in 𝐏{\mathbf{P}}. This implies 𝐋≠𝐏{\mathbf{L}}{}\not={\mathbf{P}}.

1 Introduction

It is known that the set

A={(M,x,1t)∣ TM ​M​ accepts ​x​ within ​t​ steps}A=\{(M,x,1^{t})\mid\text{ TM }M\text{ accepts }x\text{ within }t\text{ steps}\}

is logspace-complete for 𝐏{\mathbf{P}} [HS11, page 176, Th. 7.24].
This means βˆ€X:X≀logmA\forall X:X\leq^{m}_{\log}A.

In this paper, we look for logspace-incomplete sets in 𝐏{\mathbf{P}}. We observe the following sets:

U(f):={(M,x,1t,1s)∣\displaystyle U(f)=\{(M,x,1^{t},1^{s})\mid TM ​M​ accepts ​x​ within ​t​ steps and\displaystyle\text{ TM }M\text{ accepts }x\text{ within }t\text{ steps and}
withinΒ f(s)Β tape space}\displaystyle\text{ within }f(s)\text{ tape space}\}

For this reason, we use the sets:

B​(f):={(M,x,1s)∣ TM ​M​ accepts ​x​ within ​f​(s)​ tape space}B(f):=\{(M,x,1^{s})\mid\text{ TM }M\text{ accepts }x\text{ within }f(s)\text{ tape space}\}

The sets U​(f)U(f) are in 𝐏{\mathbf{P}}, but the sets B​(f)B(f) are easier to analyse. All these sets are connected:

Lemma 1.

U​(f)≀TlogB​(f)U(f)\leq_{T}^{\log}B(f) and U​(f)≀mlogAU(f)\leq_{m}^{\log}A

Proof.

immediately ∎

If ff is a time- and space-constructible function then

πƒπ“πˆπŒπ„β€‹(f)βŠ†πƒπ’ππ€π‚π„β€‹(f)βŠ†πƒπ“πˆπŒπ„β€‹(fβˆ—2O​(f))​[HPV75]{\mathbf{DTIME}}(f)\subseteq{\mathbf{DSPACE}}(f)\subseteq{\mathbf{DTIME}}(f*2^{O(f)})\;\cite[cite]{[\@@bibref{}{hopcroft1975time}{}{}]}

Let f:ℕ→ℝ+f:\mathbb{N}\to\mathbb{R}_{+} a sublinear function with fβˆˆΞ©β€‹(log)f\in\Omega(\log). In section 2 we will show that it is undecidable for a TM MM if sM∈O​(f​(tM))s_{M}\in O(f(t_{M})) when sMs_{M} is the used tape space of MM and tMt_{M} is the computation time. See also [Cze21].

In section 3 we will use these results to show that the sets U​(f)U(f), where ff is sub-linear and fβˆˆΞ©β€‹(log)f\in\Omega(\log), are incomplete in 𝐏{\mathbf{P}}.

Baker, Gill, and Solovay have proved the relativization barrier for P versus NP[BGS75]. Like the P versus NP problem, the L versus P problem cannot be solved with diagonalization alone. Nor can it be solved by computability methods alone. One also needs methods from complexity theory. In this paper, we combine these concepts. In section 4, we explain why we can circumvent the relativization barrier.

2 Tape Space of polynomial time TMs and the Arithmetical Hierarchy

Let K0:={M∣ TM ​M​ terminates on empty inputΒ }K_{0}:=\{M\mid\text{ TM }M\text{ terminates on empty input }\} and
K0Β―:={M∣ TM ​Mβˆ‰K0}\overline{K_{0}}:=\{M\mid\text{ TM }M\not\in K_{0}\}. Both sets are not computable, due to the halting problem[Tur36]. It is known, that K0K_{0} is Ξ£1\Sigma_{1}-complete and K0Β―\overline{K_{0}} is Ξ 1\Pi_{1}-complete[Soa87].

For a TM MM we define:

S~M​(t)\displaystyle\tilde{S}_{M}(t) :=tape space used byΒ MΒ to compute on empty input within ​t​ steps\displaystyle:=\text{tape space used by $M$ to compute on empty input within }t\text{ steps}

and

P~​(f):={Mβˆ£βˆ€t​S~M​(t)<f​(t)}\tilde{P}(f):=\{M\mid\forall t\;\tilde{S}_{M}(t)<f(t)\}
Lemma 2.

K0≀1P~​(f)K_{0}\leq_{1}\tilde{P}(f) if f∈o​(t)f\in o(t) and fβˆˆΞ©β€‹(log⁑(t))f\in\Omega(\log(t))

Proof.

There is a one-one reduction that transforms MM to a multi-taped TM h​(M)h(M) with one tape more than MM. h​(M)h(M) does not terminate and Sh​(M)S_{h(M)} grows linearly if MM does not terminate, otherwise it is logarithmic.

Algorithm 1 h​(M):h(M):
0: multi-taped TM MM with empty input
0: algorithm runs on a TM that has one more tape than MM
 whileΒ MM is not terminatedΒ do
  calculate one step on MM
  write ’11’ on the last tape
   move the head of last the tape one position to the left
 endΒ while
 ifΒ MM has terminatedΒ then
  apply binary counter to the last tape
 endΒ if

If MM does not terminate, the tape space of h​(M)h(M) grows linearly with time, so that

M∈K0⇔h​(M)∈P~​(f)M\in K_{0}\Leftrightarrow h(M)\in\tilde{P}(f)

∎

Lemma 3.

K0¯≀1P~​(f)\overline{K_{0}}\leq_{1}\tilde{P}(f) if f∈o​(t)f\in o(t) and fβˆˆΞ©β€‹(log⁑(t))f\in\Omega(\log(t))

Proof.

Similar to lemma 2, we will construct a one-one reduction, that transforms the TM MM to a non-terminating multi-taped TM g​(M)g(M). In contrast to lemma 2, Sg​(M)S_{g(M)} grows logarithmically when MM is non-terminating, and linearly otherwise.

Algorithm 2 g​(M):g(M):
0: multi-taped TM MM with empty input
0: algorithm runs on a TM that has one more tape than MM
 whileΒ MM not terminatedΒ do
  calculate one step on MM
  Reserve as much space on the last tape as is used by MM
   Overwrite reserved space with ’0”s
  repeat
   apply binary counter on the last tape
  untilΒ  reserved space is filled with ’11”s
 endΒ while
 ifΒ MM has terminatedΒ then
  loop
   write ’11’ on the last tape
    move the head of the last tape one position to the left
  endΒ loop
 endΒ if

If MM does not terminate, the tape space of g​(M)g(M) grows with the logarithm of time, so that

Mβˆ‰K0⇔g​(M)∈P~​(f)M\not\in K_{0}\Leftrightarrow g(M)\in\tilde{P}(f)

∎

Corollary 1.

K0<1P~​(f)K_{0}<_{1}\tilde{P}(f) if f∈o​(t)f\in o(t) and fβˆˆΞ©β€‹(log⁑(t))f\in\Omega(\log(t))

Proof.

K0≀1P~​(f)K_{0}\leq_{1}\tilde{P}(f) and K0¯≀1P~​(f)\overline{K_{0}}\leq_{1}\tilde{P}(f). But P~​(f)\tilde{P}(f) is neither in Ξ£1\Sigma_{1} nor in Ξ 1\Pi_{1}, due to the Hierarchy Theorem [Soa87, page 65]. So K0<1P~​(f)K_{0}<_{1}\tilde{P}(f) and K0Β―<1P~​(f)\overline{K_{0}}<_{1}\tilde{P}(f). ∎

Theorem 1.

P~​(f)∈Σ2\tilde{P}(f)\in\Sigma_{2}

Proof.

M∈P~​(f)β‡’βˆƒkβ€‹βˆ€t:S~M​(t)<kβˆ—l​(t)M\in\tilde{P}(f)\Rightarrow\exists k\forall t:\tilde{S}_{M}(t)<k*l(t) ∎

3 Space Hierarchy within 𝐏{\mathbf{P}}

In this section we use Turing-reduction instead of many-one-reduction because for any sets X≰TlogY⇒X≰mlogYX\not\leq_{T}^{\log}Y\;\Rightarrow\;X\not\leq_{m}^{\log}Y.

Theorem 2.

If hh and ll are space-constructible functions with l∈o​(h)l\in o(h) and lβˆˆΞ©β€‹(log)l\in\Omega(\log) then B​(h)β‰°TlogB​(l)B(h)\not\leq_{T}^{\log}B(l)

Proof.

Due to the space hierarchy theorem[SHI65], there is a set Xβˆˆπƒπ’ππ€π‚π„β€‹(h)X\in{\mathbf{DSPACE}}(h) with Xβˆ‰πƒπ’ππ€π‚π„β€‹(l)X\not\in{\mathbf{DSPACE}}(l). Thus X≀TlogB​(h)X\leq_{T}^{\log}B(h) and Xβ‰°TlogB​(l)X\not\leq_{T}^{\log}B(l) are valid. This implies B​(h)β‰°TlogB​(l)B(h)\not\leq_{T}^{\log}B(l). ∎

Lemma 4.

If hh and ll are space-constructible functions with l∈o​(h)l\in o(h) and l​(n)βˆˆΞ©β€‹(log⁑(n))l(n)\in\Omega(\log(n)) and h​(n)∈o​(n)h(n)\in o(n) then U​(h)β‰°TlogB​(l)U(h)\not\leq_{T}^{\log}B(l)

Proof.

Let MM be a TM and k>0k>0, both arbitrary but fixed. There is a function t:ℕ↦ℕt:\mathbb{N}\mapsto\mathbb{N} with MM accepting xx within t​(s)t(s) steps and within h​(s)h(s) tape space and |x|<k|x|<k. This means

βˆ€sβˆˆβ„•β€‹βˆ€|x|<k:(M,x,1t​(s),1s)∈U​(h)β‡’(M,x,1s)∈B​(h)\forall s\in\mathbb{N}\;\forall|x|<k:(M,x,1^{t(s)},1^{s})\in U(h)\Rightarrow(M,x,1^{s})\in B(h)

. In this case, there is no reduction function ff with the space complexity log⁑(s)\log(s) such that (M,x,1t​(s),1s)∈U​(h)⇔f​((M,x,1t​(s),1s))∈B​(l)(M,x,1^{t(s)},1^{s})\in U(h)\Leftrightarrow f\bigl{(}(M,x,1^{t(s)},1^{s})\bigr{)}\in B(l), because B​(l)<Tlog⁑(s)B​(h)B(l)<_{T}^{\log(s)}B(h). Due to corollary 1 it is undecidable whether there exists a function tt with βˆ€sβ€‹βˆ€|x|<k:(M,x,1t​(s),1s)∈U​(h)β‡’(M,x,1s)∈B​(h)\forall s\;\forall|x|<k:(M,x,1^{t(s)},1^{s})\in U(h)\Rightarrow(M,x,1^{s})\in B(h) and t∈O​(s)t\in O(s). So U​(h)β‰°TlogB​(l)U(h)\not\leq^{\log}_{T}B(l). ∎

Theorem 3.

If hh and ll are space-constructible functions with l∈o​(h)l\in o(h) and l​n​(n)βˆˆΞ©β€‹(log⁑(n))ln(n)\in\Omega(\log(n)) and h​(n)∈o​(n)h(n)\in o(n) then U​(h)β‰°TlogU​(l)U(h)\not\leq_{T}^{\log}U(l)

Proof.

U​(h)β‰°TlogB​(l)U(h)\not\leq_{T}^{\log}B(l), but U​(l)≀TlogB​(l)U(l)\leq_{T}^{\log}B(l) ∎

Corollary 2.

If k<nk<n then U​(logk)<mlogU​(logn)U(\log^{k})<_{m}^{\log}U(\log^{n})

Proof.

U​(logk)<TlogU​(logn)β‡’U​(logk)<mlogU​(logn)U(\log^{k})<_{T}^{\log}U(\log^{n})\;\Rightarrow\;U(\log^{k})<_{m}^{\log}U(\log^{n}) ∎

This means βˆ€n:U​(logn)<mlogA\forall n:U(\log^{n})<_{m}^{\log}A, so U​(logn)U(\log^{n}) is incomplete in 𝐏{\mathbf{P}}. From the existence of incomplete sets follows:

Corollary 3.

𝐋≠𝐏{\mathbf{L}}\not={\mathbf{P}}

4 Notes on the Relativization Barrier

To separate 𝐋{\mathbf{L}} and 𝐏{\mathbf{P}}, the relativization barrier applies as for 𝐏{\mathbf{P}} versus 𝐍𝐏{\mathbf{NP}} [BGS75]. Therefore, here we have mentioned the reason why the proof in this paper does not violate this barrier such as diagonalization. Trivially, U​(log)P=APU(\log)^{P}=A^{P}, so 𝐋P=PP{\mathbf{L}}^{P}=P^{P}. But from theorem 2 follows U​(log)<TlogU​(log2)U(\log)<^{\log}_{T}U(\log^{2}), so U​(log)𝐋≠A𝐋U(\log)^{\mathbf{L}}\not=A^{\mathbf{L}}.

Acknowledgments

Special thanks go to Lance Fortnow. He found several errors in the previous version of the paper[Cze21], especially in section 2. Thanks to Sonja Kutscher and Wolfgang Mulzer for improving some wordings. Thanks to the proof reader.

References

  • [BGS75] Theodore Baker, John Gill, and Robert Solovay. Relativizations of the p=?np question. SIAM Journal on computing, 4(4):431–442, 1975.
  • [Cze21] Reiner Czerwinski. Separation of PSPACE and EXP. https://arxiv.org/pdf/2104.14316.pdf, 2021.
  • [HPV75] John Hopcroft, Wolfgang Paul, and Leslie Valiant. On time versus space and related problems. In 16th Annual Symposium on Foundations of Computer Science (sfcs 1975), pages 57–64. IEEE, 1975.
  • [HS11] Steven Homer and AlanΒ L. Selman. Computability and Complexity Theory, Second Edition. Texts in Computer Science. Springer, 2011.
  • [SHI65] RichardΒ Edwin Stearns, Juris Hartmanis, and Philip M.Β Lewis II. Hierarchies of memory limited computations. In 6th Annual Symposium on Switching Circuit Theory and Logical Design, Ann Arbor, Michigan, USA, October 6-8, 1965, pages 179–190. IEEE Computer Society, 1965.
  • [Soa87] R.I. Soare. Recursively Enumerable Sets and Degrees: A Study of Computable Functions and Computably Generated Sets. Perspectives in mathematical logic. Springer-Verlag, 1987.
  • [Tur36] AlanΒ Mathison Turing. On computable numbers, with an application to the entscheidungsproblem. J. of Math, 58(345-363):5, 1936.