diff -r 31d41a0f6b5d -r 8e6cdb9c00a7 src/HOL/Library/Extended_Real.thy --- a/src/HOL/Library/Extended_Real.thy Fri Sep 02 15:19:59 2011 -0700 +++ b/src/HOL/Library/Extended_Real.thy Fri Sep 02 16:48:30 2011 -0700 @@ -1110,7 +1110,7 @@ with `S \ {}` `\ \ S` obtain x where "x \ S - {-\}" "x \ \" by auto with y `\ \ S` have "\z\real ` (S - {-\}). z \ y" by (auto simp: real_of_ereal_ord_simps) - with reals_complete2[of "real ` (S - {-\})"] `x \ S - {-\}` + with complete_real[of "real ` (S - {-\})"] `x \ S - {-\}` obtain s where s: "\y\S - {-\}. real y \ s" "\z. (\y\S - {-\}. real y \ z) \ s \ z" by auto