diff -r b388dceee892 -r 816e84ca16d6 thys/turing_basic.thy --- a/thys/turing_basic.thy Fri Jan 18 13:03:09 2013 +0000 +++ b/thys/turing_basic.thy Fri Jan 18 13:56:35 2013 +0000 @@ -71,7 +71,7 @@ fun step :: "config \ tprog \ config" where "step (s, l, r) (p, off) = - (let (a, s') = fetch p (s - off) (read r) in (s', update a (l, r)))" + (let (a, s') = fetch p (s - off) (read r) in (s', update a (l, r)))" fun steps :: "config \ tprog \ nat \ config" where @@ -93,7 +93,6 @@ (\(a, s) \ set p. s \ length p div 2 + off \ s \ off))" -(* FIXME: needed? *) lemma halt_lemma: "\wf LE; \n. (\ P (f n) \ (f (Suc n), (f n)) \ LE)\ \ \n. P (f n)" by (metis wf_iff_no_infinite_down_chain)