src/HOL/GCD.thy
changeset 58770 ae5e9b4f8daf
parent 58623 2db1df2c8467
child 58776 95e58e04e534
--- a/src/HOL/GCD.thy	Thu Oct 23 14:04:05 2014 +0200
+++ b/src/HOL/GCD.thy	Thu Oct 23 14:04:05 2014 +0200
@@ -28,7 +28,7 @@
 header {* Greatest common divisor and least common multiple *}
 
 theory GCD
-imports Fact Parity
+imports Fact
 begin
 
 declare One_nat_def [simp del]