src/HOL/Nonstandard_Analysis/NatStar.thy
changeset 67091 1393c2340eec
parent 64435 c93b0e6131c3
child 67399 eab6ce8368fa
--- a/src/HOL/Nonstandard_Analysis/NatStar.thy	Sun Nov 26 13:19:52 2017 +0100
+++ b/src/HOL/Nonstandard_Analysis/NatStar.thy	Sun Nov 26 21:08:32 2017 +0100
@@ -143,9 +143,9 @@
   by transfer (rule refl)
 
 lemma starfunNat_inverse_real_of_nat_Infinitesimal [simp]:
-  "N \<in> HNatInfinite \<Longrightarrow> ( *f* (%x. inverse (real x))) N \<in> Infinitesimal"
+  "N \<in> HNatInfinite \<Longrightarrow> ( *f* (\<lambda>x. inverse (real x))) N \<in> Infinitesimal"
   apply (rule_tac f1 = inverse in starfun_o2 [THEN subst])
-  apply (subgoal_tac "hypreal_of_hypnat N ~= 0")
+  apply (subgoal_tac "hypreal_of_hypnat N \<noteq> 0")
    apply (simp_all add: zero_less_HNatInfinite starfunNat_real_of_nat)
   done