src/HOL/ex/CodeCollections.thy
changeset 22384 33a46e6c7f04
parent 22179 1a3575de2afc
child 22473 753123c89d72
--- a/src/HOL/ex/CodeCollections.thy	Fri Mar 02 12:38:58 2007 +0100
+++ b/src/HOL/ex/CodeCollections.thy	Fri Mar 02 15:43:15 2007 +0100
@@ -17,9 +17,6 @@
 abbreviation (in ord)
   "sorted \<equiv> abs_sorted less_eq"
 
-abbreviation
-  "sorted \<equiv> abs_sorted less_eq"
-
 lemma (in order) sorted_weakening:
   assumes "sorted (x # xs)"
   shows "sorted xs"
@@ -138,7 +135,7 @@
 apply (simp_all add: "fin_*_def")
 apply (unfold split_paired_all)
 apply (rule product_all)
-apply (rule finite_class.member_fin)+
+apply (rule member_fin)+
 done
 
 instance option :: (finite) finite
@@ -149,7 +146,7 @@
   proof (cases x)
     case None then show ?thesis by auto
   next
-    case (Some x) then show ?thesis by (auto intro: finite_class.member_fin)
+    case (Some x) then show ?thesis by (auto intro: member_fin)
   qed
 qed