diff -r e33306b4c62e -r 35fe8fe12e65 thys/turing_basic.thy --- a/thys/turing_basic.thy Tue Jan 22 14:46:02 2013 +0000 +++ b/thys/turing_basic.thy Wed Jan 23 08:01:35 2013 +0100 @@ -174,6 +174,10 @@ "tm_wf (p, off) = (length p \ 2 \ length p mod 2 = 0 \ (\(a, s) \ set p. s \ length p div 2 + off \ s \ off))" +abbreviation + "tm_wf0 p \ tm_wf (p, 0)" + + 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)