src/HOL/NumberTheory/Gauss.thy
changeset 16733 236dfafbeb63
parent 16663 13e9c402308b
child 16775 c1b87ef4a1c3
--- a/src/HOL/NumberTheory/Gauss.thy	Thu Jul 07 12:36:56 2005 +0200
+++ b/src/HOL/NumberTheory/Gauss.thy	Thu Jul 07 12:39:17 2005 +0200
@@ -459,8 +459,7 @@
       by (simp add: B_def)
     then have "[setprod id A = ((-1)^(card E) * (setprod (%x. x * a) A))] 
         (mod p)"
-      apply (rule zcong_trans)
-      by (simp add: finite_A inj_on_xa_A setprod_reindex_id zcong_scalar2)
+      by(simp add:finite_A inj_on_xa_A setprod_reindex_id[symmetric])
     moreover have "setprod (%x. x * a) A = 
         setprod (%x. a) A * setprod id A"
       by (insert finite_A, induct set: Finites, auto)