adapted to new times_divide_eq simp situation
authorhaftmann
Fri, 23 Apr 2010 16:17:25 +0200
changeset 36310 e3d3b14b13cd
parent 36309 4da07afb065b
child 36311 ed3a87a7f977
adapted to new times_divide_eq simp situation
src/HOL/NSA/HDeriv.thy
--- a/src/HOL/NSA/HDeriv.thy	Fri Apr 23 16:17:25 2010 +0200
+++ b/src/HOL/NSA/HDeriv.thy	Fri Apr 23 16:17:25 2010 +0200
@@ -204,7 +204,7 @@
 apply (simp (no_asm) add: add_divide_distrib diff_divide_distrib)
 apply (drule bex_Infinitesimal_iff2 [THEN iffD2])+
 apply (auto simp add: times_divide_eq_right [symmetric]
-            simp del: times_divide_eq)
+            simp del: times_divide_eq_right times_divide_eq_left)
 apply (drule_tac D = Db in lemma_nsderiv2, assumption+)
 apply (drule_tac
      approx_minus_iff [THEN iffD2, THEN bex_Infinitesimal_iff2 [THEN iffD2]])