src/HOL/Lattices.thy
changeset 24640 85a6c200ecd3
parent 24514 540eaf87e42d
child 24749 151b3758f576
--- a/src/HOL/Lattices.thy	Tue Sep 18 18:51:07 2007 +0200
+++ b/src/HOL/Lattices.thy	Tue Sep 18 18:52:17 2007 +0200
@@ -289,8 +289,7 @@
   fix x y z
   show "max x (min y z) = min (max x y) (max x z)"
   unfolding min_def max_def
-    by (auto simp add: intro: antisym, unfold not_le,
-      auto intro: less_trans le_less_trans aux)
+  by auto
 qed (auto simp add: min_def max_def not_le less_imp_le)
 
 interpretation min_max: