add lemmas InfinitesimalI2, InfinitesimalD2
authorhuffman
Wed, 27 Sep 2006 23:53:46 +0200
changeset 20749 f7f2d03fe6f9
parent 20748 4bcf492c6c9d
child 20750 8bd4e37ff05c
add lemmas InfinitesimalI2, InfinitesimalD2
src/HOL/Hyperreal/NSA.thy
--- a/src/HOL/Hyperreal/NSA.thy	Wed Sep 27 23:41:12 2006 +0200
+++ b/src/HOL/Hyperreal/NSA.thy	Wed Sep 27 23:53:46 2006 +0200
@@ -345,6 +345,14 @@
       "x \<in> Infinitesimal ==> \<forall>r \<in> Reals. 0 < r --> hnorm x < r"
 by (simp add: Infinitesimal_def)
 
+lemma InfinitesimalI2:
+  "(\<And>r. 0 < r \<Longrightarrow> hnorm x < star_of r) \<Longrightarrow> x \<in> Infinitesimal"
+by (auto simp add: Infinitesimal_def SReal_def)
+
+lemma InfinitesimalD2:
+  "\<lbrakk>x \<in> Infinitesimal; 0 < r\<rbrakk> \<Longrightarrow> hnorm x < star_of r"
+by (auto simp add: Infinitesimal_def SReal_def)
+
 lemma Infinitesimal_zero [iff]: "0 \<in> Infinitesimal"
 by (simp add: Infinitesimal_def)