src/HOL/Old_Number_Theory/Quadratic_Reciprocity.thy
changeset 44890 22f665a2e91c
parent 44766 d4d33a4d7548
child 45627 a0336f8b6558
--- a/src/HOL/Old_Number_Theory/Quadratic_Reciprocity.thy	Sun Sep 11 22:56:05 2011 +0200
+++ b/src/HOL/Old_Number_Theory/Quadratic_Reciprocity.thy	Mon Sep 12 07:55:43 2011 +0200
@@ -527,7 +527,7 @@
   ultimately have "int(card (S1)) = setsum (%j. int(card (f1 j))) P_set"
     by auto
   also have "... = setsum (%j. q * j div p) P_set"
-    using aux3a by(fastsimp intro: setsum_cong)
+    using aux3a by(fastforce intro: setsum_cong)
   finally show ?thesis .
 qed
 
@@ -551,7 +551,7 @@
   ultimately have "int(card (S2)) = setsum (%j. int(card (f2 j))) Q_set"
     by auto
   also have "... = setsum (%j. p * j div q) Q_set"
-    using aux3b by(fastsimp intro: setsum_cong)
+    using aux3b by(fastforce intro: setsum_cong)
   finally show ?thesis .
 qed