doc-src/TutorialI/Rules/Force.thy
changeset 11407 138919f1a135
parent 10341 6eb91805a012
child 11456 7eb63f63e6c6
--- a/doc-src/TutorialI/Rules/Force.thy	Wed Jul 11 13:57:01 2001 +0200
+++ b/doc-src/TutorialI/Rules/Force.thy	Wed Jul 11 14:00:48 2001 +0200
@@ -1,6 +1,14 @@
 (* ID:         $Id$ *)
-theory Force = Main:
+theory Force = Divides: (*Divides rather than Main so that the first proof
+                         isn't done by the nat_divide_cancel_factor simprocs.*)
+
+declare div_mult_self_is_m [simp del];
 
+lemma div_mult_self_is_m: 
+      "0<n \<Longrightarrow> (m*n) div n = (m::nat)"
+apply (insert mod_div_equality [of "m*n" n])
+apply simp
+done
 
 
 lemma "(\<forall>x. P x) \<and> (\<exists>x. Q x) \<longrightarrow> (\<forall>x. P x \<and> Q x)"