src/HOL/GCD.thy
changeset 29655 ac31940cfb69
parent 28952 15a4b2cf8c34
child 29700 22faf21db3df
--- a/src/HOL/GCD.thy	Wed Jan 28 11:03:16 2009 +0100
+++ b/src/HOL/GCD.thy	Wed Jan 28 11:03:42 2009 +0100
@@ -1,5 +1,4 @@
 (*  Title:      HOL/GCD.thy
-    ID:         $Id$
     Author:     Christophe Tabacznyj and Lawrence C Paulson
     Copyright   1996  University of Cambridge
 *)
@@ -7,7 +6,7 @@
 header {* The Greatest Common Divisor *}
 
 theory GCD
-imports Plain Presburger
+imports Plain Presburger Main
 begin
 
 text {*