src/HOL/ex/Termination.thy
changeset 61933 cf58b5b794b2
parent 61343 5b5656a63bd6
child 66453 cc19f7ca2ed6
--- a/src/HOL/ex/Termination.thy	Sat Dec 26 15:44:14 2015 +0100
+++ b/src/HOL/ex/Termination.thy	Sat Dec 26 15:59:27 2015 +0100
@@ -9,7 +9,7 @@
 imports Main "~~/src/HOL/Library/Multiset"
 begin
 
-subsection \<open>Manually giving termination relations using @{text relation} and
+subsection \<open>Manually giving termination relations using \<open>relation\<close> and
 @{term measure}\<close>
 
 function sum :: "nat \<Rightarrow> nat \<Rightarrow> nat"
@@ -29,10 +29,10 @@
 termination by (relation "measures [\<lambda>(i, N). N, \<lambda>(i,N). N + 1 - i]") auto
 
 
-subsection \<open>@{text lexicographic_order}: Trivial examples\<close>
+subsection \<open>\<open>lexicographic_order\<close>: Trivial examples\<close>
 
 text \<open>
-  The @{text fun} command uses the method @{text lexicographic_order} by default,
+  The \<open>fun\<close> command uses the method \<open>lexicographic_order\<close> by default,
   so it is not explicitly invoked.
 \<close>
 
@@ -168,9 +168,9 @@
 
 
 
-subsection \<open>Refined analysis: The @{text size_change} method\<close>
+subsection \<open>Refined analysis: The \<open>size_change\<close> method\<close>
 
-text \<open>Unsolvable for @{text lexicographic_order}\<close>
+text \<open>Unsolvable for \<open>lexicographic_order\<close>\<close>
 
 function fun1 :: "nat * nat \<Rightarrow> nat"
 where
@@ -183,7 +183,7 @@
 
 
 text \<open>
-  @{text lexicographic_order} can do the following, but it is much slower. 
+  \<open>lexicographic_order\<close> can do the following, but it is much slower. 
 \<close>
 
 function
@@ -227,7 +227,7 @@
            0
       )"
 by pat_completeness auto
-termination by size_change -- \<open>requires Multiset\<close>
+termination by size_change \<comment> \<open>requires Multiset\<close>
 
 definition negate :: "int \<Rightarrow> int"
 where "negate i = - i"