src/HOL/GCD.thy
changeset 30738 0842e906300c
parent 30242 aea5d7fa7ef5
child 31706 1db0c8f235fb
--- a/src/HOL/GCD.thy	Fri Mar 27 10:05:08 2009 +0100
+++ b/src/HOL/GCD.thy	Fri Mar 27 10:05:11 2009 +0100
@@ -6,7 +6,7 @@
 header {* The Greatest Common Divisor *}
 
 theory GCD
-imports Plain Presburger Main
+imports Main
 begin
 
 text {*