src/HOL/Integ/NatSimprocs.thy
changeset 17149 e2b19c92ef51
parent 17085 5b57f995a179
child 17472 bcbf48d59059
--- a/src/HOL/Integ/NatSimprocs.thy	Fri Aug 26 08:42:52 2005 +0200
+++ b/src/HOL/Integ/NatSimprocs.thy	Fri Aug 26 10:01:06 2005 +0200
@@ -362,6 +362,13 @@
 
 lemmas half_gt_zero = half_gt_zero_iff [THEN iffD2, simp]
 
+(* The following lemma should appear in Divides.thy, but there the proof
+   doesn't work. *)
+
+lemma nat_dvd_not_less:
+  "[| 0 < m; m < n |] ==> \<not> n dvd (m::nat)"
+  by (unfold dvd_def) auto
+
 ML
 {*
 val divide_minus1 = thm "divide_minus1";