--- 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 \<Rightarrow> tape \<Rightarrow> bool"
where
- "inv_end2 x (l, r) = (\<exists> i j. i + j = Suc x \<and> x > 0 \<and> l = Oc\<up>i @ [Bk] \<and> r = Bk\<up>j @ Oc\<up>)"
+ "inv_end2 x (l, r) = (\<exists> i j. i + j = Suc x \<and> x > 0 \<and> l = Oc\<up>i @ [Bk] \<and> r = Bk\<up>j @ Oc\<up>x)"
fun inv_end3 :: "nat \<Rightarrow> tape \<Rightarrow> bool"
where