src/HOL/Imperative_HOL/Heap_Monad.thy
changeset 37816 e550439d4422
parent 37792 ba0bc31b90d7
child 37828 9e1758c7ff06
--- a/src/HOL/Imperative_HOL/Heap_Monad.thy	Wed Jul 14 12:27:43 2010 +0200
+++ b/src/HOL/Imperative_HOL/Heap_Monad.thy	Wed Jul 14 12:27:44 2010 +0200
@@ -266,10 +266,9 @@
 
 setup {*
   Adhoc_Overloading.add_variant 
-    @{const_name Monad_Syntax.bindM} @{const_name Heap_Monad.bind}
+    @{const_name Monad_Syntax.bind} @{const_name Heap_Monad.bind}
 *}
 
-
 lemma execute_bind [execute_simps]:
   "execute f h = Some (x, h') \<Longrightarrow> execute (f \<guillemotright>= g) h = execute (g x) h'"
   "execute f h = None \<Longrightarrow> execute (f \<guillemotright>= g) h = None"