src/HOL/PReal.thy
changeset 29197 6d4cb27ed19c
parent 28952 15a4b2cf8c34
child 29667 53103fc8ffa3
--- a/src/HOL/PReal.thy	Mon Dec 29 13:23:53 2008 +0100
+++ b/src/HOL/PReal.thy	Mon Dec 29 14:08:08 2008 +0100
@@ -9,7 +9,7 @@
 header {* Positive real numbers *}
 
 theory PReal
-imports Rational "~~/src/HOL/Library/Dense_Linear_Order"
+imports Rational Dense_Linear_Order
 begin
 
 text{*Could be generalized and moved to @{text Ring_and_Field}*}