src/HOL/Real/PReal.thy
changeset 14387 e96d5c42c4b0
parent 14378 69c4d5997669
child 14430 5cb24165a2e1
--- a/src/HOL/Real/PReal.thy	Sat Feb 14 02:06:12 2004 +0100
+++ b/src/HOL/Real/PReal.thy	Sun Feb 15 10:46:37 2004 +0100
@@ -7,7 +7,7 @@
                   provides some of the definitions.
 *)
 
-theory PReal = RatArith:
+theory PReal = Rational:
 
 text{*Could be generalized and moved to @{text Ring_and_Field}*}
 lemma add_eq_exists: "\<exists>x. a+x = (b::rat)"