src/HOL/Hyperreal/NatStar.ML
changeset 14268 5cf13e80be0e
parent 13810 c3fbfd472365
child 14371 c78c7da09519
--- a/src/HOL/Hyperreal/NatStar.ML	Tue Nov 25 10:37:03 2003 +0100
+++ b/src/HOL/Hyperreal/NatStar.ML	Thu Nov 27 10:47:55 2003 +0100
@@ -479,3 +479,15 @@
 by (dres_inst_tac [("x","hypnat_of_nat(x)")] fun_cong 1);
 by (auto_tac (claset(), simpset() addsimps [starfunNat,hypnat_of_nat_def]));
 qed "starfun_eq_iff";
+
+
+
+(*MOVE UP*)
+
+Goal "N : HNatInfinite \
+\     ==> ( *fNat* (%x. inverse (real x))) N : Infinitesimal";
+by (res_inst_tac [("f1","inverse")]  (starfun_stafunNat_o2 RS subst) 1);
+by (subgoal_tac "hypreal_of_hypnat N ~= 0" 1);
+by (auto_tac (claset(),simpset() addsimps [starfunNat_real_of_nat]));
+qed "starfunNat_inverse_real_of_nat_Infinitesimal";
+Addsimps [starfunNat_inverse_real_of_nat_Infinitesimal];