src/ZF/ex/Primes.thy
changeset 32960 69916a850301
parent 24893 b8ef7afe3a6b
child 45602 2a858377c3d2
--- a/src/ZF/ex/Primes.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/ex/Primes.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      ZF/ex/Primes.thy
-    ID:         $Id$
     Author:     Christophe Tabacznyj and Lawrence C Paulson
     Copyright   1996  University of Cambridge
 *)
@@ -20,8 +19,8 @@
 definition
   gcd     :: "[i,i]=>i"       --{*Euclid's algorithm for the gcd*}  where
     "gcd(m,n) == transrec(natify(n),
-			%n f. \<lambda>m \<in> nat.
-			        if n=0 then m else f`(m mod n)`n) ` natify(m)"
+                        %n f. \<lambda>m \<in> nat.
+                                if n=0 then m else f`(m mod n)`n) ` natify(m)"
 
 definition
   coprime :: "[i,i]=>o"       --{*the coprime relation*}  where