added setsum_pos_nat
authornipkow
Wed, 01 Apr 2009 16:55:31 +0200
changeset 30839 bf99ceb7d015
parent 30838 d09a0794d457
child 30840 98809b3f5e3c
child 30850 5e20f9c20086
added setsum_pos_nat
src/HOL/Int.thy
--- a/src/HOL/Int.thy	Wed Apr 01 16:03:18 2009 +0200
+++ b/src/HOL/Int.thy	Wed Apr 01 16:55:31 2009 +0200
@@ -1408,6 +1408,10 @@
     "finite A ==> (\<forall>x \<in> A. f x \<noteq> (0::nat)) ==> setprod f A \<noteq> 0"
   by (rule setprod_nonzero, auto)
 
+lemma setprod_pos_nat:
+  "finite S ==> (ALL x : S. f x > (0::nat)) ==> setprod f S > 0"
+using setprod_nonzero_nat by simp
+
 lemma setprod_zero_eq_nat:
     "finite A ==> (setprod f A = (0::nat)) = (\<exists>x \<in> A. f x = 0)"
   by (rule setprod_zero_eq, auto)