src/ZF/Int_ZF.thy
changeset 32960 69916a850301
parent 26056 6a0801279f4c
child 41777 1f7cbe39d425
--- a/src/ZF/Int_ZF.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/Int_ZF.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,8 +1,6 @@
 (*  Title:      ZF/Int.thy
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1993  University of Cambridge
-
 *)
 
 header{*The Integers as Equivalence Classes Over Pairs of Natural Numbers*}
@@ -55,7 +53,7 @@
   --{*could be replaced by an absolute value function from int to int?*}
     "zmagnitude(z) ==
      THE m. m\<in>nat & ((~ znegative(z) & z = $# m) |
-		       (znegative(z) & $- z = $# m))"
+                       (znegative(z) & $- z = $# m))"
 
 definition
   raw_zmult   ::      "[i,i]=>i"  where