src/HOL/Library/Commutative_Ring.thy
changeset 28952 15a4b2cf8c34
parent 27487 c8a6ce181805
child 29667 53103fc8ffa3
--- a/src/HOL/Library/Commutative_Ring.thy	Wed Dec 03 09:53:58 2008 +0100
+++ b/src/HOL/Library/Commutative_Ring.thy	Wed Dec 03 15:58:44 2008 +0100
@@ -1,5 +1,4 @@
-(*  ID:         $Id$
-    Author:     Bernhard Haeupler
+(*  Author:     Bernhard Haeupler
 
 Proving equalities in commutative rings done "right" in Isabelle/HOL.
 *)
@@ -7,7 +6,7 @@
 header {* Proving equalities in commutative rings *}
 
 theory Commutative_Ring
-imports Plain "~~/src/HOL/List" Parity
+imports Plain "~~/src/HOL/List" "~~/src/HOL/Parity"
 uses ("comm_ring.ML")
 begin