# HG changeset patch # User Christian Urban # Date 1369442011 -3600 # Node ID bc2df9620f26f02d8a0facec46b9bc539d1ca3be # Parent aa102c18213287fa15785961811577f4d2082956 tuned diff -r aa102c182132 -r bc2df9620f26 thys2/UF_Rec.thy --- a/thys2/UF_Rec.thy Sat May 25 01:32:35 2013 +0100 +++ b/thys2/UF_Rec.thy Sat May 25 01:33:31 2013 +0100 @@ -699,47 +699,6 @@ by (simp add: rec_uf_def) -subsection {* Relating interperter functions to the execution of TMs *} - -lemma rec_step: - assumes "(\ (s, l, r). s \ length tp div 2) c" - shows "Trpl_code (step0 c tp) = Newconf (Code tp) (Trpl_code c)" -apply(cases c) -apply(simp only: Trpl_code.simps) -apply(simp only: Let_def step.simps) -apply(case_tac "fetch tp (a - 0) (read ca)") -apply(simp only: prod.cases) -apply(case_tac "update aa (b, ca)") -apply(simp only: prod.cases) -apply(simp only: Trpl_code.simps) -apply(simp only: Newconf.simps) -apply(simp only: Left.simps) -oops - -lemma rec_steps: - assumes "tm_wf0 tp" - shows "Trpl_code (steps0 (1, Bk \ l, ) tp stp) = Conf stp (Code tp) (bl2wc ())" -apply(induct stp) -apply(simp) -apply(simp) -oops - - -lemma F_correct: - assumes tm: "steps0 (1, Bk \ l, ) tp stp = (0, Bk \ m, Oc \ rs @ Bk \ n)" - and wf: "tm_wf0 tp" "0 < rs" - shows "rec_eval rec_uf [Code tp, bl2wc ()] = (rs - Suc 0)" -proof - - from least_steps[OF tm] - obtain stp_least where - before: "\stp' < stp_least. \ is_final (steps0 (1, Bk \ l, ) tp stp')" and - after: "\stp' \ stp_least. is_final (steps0 (1, Bk \ l, ) tp stp')" by blast - have "Halt (Code tp) (bl2wc ()) = stp_least" sorry - show ?thesis - apply(simp only: uf_lemma) - apply(simp only: UF.simps) - apply(simp only: Halt.simps) - oops end