src/HOL/Groups_Big.thy
changeset 62378 85ed00c1fe7c
parent 62377 ace69956d018
child 62481 b5d8e57826df
--- a/src/HOL/Groups_Big.thy	Fri Feb 12 16:09:07 2016 +0100
+++ b/src/HOL/Groups_Big.thy	Fri Feb 19 13:40:50 2016 +0100
@@ -1195,6 +1195,6 @@
 
 lemma setprod_pos_nat_iff [simp]:
   "finite A \<Longrightarrow> setprod f A > 0 \<longleftrightarrow> (\<forall>a\<in>A. f a > (0::nat))"
-  using setprod_zero_iff by (simp del:neq0_conv add:neq0_conv [symmetric])
+  using setprod_zero_iff by (simp del: neq0_conv add: zero_less_iff_neq_zero)
 
 end