# HG changeset patch # User huffman # Date 1159394026 -7200 # Node ID f7f2d03fe6f9a1ed33f729562828a14cbc880921 # Parent 4bcf492c6c9dbb53648074eb5da165615b1f353f add lemmas InfinitesimalI2, InfinitesimalD2 diff -r 4bcf492c6c9d -r f7f2d03fe6f9 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 \ Infinitesimal ==> \r \ Reals. 0 < r --> hnorm x < r" by (simp add: Infinitesimal_def) +lemma InfinitesimalI2: + "(\r. 0 < r \ hnorm x < star_of r) \ x \ Infinitesimal" +by (auto simp add: Infinitesimal_def SReal_def) + +lemma InfinitesimalD2: + "\x \ Infinitesimal; 0 < r\ \ hnorm x < star_of r" +by (auto simp add: Infinitesimal_def SReal_def) + lemma Infinitesimal_zero [iff]: "0 \ Infinitesimal" by (simp add: Infinitesimal_def)