Theory Multi_Single_TM_Translation
section ‹Translating Multitape TMs to Singletape TMs›
text ‹In this section we define the mapping from a multitape Turing machine to a singletape
Turing machine. We further define soundness of the translation via several relations
which establish a connection between configurations of both kinds of Turing machines.
The translation works both for deterministic and non-deterministic TMs. Moreover,
we verify a quadratic overhead in runtime.
›
theory Multi_Single_TM_Translation
imports
Multitape_TM
Singletape_TM
STM_Renaming
begin
subsection ‹Definition of the Translation›