src/HOL/Library/Fraction_Field.thy
changeset 35372 ca158c7b1144
parent 31998 2c7a24f74db9
child 36312 26eea417ccc4
--- a/src/HOL/Library/Fraction_Field.thy	Wed Feb 24 14:19:54 2010 +0100
+++ b/src/HOL/Library/Fraction_Field.thy	Wed Feb 24 14:34:40 2010 +0100
@@ -1,12 +1,12 @@
-(*  Title:      Fraction_Field.thy
+(*  Title:      HOL/Library/Fraction_Field.thy
     Author:     Amine Chaieb, University of Cambridge
 *)
 
 header{* A formalization of the fraction field of any integral domain 
-         A generalization of Rational.thy from int to any integral domain *}
+         A generalization of Rat.thy from int to any integral domain *}
 
 theory Fraction_Field
-imports Main (* Equiv_Relations Plain *)
+imports Main
 begin
 
 subsection {* General fractions construction *}