diff -r 2f765afc1f7e -r 9192a969f044 thys/uncomputable.thy --- a/thys/uncomputable.thy Wed Jan 16 10:12:43 2013 +0000 +++ b/thys/uncomputable.thy Wed Jan 16 10:20:49 2013 +0000 @@ -696,7 +696,7 @@ fun inv_end2 :: "nat \ tape \ bool" where - "inv_end2 x (l, r) = (\ i j. i + j = Suc x \ x > 0 \ l = Oc\i @ [Bk] \ r = Bk\j @ Oc\)" + "inv_end2 x (l, r) = (\ i j. i + j = Suc x \ x > 0 \ l = Oc\i @ [Bk] \ r = Bk\j @ Oc\x)" fun inv_end3 :: "nat \ tape \ bool" where