diff -r 8d2cc27f45f3 -r 4805c6333fef Correctness.thy --- a/Correctness.thy Thu Jan 28 14:26:10 2016 +0000 +++ b/Correctness.thy Thu Jan 28 14:57:36 2016 +0000 @@ -802,7 +802,7 @@ *} lemma live: "runing (t @ s) \ {}" -proof(cases "th \ runing (t@s)") +proof(cases "th \ runing (t @ s)") case True thus ?thesis by auto next case False