src/HOL/Divides.thy
changeset 29404 ee15ccdeaa72
parent 29403 fe17df4e4ab3
child 29405 98ab21b14f09
--- a/src/HOL/Divides.thy	Thu Jan 08 08:24:08 2009 -0800
+++ b/src/HOL/Divides.thy	Thu Jan 08 08:36:16 2009 -0800
@@ -248,6 +248,23 @@
     by (simp only: mod_mult_eq [symmetric])
 qed
 
+lemma mod_mod_cancel:
+  assumes "c dvd b"
+  shows "a mod b mod c = a mod c"
+proof -
+  from `c dvd b` obtain k where "b = c * k"
+    by (rule dvdE)
+  have "a mod b mod c = a mod (c * k) mod c"
+    by (simp only: `b = c * k`)
+  also have "\<dots> = (a mod (c * k) + a div (c * k) * k * c) mod c"
+    by (simp only: mod_mult_self1)
+  also have "\<dots> = (a div (c * k) * (c * k) + a mod (c * k)) mod c"
+    by (simp only: add_ac mult_ac)
+  also have "\<dots> = a mod c"
+    by (simp only: mod_div_equality)
+  finally show ?thesis .
+qed
+
 end