src/HOL/Library/Fraction_Field.thy
changeset 39910 10097e0a9dbd
parent 37765 26bdfb7b680b
child 40815 6e2d17cc0d1d
--- a/src/HOL/Library/Fraction_Field.thy	Fri Oct 01 14:15:49 2010 +0200
+++ b/src/HOL/Library/Fraction_Field.thy	Fri Oct 01 16:05:25 2010 +0200
@@ -319,7 +319,7 @@
 
 definition
   le_fract_def:
-   "q \<le> r \<longleftrightarrow> contents (\<Union>x \<in> Rep_fract q. \<Union>y \<in> Rep_fract r.
+   "q \<le> r \<longleftrightarrow> the_elem (\<Union>x \<in> Rep_fract q. \<Union>y \<in> Rep_fract r.
       {(fst x * snd y)*(snd x * snd y) \<le> (fst y * snd x)*(snd x * snd y)})"
 
 definition