src/HOL/Lattices.thy
changeset 28823 dcbef866c9e2
parent 28692 a2bc5ce0c9fc
child 29223 e09c53289830
--- a/src/HOL/Lattices.thy	Mon Nov 17 17:00:27 2008 +0100
+++ b/src/HOL/Lattices.thy	Mon Nov 17 17:00:55 2008 +0100
@@ -291,7 +291,7 @@
 
 lemma (in linorder) distrib_lattice_min_max:
   "distrib_lattice (op \<le>) (op <) min max"
-proof unfold_locales
+proof
   have aux: "\<And>x y \<Colon> 'a. x < y \<Longrightarrow> y \<le> x \<Longrightarrow> x = y"
     by (auto simp add: less_le antisym)
   fix x y z