diff -r bac8921e2901 -r d56e4eeae967 src/HOL/Real.thy --- a/src/HOL/Real.thy Wed Nov 11 11:27:44 2020 +0000 +++ b/src/HOL/Real.thy Wed Nov 11 14:27:17 2020 +0000 @@ -950,24 +950,6 @@ lifting_forget real.lifting -subsection \More Lemmas\ - -text \BH: These lemmas should not be necessary; they should be - covered by existing simp rules and simplification procedures.\ - -lemma real_mult_less_iff1 [simp]: "0 < z \ x * z < y * z \ x < y" - for x y z :: real - by simp (* solved by linordered_ring_less_cancel_factor simproc *) - -lemma real_mult_le_cancel_iff1 [simp]: "0 < z \ x * z \ y * z \ x \ y" - for x y z :: real - by simp (* solved by linordered_ring_le_cancel_factor simproc *) - -lemma real_mult_le_cancel_iff2 [simp]: "0 < z \ z * x \ z * y \ x \ y" - for x y z :: real - by simp (* solved by linordered_ring_le_cancel_factor simproc *) - - subsection \Embedding numbers into the Reals\ abbreviation real_of_nat :: "nat \ real"