diff -r 758e7acdea2f -r cc61fd03e589 src/HOL/Hyperreal/NSA.thy --- a/src/HOL/Hyperreal/NSA.thy Fri Mar 19 10:50:06 2004 +0100 +++ b/src/HOL/Hyperreal/NSA.thy Fri Mar 19 10:51:03 2004 +0100 @@ -154,7 +154,7 @@ lemma SReal_dense: "[| (x::hypreal) \ Reals; y \ Reals; x \r \ Reals. x 0 < r/(2::hypreal)" -by auto - lemma Infinitesimal_add: "[| x \ Infinitesimal; y \ Infinitesimal |] ==> (x+y) \ Infinitesimal" apply (auto simp add: Infinitesimal_def) apply (rule hypreal_sum_of_halves [THEN subst]) -apply (drule hypreal_half_gt_zero) +apply (drule half_gt_zero) apply (blast intro: hrabs_add_less hrabs_add_less SReal_divide_number_of) done @@ -488,6 +485,9 @@ by (simp add: approx_def Infinitesimal_def) declare approx_refl [iff] +lemma hypreal_minus_distrib1: "-(y + -(x::hypreal)) = x + -y" +by (simp add: hypreal_add_commute) + lemma approx_sym: "x @= y ==> y @= x" apply (simp add: approx_def) apply (rule hypreal_minus_distrib1 [THEN subst]) @@ -562,7 +562,6 @@ val InfinitesimalD = thm "InfinitesimalD"; val Infinitesimal_zero = thm "Infinitesimal_zero"; val hypreal_sum_of_halves = thm "hypreal_sum_of_halves"; -val hypreal_half_gt_zero = thm "hypreal_half_gt_zero"; val Infinitesimal_add = thm "Infinitesimal_add"; val Infinitesimal_minus_iff = thm "Infinitesimal_minus_iff"; val Infinitesimal_diff = thm "Infinitesimal_diff";