src/HOL/Lattices.thy
changeset 29223 e09c53289830
parent 28823 dcbef866c9e2
child 29509 1ff0f3f08a7b
--- a/src/HOL/Lattices.thy	Wed Dec 10 17:19:25 2008 +0100
+++ b/src/HOL/Lattices.thy	Thu Dec 11 18:30:26 2008 +0100
@@ -300,7 +300,7 @@
   by auto
 qed (auto simp add: min_def max_def not_le less_imp_le)
 
-interpretation min_max:
+class_interpretation min_max:
   distrib_lattice ["op \<le> \<Colon> 'a\<Colon>linorder \<Rightarrow> 'a \<Rightarrow> bool" "op <" min max]
   by (rule distrib_lattice_min_max)