| changeset 36977 | 71c8973a604b |
| parent 36635 | 080b755377c0 |
| child 39198 | f967a16dfcdd |
--- a/src/HOL/Big_Operators.thy Mon May 17 18:51:25 2010 -0700 +++ b/src/HOL/Big_Operators.thy Mon May 17 18:59:59 2010 -0700 @@ -673,7 +673,7 @@ proof induct case empty thus ?case by simp next - case (insert x A) thus ?case by (auto simp: add_nonneg_nonneg) + case (insert x A) thus ?case by auto qed next case False thus ?thesis by (simp add: setsum_def)