src/HOL/Library/Commutative_Ring.thy
changeset 27368 9f90ac19e32b
parent 25595 6c48275f9c76
child 27487 c8a6ce181805
--- a/src/HOL/Library/Commutative_Ring.thy	Thu Jun 26 10:06:54 2008 +0200
+++ b/src/HOL/Library/Commutative_Ring.thy	Thu Jun 26 10:07:01 2008 +0200
@@ -7,7 +7,7 @@
 header {* Proving equalities in commutative rings *}
 
 theory Commutative_Ring
-imports List Parity
+imports Plain List Parity
 uses ("comm_ring.ML")
 begin