src/HOL/ex/Parallel_Example.thy
changeset 61933 cf58b5b794b2
parent 61433 a4c0de1df3d8
child 63882 018998c00003
--- 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' \<Rightarrow> let n = m - length ps' in takeWhile Not ps @ p # sieve m (mark n n ps'))"
 by pat_completeness auto
 
-termination -- \<open>tuning of this proof is left as an exercise to the reader\<close>
+termination \<comment> \<open>tuning of this proof is left as an exercise to the reader\<close>
   apply (relation "measure (length \<circ> snd)")
   apply rule
   apply (auto simp add: length_dropWhile_le)
@@ -67,7 +67,7 @@
     else [])" 
 by pat_completeness auto
 
-termination factorise_from -- \<open>tuning of this proof is left as an exercise to the reader\<close>
+termination factorise_from \<comment> \<open>tuning of this proof is left as an exercise to the reader\<close>
 term measure
 apply (relation "measure (\<lambda>(k, n). 2 * n - k)")
 apply (auto simp add: prod_eq_iff)