tuned proof
authorhaftmann
Fri, 24 Oct 2008 17:48:36 +0200
changeset 28684 48faac324061
parent 28683 59c01ec6cb8d
child 28685 275122631271
tuned proof
src/HOL/Library/Enum.thy
--- a/src/HOL/Library/Enum.thy	Fri Oct 24 17:48:35 2008 +0200
+++ b/src/HOL/Library/Enum.thy	Fri Oct 24 17:48:36 2008 +0200
@@ -53,7 +53,7 @@
   fixes f g :: "'a\<Colon>enum \<Rightarrow> 'b\<Colon>order"
   shows "f \<le> g \<longleftrightarrow> list_all (\<lambda>x. f x \<le> g x) enum"
     and "f < g \<longleftrightarrow> f \<le> g \<and> \<not> list_all (\<lambda>x. f x = g x) enum"
-  by (simp_all add: list_all_iff enum_all expand_fun_eq le_fun_def less_fun_def order_less_le)
+  by (simp_all add: list_all_iff enum_all expand_fun_eq le_fun_def order_less_le)
 
 
 subsection {* Quantifiers *}