diff -r 5bc338cee4a0 -r dd675800469d src/HOL/Real.thy --- a/src/HOL/Real.thy Wed Oct 09 23:00:52 2019 +0200 +++ b/src/HOL/Real.thy Wed Oct 09 14:51:54 2019 +0000 @@ -816,7 +816,7 @@ then have "\n. y < r * 2 ^ n" by (metis divide_less_eq less_trans mult.commute of_nat_less_two_power that) then show ?thesis - by (simp add: divide_simps) + by (simp add: field_split_simps) qed have PA: "\ P (A n)" for n by (induct n) (simp_all add: a)