src/HOL/Multivariate_Analysis/Extended_Real_Limits.thy
changeset 45051 c478d1876371
parent 45032 5a4d62f9e88d
child 47761 dfe747e72fa8
--- a/src/HOL/Multivariate_Analysis/Extended_Real_Limits.thy	Thu Sep 22 13:17:14 2011 -0700
+++ b/src/HOL/Multivariate_Analysis/Extended_Real_Limits.thy	Thu Sep 22 14:12:16 2011 -0700
@@ -667,7 +667,7 @@
        using a[rule_format, of "{B<..}"] mono_greaterThan by auto
     { fix y assume "y:(S Int ball x d - {x})"
       hence "y:S & 0 < dist y x & dist y x < d" unfolding ball_def apply (simp add: dist_commute)
-         by (metis dist_eq_0_iff real_less_def zero_le_dist)
+         by (metis dist_eq_0_iff less_le zero_le_dist)
       hence "B <= f y" using d_def by auto
     } hence "B <= INFI (S Int ball x d - {x}) f" apply (subst INF_greatest) by auto
     also have "...<=?l" apply (subst SUP_upper) using d_def by auto
@@ -714,7 +714,7 @@
        using a[rule_format, of "{..<B}"] by auto
     { fix y assume "y:(S Int ball x d - {x})"
       hence "y:S & 0 < dist y x & dist y x < d" unfolding ball_def apply (simp add: dist_commute)
-         by (metis dist_eq_0_iff real_less_def zero_le_dist)
+         by (metis dist_eq_0_iff less_le zero_le_dist)
       hence "f y <= B" using d_def by auto
     } hence "SUPR (S Int ball x d - {x}) f <= B" apply (subst SUP_least) by auto
     moreover have "?l<=SUPR (S Int ball x d - {x}) f" apply (subst INF_lower) using d_def by auto