src/HOL/NSA/NSA.thy
changeset 34146 14595e0c27e8
parent 32960 69916a850301
child 34974 18b41bba42b5
--- a/src/HOL/NSA/NSA.thy	Fri Dec 18 18:48:27 2009 -0800
+++ b/src/HOL/NSA/NSA.thy	Fri Dec 18 19:00:11 2009 -0800
@@ -1711,7 +1711,7 @@
 lemma Infinitesimal_add_not_zero:
      "[| h \<in> Infinitesimal; x \<noteq> 0 |] ==> star_of x + h \<noteq> 0"
 apply auto
-apply (subgoal_tac "h = - star_of x", auto intro: equals_zero_I [symmetric])
+apply (subgoal_tac "h = - star_of x", auto intro: minus_unique [symmetric])
 done
 
 lemma Infinitesimal_square_cancel [simp]: