src/HOL/ex/CodeCollections.thy
changeset 21319 cf814e36f788
parent 21125 9b7d35ca1eef
child 21404 eb85850d3eb7
--- a/src/HOL/ex/CodeCollections.thy	Mon Nov 13 12:10:49 2006 +0100
+++ b/src/HOL/ex/CodeCollections.thy	Mon Nov 13 13:51:22 2006 +0100
@@ -72,8 +72,6 @@
 | "abs_sorted cmp [x] = True"
 | "abs_sorted cmp (x#y#xs) = (cmp x y \<and> abs_sorted cmp (y#xs))"
 
-termination by (auto_term "measure (length o snd)")
-
 thm abs_sorted.simps
 
 abbreviation (in ordered)
@@ -117,8 +115,6 @@
 | "le_option' (Some x) None = False"
 | "le_option' (Some x) (Some y) = x <<= y"
 
-termination by (auto_term "{}")
-
 instance option :: (ordered) ordered
   "x <<= y == le_option' x y"
 proof (default, unfold ordered_option_def)
@@ -147,7 +143,6 @@
 fun le_pair' :: "'a::ordered \<times> 'b::ordered \<Rightarrow> 'a \<times> 'b \<Rightarrow> bool"
 where
   "le_pair' (x1, y1) (x2, y2) = (x1 << x2 \<or> x1 = x2 \<and> y1 <<= y2)"
-termination by (auto_term "{}")
 
 instance * :: (ordered, ordered) ordered
   "x <<= y == le_pair' x y"
@@ -169,8 +164,6 @@
 | "le_list' (x#xs) [] = False"
 | "le_list' (x#xs) (y#ys) = (x << y \<or> x = y \<and> le_list' xs ys)"
 
-termination by (auto_term "measure (length o fst)")
-
 instance (ordered) list :: ordered
   "xs <<= ys == le_list' xs ys"
 proof (default, unfold "ordered_list_def")