src/ZF/Tools/numeral_syntax.ML
changeset 32960 69916a850301
parent 26190 cf51a23c0cd0
child 35112 ff6f60e6ab85
--- a/src/ZF/Tools/numeral_syntax.ML	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/Tools/numeral_syntax.ML	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      ZF/Tools/numeral_syntax.ML
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
 
 Concrete syntax for generic numerals.  Assumes consts and syntax of
@@ -37,12 +36,12 @@
 
 fun mk_bin i =
   let fun bin_of_int 0  = []
-  	    | bin_of_int ~1 = [~1]
-    	| bin_of_int n  = (n mod 2) :: bin_of_int (n div 2);
+        | bin_of_int ~1 = [~1]
+        | bin_of_int n  = (n mod 2) :: bin_of_int (n div 2);
 
       fun term_of [] = @{const Pls}
-	    | term_of [~1] = @{const Min}
-	    | term_of (b :: bs) = @{const Bit} $ term_of bs $ mk_bit b;
+            | term_of [~1] = @{const Min}
+            | term_of (b :: bs) = @{const Bit} $ term_of bs $ mk_bit b;
   in
     term_of (bin_of_int i)
   end;
@@ -72,9 +71,9 @@
   let
     val rev_digs = bin_of t;
     val (sign, zs) =
-	(case rev rev_digs of
-	     ~1 :: bs => ("-", prefix_len (equal 1) bs)
-	   | bs =>       ("",  prefix_len (equal 0) bs));
+        (case rev rev_digs of
+             ~1 :: bs => ("-", prefix_len (equal 1) bs)
+           | bs =>       ("",  prefix_len (equal 0) bs));
     val num = string_of_int (abs (integ_of rev_digs));
   in
     "#" ^ sign ^ implode (replicate zs "0") ^ num