src/HOL/Integ/Bin.thy
changeset 3795 e687069e7257
parent 2988 d38f330e58b3
child 4709 d24168720303
--- a/src/HOL/Integ/Bin.thy	Mon Oct 06 19:15:02 1997 +0200
+++ b/src/HOL/Integ/Bin.thy	Mon Oct 06 19:15:22 1997 +0200
@@ -155,8 +155,8 @@
 
   fun int_tr (*"_Int"*) [t as Free (str, _)] =
         (const "integ_of_bin" $
-          (mk_bin str handle ERROR => raise_term "int_tr" [t]))
-    | int_tr (*"_Int"*) ts = raise_term "int_tr" ts;
+          (mk_bin str handle ERROR => raise TERM ("int_tr", [t])))
+    | int_tr (*"_Int"*) ts = raise TERM ("int_tr", ts);
 
   fun int_tr' (*"integ_of"*) [t] = const "_Int" $ free (dest_bin t)
     | int_tr' (*"integ_of"*) _ = raise Match;