src/HOL/Library/Abstract_Rat.thy
changeset 27368 9f90ac19e32b
parent 26509 294708d83e83
child 27556 292098f2efdf
--- a/src/HOL/Library/Abstract_Rat.thy	Thu Jun 26 10:06:54 2008 +0200
+++ b/src/HOL/Library/Abstract_Rat.thy	Thu Jun 26 10:07:01 2008 +0200
@@ -6,7 +6,7 @@
 header {* Abstract rational numbers *}
 
 theory Abstract_Rat
-imports GCD
+imports Plain GCD
 begin
 
 types Num = "int \<times> int"