src/HOL/Lattices.thy
changeset 30729 461ee3e49ad3
parent 30302 5ffa9d4dbea7
child 31991 37390299214a
--- a/src/HOL/Lattices.thy	Thu Mar 26 19:24:21 2009 +0100
+++ b/src/HOL/Lattices.thy	Thu Mar 26 20:08:55 2009 +0100
@@ -299,7 +299,7 @@
   by auto
 qed (auto simp add: min_def max_def not_le less_imp_le)
 
-interpretation min_max!: distrib_lattice "op \<le> :: 'a::linorder \<Rightarrow> 'a \<Rightarrow> bool" "op <" min max
+interpretation min_max: distrib_lattice "op \<le> :: 'a::linorder \<Rightarrow> 'a \<Rightarrow> bool" "op <" min max
   by (rule distrib_lattice_min_max)
 
 lemma inf_min: "inf = (min \<Colon> 'a\<Colon>{lower_semilattice, linorder} \<Rightarrow> 'a \<Rightarrow> 'a)"