src/HOLCF/Completion.thy
changeset 30729 461ee3e49ad3
parent 29252 ea97aa6aeba2
child 31076 99fe356cbbc2
--- a/src/HOLCF/Completion.thy	Thu Mar 26 19:24:21 2009 +0100
+++ b/src/HOLCF/Completion.thy	Thu Mar 26 20:08:55 2009 +0100
@@ -156,7 +156,7 @@
 
 end
 
-interpretation sq_le!: preorder "sq_le :: 'a::po \<Rightarrow> 'a \<Rightarrow> bool"
+interpretation sq_le: preorder "sq_le :: 'a::po \<Rightarrow> 'a \<Rightarrow> bool"
 apply unfold_locales
 apply (rule refl_less)
 apply (erule (1) trans_less)