Paper/Paper.thy
changeset 132 264ff7014657
parent 130 1e89c65f844b
child 133 ca7fb6848715
equal deleted inserted replaced
131:e995ae949731 132:264ff7014657
  1320 
  1320 
  1321   \noindent
  1321   \noindent
  1322   which means that if the recursive function @{text r} with arguments @{text ns} evaluates
  1322   which means that if the recursive function @{text r} with arguments @{text ns} evaluates
  1323   to @{text n}, then the corresponding Turing machine @{term "tm_of_rec r"} if started
  1323   to @{text n}, then the corresponding Turing machine @{term "tm_of_rec r"} if started
  1324   with the standard tape @{term "([Bk, Bk], <ns::nat list>)"} will terminate
  1324   with the standard tape @{term "([Bk, Bk], <ns::nat list>)"} will terminate
  1325   with the standard tape @{term "(Bk \<up> l, <n::nat> @ Bk \<up> m)"} for some @{text l} and @{text m}.
  1325   with the standard tape @{term "(Bk \<up> k, <n::nat> @ Bk \<up> l)"} for some @{text k} and @{text l}.
  1326 
  1326 
  1327   and the also the definition of the
  1327   and the also the definition of the
  1328   universal function (we refer the reader to our formalisation).
  1328   universal function (we refer the reader to our formalisation).
  1329   
  1329   
  1330 *}
  1330 *}