src/HOL/Rings.thy
changeset 63359 99b51ba8da1c
parent 63325 1086d56cde86
child 63456 3365c8ec67bd
--- a/src/HOL/Rings.thy	Fri Jul 01 08:19:53 2016 +0200
+++ b/src/HOL/Rings.thy	Fri Jul 01 08:35:15 2016 +0200
@@ -757,6 +757,17 @@
   finally show ?thesis .
 qed
 
+lemma dvd_mult_imp_div:
+  assumes "a * c dvd b"
+  shows "a dvd b div c"
+proof (cases "c = 0")
+  case True then show ?thesis by simp
+next
+  case False
+  from \<open>a * c dvd b\<close> obtain d where "b = a * c * d" ..
+  with False show ?thesis by (simp add: mult.commute [of a] mult.assoc)
+qed
+
 
 text \<open>Units: invertible elements in a ring\<close>