automatic classical rule to derive a dvd b from b mod a = 0
authorhaftmann
Tue, 22 May 2018 18:14:29 +0000
changeset 68252 8b284d24f434
parent 68251 54a127873735
child 68253 a8660a39e304
automatic classical rule to derive a dvd b from b mod a = 0
src/HOL/Rings.thy
--- a/src/HOL/Rings.thy	Tue May 22 18:14:29 2018 +0000
+++ b/src/HOL/Rings.thy	Tue May 22 18:14:29 2018 +0000
@@ -1712,7 +1712,7 @@
   "b mod a = 0" if "a dvd b"
   using that minus_div_mult_eq_mod [of b a] by simp
 
-lemma mod_0_imp_dvd: 
+lemma mod_0_imp_dvd [dest!]: 
   "b dvd a" if "a mod b = 0"
 proof -
   have "b dvd (a div b) * b" by simp