changeset 36350 | bc7982c54e37 |
parent 35416 | d8d7d1b785af |
child 41541 | 1fa4725c4656 |
--- a/src/HOL/Number_Theory/Residues.thy Mon Apr 26 11:34:17 2010 +0200 +++ b/src/HOL/Number_Theory/Residues.thy Mon Apr 26 11:34:19 2010 +0200 @@ -69,7 +69,7 @@ apply (subst mod_add_eq [symmetric]) apply (subst mult_commute) apply (subst zmod_zmult1_eq [symmetric]) - apply (simp add: ring_simps) + apply (simp add: field_simps) done end