(* Title: thys/Turing.thy Author: Jian Xu, Xingyuan Zhang, and Christian Urban Modifications: Sebastiaan Joosten Modifications, comments by Franz Regensburger (FABR) 02/2022 *) chapter ‹Turing Machines› theory Turing imports Main begin section ‹Some lemmas about natural numbers used for rewriting› (* ------ Important properties used in subsequent theories ------ *) (* Num.numeral_1_eq_Suc_0: Numeral1 = Suc 0 Num.numeral_2_eq_2: 2 = Suc (Suc 0) Num.numeral_3_eq_3: 3 = Suc (Suc (Suc 0)) *) lemma numeral_4_eq_4: "4 = Suc 3" by auto lemma numeral_eqs_upto_12: shows "2 = Suc 1" and "3 = Suc 2" and "4 = Suc 3" and "5 = Suc 4" and "6 = Suc 5" and "7 = Suc 6" and "8 = Suc 7" and "9 = Suc 8" and "10 = Suc 9" and "11 = Suc 10" and "12 = Suc 11" by simp_all section ‹Basic Definitions for Turing Machines›