src/HOL/Library/Heap_Monad.thy
changeset 28562 4e74209f113e
parent 28145 af3923ed4786
child 28663 bd8438543bf2
--- a/src/HOL/Library/Heap_Monad.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/Library/Heap_Monad.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -266,14 +266,14 @@
 definition
   Fail :: "message_string \<Rightarrow> exception"
 where
-  [code func del]: "Fail s = Exn"
+  [code del]: "Fail s = Exn"
 
 definition
   raise_exc :: "exception \<Rightarrow> 'a Heap"
 where
-  [code func del]: "raise_exc e = raise []"
+  [code del]: "raise_exc e = raise []"
 
-lemma raise_raise_exc [code func, code inline]:
+lemma raise_raise_exc [code, code inline]:
   "raise s = raise_exc (Fail (STR s))"
   unfolding Fail_def raise_exc_def raise_def ..