| changeset 51173 | 3cbb4e95a565 |
| parent 50422 | ee729dbd1b7f |
| child 51299 | 30b014246e21 |
--- a/src/HOL/Divides.thy Sun Feb 17 20:45:49 2013 +0100 +++ b/src/HOL/Divides.thy Sun Feb 17 21:29:30 2013 +0100 @@ -740,6 +740,10 @@ shows "m mod n < (n::nat)" using assms divmod_nat_rel [of m n] unfolding divmod_nat_rel_def by auto +lemma mod_Suc_le_divisor [simp]: + "m mod Suc n \<le> n" + using mod_less_divisor [of "Suc n" m] by arith + lemma mod_less_eq_dividend [simp]: fixes m n :: nat shows "m mod n \<le> m"