src/ZF/ex/Bin.thy
changeset 4709 d24168720303
parent 3795 e687069e7257
child 5512 4327eec06849
--- a/src/ZF/ex/Bin.thy	Mon Mar 09 16:15:24 1998 +0100
+++ b/src/ZF/ex/Bin.thy	Mon Mar 09 16:16:21 1998 +0100
@@ -117,7 +117,7 @@
   fun mk_bin str =
     let
       val (sign, digs) =
-        (case explode str of
+        (case Symbol.explode str of
           "#" :: "~" :: cs => (~1, cs)
         | "#" :: cs => (1, cs)
         | _ => raise ERROR);
@@ -132,7 +132,7 @@
         | term_of [~1] = const "Minus"
         | term_of (b :: bs) = const "Bcons" $ term_of bs $ mk_bit b;
     in
-      term_of (bin_of (sign * (#1 (scan_int digs))))
+      term_of (bin_of (sign * (#1 (read_int digs))))
     end;
 
   fun dest_bin tm =