src/HOL/Real/RealInt.ML
changeset 11713 883d559b0b8c
parent 11597 cd6d2eddf75f
child 12613 279facb4253a
--- a/src/HOL/Real/RealInt.ML	Mon Oct 08 14:30:28 2001 +0200
+++ b/src/HOL/Real/RealInt.ML	Mon Oct 08 15:23:20 2001 +0200
@@ -39,7 +39,7 @@
 by (simp_tac (simpset() addsimps [real_of_int, preal_add_commute]) 1);
 qed "real_of_int_zero";
 
-Goalw [int_def,real_one_def] "real (int 1) = 1r";
+Goalw [int_def,real_one_def] "real (int 1) = (1::real)";
 by (auto_tac (claset(),
 	      simpset() addsimps [real_of_int,
 				  preal_of_prat_add RS sym,pnat_two_eq,
@@ -80,7 +80,7 @@
 qed "real_of_int_mult";
 Addsimps [real_of_int_mult RS sym];
 
-Goal "real (int (Suc n)) = real (int n) + 1r";
+Goal "real (int (Suc n)) = real (int n) + (1::real)";
 by (simp_tac (simpset() addsimps [real_of_int_one RS sym, zadd_int] @ 
                                  zadd_ac) 1);
 qed "real_of_int_Suc";