| changeset 70817 | dd675800469d |
| parent 70356 | 4a327c061870 |
| child 71043 | 2fab72ab919a |
--- 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 "\<exists>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: "\<not> P (A n)" for n by (induct n) (simp_all add: a)