merged
authorhaftmann
Fri, 30 Oct 2009 18:33:21 +0100
changeset 33367 2912bf1871ba
parent 33363 1d11893b0d74 (current diff)
parent 33366 b0096ac3b731 (diff)
child 33368 b1cf34f1855c
merged
--- a/src/HOL/Divides.thy	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/HOL/Divides.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -131,7 +131,7 @@
   note that ultimately show thesis by blast
 qed
 
-lemma dvd_eq_mod_eq_0 [code_unfold]: "a dvd b \<longleftrightarrow> b mod a = 0"
+lemma dvd_eq_mod_eq_0 [code, code_unfold, code_inline del]: "a dvd b \<longleftrightarrow> b mod a = 0"
 proof
   assume "b mod a = 0"
   with mod_div_equality [of b a] have "b div a * a = b" by simp
@@ -2460,4 +2460,13 @@
   then show ?thesis by (simp add: divmod_int_pdivmod)
 qed
 
+code_modulename SML
+  Divides Arith
+
+code_modulename OCaml
+  Divides Arith
+
+code_modulename Haskell
+  Divides Arith
+
 end
--- a/src/HOL/HOL.thy	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/HOL/HOL.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -1818,7 +1818,7 @@
 
 code_datatype "TYPE('a\<Colon>{})"
 
-code_datatype Trueprop "prop"
+code_datatype "prop" Trueprop
 
 text {* Code equations *}
 
--- a/src/HOL/Int.thy	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/HOL/Int.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -2246,13 +2246,13 @@
   by simp
 
 code_modulename SML
-  Int Integer
+  Int Arith
 
 code_modulename OCaml
-  Int Integer
+  Int Arith
 
 code_modulename Haskell
-  Int Integer
+  Int Arith
 
 types_code
   "int" ("int")
--- a/src/HOL/Library/Efficient_Nat.thy	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/HOL/Library/Efficient_Nat.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -424,22 +424,13 @@
 text {* Module names *}
 
 code_modulename SML
-  Nat Integer
-  Divides Integer
-  Ring_and_Field Integer
-  Efficient_Nat Integer
+  Efficient_Nat Arith
 
 code_modulename OCaml
-  Nat Integer
-  Divides Integer
-  Ring_and_Field Integer
-  Efficient_Nat Integer
+  Efficient_Nat Arith
 
 code_modulename Haskell
-  Nat Integer
-  Divides Integer
-  Ring_and_Field Integer
-  Efficient_Nat Integer
+  Efficient_Nat Arith
 
 hide const int
 
--- a/src/HOL/Nat.thy	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/HOL/Nat.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -1674,4 +1674,16 @@
 class size =
   fixes size :: "'a \<Rightarrow> nat" -- {* see further theory @{text Wellfounded} *}
 
