src/HOL/GCD.thy
changeset 33318 ddd97d9dfbfb
parent 33197 de6285ebcc05
child 33657 a4179bf442d1
--- a/src/HOL/GCD.thy	Thu Oct 29 08:14:39 2009 +0100
+++ b/src/HOL/GCD.thy	Thu Oct 29 11:41:36 2009 +0100
@@ -28,7 +28,7 @@
 header {* GCD *}
 
 theory GCD
-imports Fact
+imports Fact Parity
 begin
 
 declare One_nat_def [simp del]