src/HOL/Orderings.thy
changeset 46884 154dc6ec0041
parent 46882 6242b4bc05bc
child 46950 d0181abdbdac
--- a/src/HOL/Orderings.thy	Mon Mar 12 15:12:22 2012 +0100
+++ b/src/HOL/Orderings.thy	Mon Mar 12 21:41:11 2012 +0100
@@ -1304,7 +1304,7 @@
   by (simp add: bot_fun_def)
 
 instance proof
-qed (simp add: le_fun_def bot_apply)
+qed (simp add: le_fun_def)
 
 end
 
@@ -1320,7 +1320,7 @@
   by (simp add: top_fun_def)
 
 instance proof
-qed (simp add: le_fun_def top_apply)
+qed (simp add: le_fun_def)
 
 end