+
+subsection {* code module namespace *}
+
+code_modulename SML
+  Nat Arith
+
+code_modulename OCaml
+  Nat Arith
+
+code_modulename Haskell
+  Nat Arith
+
 end
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Numeral_Simprocs.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -0,0 +1,120 @@
+(* Author: Various *)
+
+header {* Combination and Cancellation Simprocs for Numeral Expressions *}
+
+theory Numeral_Simprocs
+imports Divides
+uses
+  "~~/src/Provers/Arith/assoc_fold.ML"
+  "~~/src/Provers/Arith/cancel_numerals.ML"
+  "~~/src/Provers/Arith/combine_numerals.ML"
+  "~~/src/Provers/Arith/cancel_numeral_factor.ML"
+  "~~/src/Provers/Arith/extract_common_term.ML"
+  ("Tools/numeral_simprocs.ML")
+  ("Tools/nat_numeral_simprocs.ML")
+begin
+
+declare split_div [of _ _ "number_of k", standard, arith_split]
+declare split_mod [of _ _ "number_of k", standard, arith_split]
+
+text {* For @{text combine_numerals} *}
+
+lemma left_add_mult_distrib: "i*u + (j*u + k) = (i+j)*u + (k::nat)"
+by (simp add: add_mult_distrib)
+
+text {* For @{text cancel_numerals} *}
+
+lemma nat_diff_add_eq1:
+     "j <= (i::nat) ==> ((i*u + m) - (j*u + n)) = (((i-j)*u + m) - n)"
+by (simp split add: nat_diff_split add: add_mult_distrib)
+
+lemma nat_diff_add_eq2:
+     "i <= (j::nat) ==> ((i*u + m) - (j*u + n)) = (m - ((j-i)*u + n))"
+by (simp split add: nat_diff_split add: add_mult_distrib)
+
+lemma nat_eq_add_iff1:
+     "j <= (i::nat) ==> (i*u + m = j*u + n) = ((i-j)*u + m = n)"
+by (auto split add: nat_diff_split simp add: add_mult_distrib)
+
+lemma nat_eq_add_iff2:
+     "i <= (j::nat) ==> (i*u + m = j*u + n) = (m = (j-i)*u + n)"
+by (auto split add: nat_diff_split simp add: add_mult_distrib)
+
+lemma nat_less_add_iff1:
+     "j <= (i::nat) ==> (i*u + m < j*u + n) = ((i-j)*u + m < n)"
+by (auto split add: nat_diff_split simp add: add_mult_distrib)
+
+lemma nat_less_add_iff2:
+     "i <= (j::nat) ==> (i*u + m < j*u + n) = (m < (j-i)*u + n)"
+by (auto split add: nat_diff_split simp add: add_mult_distrib)
+
+lemma nat_le_add_iff1:
+     "j <= (i::nat) ==> (i*u + m <= j*u + n) = ((i-j)*u + m <= n)"
+by (auto split add: nat_diff_split simp add: add_mult_distrib)
+
+lemma nat_le_add_iff2:
+     "i <= (j::nat) ==> (i*u + m <= j*u + n) = (m <= (j-i)*u + n)"
+by (auto split add: nat_diff_split simp add: add_mult_distrib)
+
+text {* For @{text cancel_numeral_factors} *}
+
+lemma nat_mult_le_cancel1: "(0::nat) < k ==> (k*m <= k*n) = (m<=n)"
+by auto
+
+lemma nat_mult_less_cancel1: "(0::nat) < k ==> (k*m < k*n) = (m<n)"
+by auto
+
+lemma nat_mult_eq_cancel1: "(0::nat) < k ==> (k*m = k*n) = (m=n)"
+by auto
+
+lemma nat_mult_div_cancel1: "(0::nat) < k ==> (k*m) div (k*n) = (m div n)"
+by auto
+
+lemma nat_mult_dvd_cancel_disj[simp]:
+  "(k*m) dvd (k*n) = (k=0 | m dvd (n::nat))"
+by(auto simp: dvd_eq_mod_eq_0 mod_mult_distrib2[symmetric])
+
+lemma nat_mult_dvd_cancel1: "0 < k \<Longrightarrow> (k*m) dvd (k*n::nat) = (m dvd n)"
+by(auto)
+
+text {* For @{text cancel_factor} *}
+
+lemma nat_mult_le_cancel_disj: "(k*m <= k*n) = ((0::nat) < k --> m<=n)"
+by auto
+
+lemma nat_mult_less_cancel_disj: "(k*m < k*n) = ((0::nat) < k & m<n)"
+by auto
+
+lemma nat_mult_eq_cancel_disj: "(k*m = k*n) = (k = (0::nat) | m=n)"
+by auto
+
+lemma nat_mult_div_cancel_disj[simp]:
+     "(k*m) div (k*n) = (if k = (0::nat) then 0 else m div n)"
+by (simp add: nat_mult_div_cancel1)
+
+
+use "Tools/numeral_simprocs.ML"
+
+use "Tools/nat_numeral_simprocs.ML"
+
+declaration {* 
+  K (Lin_Arith.add_simps (@{thms neg_simps} @ [@{thm Suc_nat_number_of}, @{thm int_nat_number_of}])
+  #> Lin_Arith.add_simps (@{thms ring_distribs} @ [@{thm Let_number_of}, @{thm Let_0}, @{thm Let_1},
+     @{thm nat_0}, @{thm nat_1},
+     @{thm add_nat_number_of}, @{thm diff_nat_number_of}, @{thm mult_nat_number_of},
+     @{thm eq_nat_number_of}, @{thm less_nat_number_of}, @{thm le_number_of_eq_not_less},
+     @{thm le_Suc_number_of}, @{thm le_number_of_Suc},
+     @{thm less_Suc_number_of}, @{thm less_number_of_Suc},
+     @{thm Suc_eq_number_of}, @{thm eq_number_of_Suc},
+     @{thm mult_Suc}, @{thm mult_Suc_right},
+     @{thm add_Suc}, @{thm add_Suc_right},
+     @{thm eq_number_of_0}, @{thm eq_0_number_of}, @{thm less_0_number_of},
+     @{thm of_int_number_of_eq}, @{thm of_nat_number_of_eq}, @{thm nat_number_of},
+     @{thm if_True}, @{thm if_False}])
+  #> Lin_Arith.add_simprocs (Numeral_Simprocs.assoc_fold_simproc
+      :: Numeral_Simprocs.combine_numerals
+      :: Numeral_Simprocs.cancel_numerals)
+  #> Lin_Arith.add_simprocs (Nat_Numeral_Simprocs.combine_numerals :: Nat_Numeral_Simprocs.cancel_numerals))
+*}
+
+end
\ No newline at end of file
--- a/src/HOL/OrderedGroup.thy	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/HOL/OrderedGroup.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -1409,4 +1409,13 @@
   Addsimprocs [ab_group_add_cancel.sum_conv, ab_group_add_cancel.rel_conv];
 *}
 
+code_modulename SML
+  OrderedGroup Arith
+
+code_modulename OCaml
+  OrderedGroup Arith
+
+code_modulename Haskell
+  OrderedGroup Arith
+
 end
--- a/src/HOL/Power.thy	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/HOL/Power.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -467,4 +467,13 @@
 
 declare power.power.simps [code]
 
+code_modulename SML
+  Power Arith
+
+code_modulename OCaml
+  Power Arith
+
+code_modulename Haskell
+  Power Arith
+
 end
--- a/src/HOL/Ring_and_Field.thy	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/HOL/Ring_and_Field.thy	Fri Oct 30 18:33:21 2009 +0100
@@ -2374,4 +2374,14 @@
   then show ?thesis by simp
 qed
 
+
+code_modulename SML
+  Ring_and_Field Arith
+
+code_modulename OCaml
+  Ring_and_Field Arith
+
+code_modulename Haskell
+  Ring_and_Field Arith
+
 end
--- a/src/Pure/pure_thy.ML	Fri Oct 30 14:52:14 2009 +0100
+++ b/src/Pure/pure_thy.ML	Fri Oct 30 18:33:21 2009 +0100
@@ -268,7 +268,8 @@
 (* main content *)
 
 val _ = Context.>> (Context.map_theory
-  (OldApplSyntax.init #>
+  (Sign.map_naming (Name_Space.set_theory_name Context.PureN) #>
+   OldApplSyntax.init #>
    Sign.add_types
    [(Binding.name "fun", 2, NoSyn),
     (Binding.name "prop", 0, NoSyn),