Fixed splitting of div and mod on integers (split theorem differed from implementation).
authorwebertj
Tue, 17 Nov 2009 11:10:22 +0000
changeset 33730 1755ca4ec022
parent 33729 3101453e0b1c
child 33736 ac81358132fd
Fixed splitting of div and mod on integers (split theorem differed from implementation).
src/HOL/Divides.thy
--- a/src/HOL/Divides.thy	Tue Nov 17 10:18:51 2009 +0000
+++ b/src/HOL/Divides.thy	Tue Nov 17 11:10:22 2009 +0000
@@ -2030,9 +2030,9 @@
                       split_neg_lemma [of concl: "%x y. P y"])
 done
 
-(* Enable arith to deal with @{term div} and @{term mod} when
-   these are applied to some constant that is of the form
-   @{term "number_of k"}: *)
+text {* Enable (lin)arith to deal with @{const div} and @{const mod}
+  when these are applied to some constant that is of the form
+  @{term "number_of k"}: *}
 declare split_zdiv [of _ _ "number_of k", standard, arith_split]
 declare split_zmod [of _ _ "number_of k", standard, arith_split]