IntEx.thy
changeset 232 38810e1df801
parent 228 268a727b0f10
child 239 02b14a21761a
--- a/IntEx.thy	Wed Oct 28 20:01:20 2009 +0100
+++ b/IntEx.thy	Thu Oct 29 07:29:12 2009 +0100
@@ -111,7 +111,7 @@
   done
 
 lemma ho_plus_rsp:
-  "IntEx.intrel ===> IntEx.intrel ===> IntEx.intrel my_plus my_plus"
+  "(intrel ===> intrel ===> intrel) my_plus my_plus"
   by (simp)
 
 ML {* val consts = [@{const_name "my_plus"}] *}