src/HOL/Lattices.thy
changeset 23018 1d29bc31b0cb
parent 22916 8caf6da610e2
child 23087 ad7244663431
--- a/src/HOL/Lattices.thy	Sat May 19 11:33:21 2007 +0200
+++ b/src/HOL/Lattices.thy	Sat May 19 11:33:22 2007 +0200
@@ -282,7 +282,7 @@
   special case of @{const inf}/@{const sup} *}
 
 lemma (in linorder) distrib_lattice_min_max:
-  "distrib_lattice_pred (op \<^loc>\<le>) (op \<^loc><) min max"
+  "distrib_lattice (op \<^loc>\<le>) (op \<^loc><) min max"
 proof unfold_locales
   have aux: "\<And>x y \<Colon> 'a. x \<^loc>< y \<Longrightarrow> y \<^loc>\<le> x \<Longrightarrow> x = y"
     by (auto simp add: less_le antisym)