# HG changeset patch # User haftmann # Date 1268916993 -3600 # Node ID b57c3afd14841edfebb5fadac16bc57e8bdae896 # Parent 8e81f71d0460fade0a9c3eaec3dcef7ee87c07e5 dropped odd interpretation of comm_monoid_mult into comm_monoid_add; consider Min.insert_idem as default simp rule diff -r 8e81f71d0460 -r b57c3afd1484 src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy --- a/src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy Thu Mar 18 13:56:32 2010 +0100 +++ b/src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy Thu Mar 18 13:56:33 2010 +0100 @@ -1459,7 +1459,7 @@ { fix x::"'a" assume "x \ 0 \ dist x 0 < d" hence "f (a + x) \ S" using d apply(erule_tac x="x+a" in allE) - by(auto simp add: comm_monoid_add.mult_commute dist_norm dist_commute) + by (auto simp add: add_commute dist_norm dist_commute) } hence "\d>0. \x. x \ 0 \ dist x 0 < d \ f (a + x) \ S" using d(1) by auto @@ -1476,7 +1476,7 @@ unfolding Limits.eventually_at by fast { fix x::"'a" assume "x \ a \ dist x a < d" hence "f x \ S" using d apply(erule_tac x="x-a" in allE) - by(auto simp add: comm_monoid_add.mult_commute dist_norm dist_commute) + by(auto simp add: add_commute dist_norm dist_commute) } hence "\d>0. \x. x \ a \ dist x a < d \ f x \ S" using d(1) by auto hence "eventually (\x. f x \ S) (at a)" unfolding Limits.eventually_at . @@ -2755,8 +2755,8 @@ have "d>0" using `e>0` unfolding d_def e_def using zero_le_dist[of _ l', unfolded order_le_less] by auto obtain k where k:"f k \ l'" "dist (f k) l' < d" using `d>0` and assms(3)[unfolded islimpt_approachable, THEN spec[where x="d"]] by auto have "k\N" using k(1)[unfolded dist_nz] using k(2)[unfolded d_def] - by force - hence "dist l' l < e" using N[THEN spec[where x=k]] using k(2)[unfolded d_def] and dist_triangle_half_r[of "f k" l' e l] by auto + by (force simp del: Min.insert_idem) + hence "dist l' l < e" using N[THEN spec[where x=k]] using k(2)[unfolded d_def] and dist_triangle_half_r[of "f k" l' e l] by (auto simp del: Min.insert_idem) thus False unfolding e_def by auto qed