# HG changeset patch # User haftmann # Date 1181064189 -7200 # Node ID 0c227412b285fef46cd553334ae24d7512887e1f # Parent 0fafccb015e641be1e45878cf4f89f92fe41d0f0 tuned boostrap diff -r 0fafccb015e6 -r 0c227412b285 src/HOL/HOL.thy --- a/src/HOL/HOL.thy Tue Jun 05 19:22:01 2007 +0200 +++ b/src/HOL/HOL.thy Tue Jun 05 19:23:09 2007 +0200 @@ -10,31 +10,22 @@ uses "~~/src/Tools/integer.ML" "hologic.ML" - "~~/src/Provers/splitter.ML" - "~~/src/Provers/hypsubst.ML" "~~/src/Tools/IsaPlanner/zipper.ML" "~~/src/Tools/IsaPlanner/isand.ML" "~~/src/Tools/IsaPlanner/rw_tools.ML" "~~/src/Tools/IsaPlanner/rw_inst.ML" - "~~/src/Provers/eqsubst.ML" + "~~/src/Provers/project_rule.ML" "~~/src/Provers/induct_method.ML" + "~~/src/Provers/hypsubst.ML" + "~~/src/Provers/splitter.ML" "~~/src/Provers/classical.ML" "~~/src/Provers/blast.ML" "~~/src/Provers/clasimp.ML" - "~~/src/Tools/rat.ML" - "~~/src/Provers/Arith/fast_lin_arith.ML" - "~~/src/Provers/Arith/cancel_sums.ML" + "~~/src/Provers/eqsubst.ML" "~~/src/Provers/quantifier1.ML" - "~~/src/Provers/project_rule.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" - "~~/src/Provers/quasi.ML" - "~~/src/Provers/order.ML" ("simpdata.ML") + "Tools/res_atpset.ML" ("~~/src/HOL/Tools/recfun_codegen.ML") - "Tools/res_atpset.ML" begin subsection {* Primitive logic *} diff -r 0fafccb015e6 -r 0c227412b285 src/HOL/IntArith.thy --- a/src/HOL/IntArith.thy Tue Jun 05 19:22:01 2007 +0200 +++ b/src/HOL/IntArith.thy Tue Jun 05 19:23:09 2007 +0200 @@ -7,7 +7,11 @@ theory IntArith imports Numeral Wellfounded_Relations -uses "~~/src/Provers/Arith/assoc_fold.ML" ("int_arith1.ML") +uses + "~~/src/Provers/Arith/assoc_fold.ML" + "~~/src/Provers/Arith/cancel_numerals.ML" + "~~/src/Provers/Arith/combine_numerals.ML" + ("int_arith1.ML") begin text{*Duplicate: can't understand why it's necessary*} diff -r 0fafccb015e6 -r 0c227412b285 src/HOL/Nat.thy --- a/src/HOL/Nat.thy Tue Jun 05 19:22:01 2007 +0200 +++ b/src/HOL/Nat.thy Tue Jun 05 19:23:09 2007 +0200 @@ -10,7 +10,11 @@ theory Nat imports Wellfounded_Recursion Ring_and_Field -uses ("arith_data.ML") +uses + "~~/src/Tools/rat.ML" + "~~/src/Provers/Arith/fast_lin_arith.ML" + "~~/src/Provers/Arith/cancel_sums.ML" + ("arith_data.ML") begin subsection {* Type @{text ind} *} diff -r 0fafccb015e6 -r 0c227412b285 src/HOL/NatSimprocs.thy --- a/src/HOL/NatSimprocs.thy Tue Jun 05 19:22:01 2007 +0200 +++ b/src/HOL/NatSimprocs.thy Tue Jun 05 19:23:09 2007 +0200 @@ -7,7 +7,11 @@ theory NatSimprocs imports Groebner_Basis -uses "int_factor_simprocs.ML" "nat_simprocs.ML" +uses + "~~/src/Provers/Arith/cancel_numeral_factor.ML" + "~~/src/Provers/Arith/extract_common_term.ML" + "int_factor_simprocs.ML" + "nat_simprocs.ML" begin setup nat_simprocs_setup diff -r 0fafccb015e6 -r 0c227412b285 src/HOL/Orderings.thy --- a/src/HOL/Orderings.thy Tue Jun 05 19:22:01 2007 +0200 +++ b/src/HOL/Orderings.thy Tue Jun 05 19:23:09 2007 +0200 @@ -7,6 +7,9 @@ theory Orderings imports HOL +uses + (*"~~/src/Provers/quasi.ML"*) + "~~/src/Provers/order.ML" begin subsection {* Order syntax *}