diff -r 81d34cf268d8 -r 3c5040d5694a src/HOL/Multivariate_Analysis/Derivative.thy --- a/src/HOL/Multivariate_Analysis/Derivative.thy Tue Dec 08 20:21:59 2015 +0100 +++ b/src/HOL/Multivariate_Analysis/Derivative.thy Wed Dec 09 17:35:22 2015 +0000 @@ -290,13 +290,13 @@ unfolding eventually_nhds_metric by (safe, rule_tac x="d / 2" in exI, auto) lemma le_nhds: "F \ nhds a \ (\S. open S \ a \ S \ eventually (\x. x \ S) F)" - unfolding le_filter_def eventually_nhds by (fast elim: eventually_elim1) + unfolding le_filter_def eventually_nhds by (fast elim: eventually_mono) lemma le_nhds_metric: "F \ nhds a \ (\e>0. eventually (\x. dist x a < e) F)" - unfolding le_filter_def eventually_nhds_metric by (fast elim: eventually_elim1) + unfolding le_filter_def eventually_nhds_metric by (fast elim: eventually_mono) lemma le_nhds_metric_le: "F \ nhds a \ (\e>0. eventually (\x. dist x a \ e) F)" - unfolding le_filter_def eventually_nhds_metric_le by (fast elim: eventually_elim1) + unfolding le_filter_def eventually_nhds_metric_le by (fast elim: eventually_mono) text \Several results are easier using a "multiplied-out" variant. (I got this idea from Dieudonne's proof of the chain rule).\ @@ -2016,15 +2016,15 @@ case True have "eventually (\n. norm (f' n x u - g' x u) \ e * norm u) sequentially" using assms(3)[folded eventually_sequentially] and \0 < e\ and \x \ s\ - by (fast elim: eventually_elim1) + by (fast elim: eventually_mono) then show ?thesis - using \u = 0\ and \0 < e\ by (auto elim: eventually_elim1) + using \u = 0\ and \0 < e\ by (auto elim: eventually_mono) next case False with \0 < e\ have "0 < e / norm u" by simp then have "eventually (\n. norm (f' n x u - g' x u) \ e / norm u * norm u) sequentially" using assms(3)[folded eventually_sequentially] and \x \ s\ - by (fast elim: eventually_elim1) + by (fast elim: eventually_mono) then show ?thesis using \u \ 0\ by simp qed @@ -2250,7 +2250,7 @@ also have "(g has_field_derivative g' x) (at x) \ ((\x. \n. f n x) has_field_derivative g' x) (at x)" using eventually_nhds_in_nhd[OF \x \ interior s\] interior_subset[of s] g(1) - by (intro DERIV_cong_ev) (auto elim!: eventually_elim1 simp: sums_iff) + by (intro DERIV_cong_ev) (auto elim!: eventually_mono simp: sums_iff) finally show "((\x. \n. f n x) has_field_derivative g' x) (at x)" . qed