src/HOL/Hyperreal/Integration.thy
changeset 25112 98824cc791c0
parent 24742 73b8b42a36b6
child 25134 3d4953e88449
--- a/src/HOL/Hyperreal/Integration.thy	Sat Oct 20 12:09:30 2007 +0200
+++ b/src/HOL/Hyperreal/Integration.thy	Sat Oct 20 12:09:33 2007 +0200
@@ -149,12 +149,13 @@
 apply (rule_tac t = a in partition_lhs [THEN subst], assumption)
 apply (cut_tac x = "Suc n" and y = "psize D" in linorder_le_less_linear)
 apply (frule partition [THEN iffD1], safe)
+using neq0_conv
  apply (blast intro: partition_lt less_le_trans)
 apply (rotate_tac 3)
 apply (drule_tac x = "Suc n" in spec)
 apply (erule impE)
 apply (erule less_imp_le)
-apply (frule partition_rhs)
+apply (frule partition_rhs, simp only: neq0_conv)
 apply (drule partition_gt, assumption)
 apply (simp (no_asm_simp))
 done