diff -r 2e48182cc82c -r cf58b5b794b2 src/HOL/ex/Parallel_Example.thy --- a/src/HOL/ex/Parallel_Example.thy Sat Dec 26 15:44:14 2015 +0100 +++ b/src/HOL/ex/Parallel_Example.thy Sat Dec 26 15:59:27 2015 +0100 @@ -34,7 +34,7 @@ | p#ps' \ let n = m - length ps' in takeWhile Not ps @ p # sieve m (mark n n ps'))" by pat_completeness auto -termination -- \tuning of this proof is left as an exercise to the reader\ +termination \ \tuning of this proof is left as an exercise to the reader\ apply (relation "measure (length \ snd)") apply rule apply (auto simp add: length_dropWhile_le) @@ -67,7 +67,7 @@ else [])" by pat_completeness auto -termination factorise_from -- \tuning of this proof is left as an exercise to the reader\ +termination factorise_from \ \tuning of this proof is left as an exercise to the reader\ term measure apply (relation "measure (\(k, n). 2 * n - k)") apply (auto simp add: prod_eq_iff)