Mon, 25 Oct 2010 13:34:57 +0200 haftmann moved sledgehammer to Plain; tuned dependencies
Mon, 25 Oct 2010 13:34:57 +0200 haftmann CONTRIBUTORS
Mon, 25 Oct 2010 12:24:38 +0200 blanchet merge
Mon, 25 Oct 2010 11:42:05 +0200 blanchet merged
Mon, 25 Oct 2010 10:38:41 +0200 blanchet updated keywords
Mon, 25 Oct 2010 10:30:46 +0200 blanchet introduced manual version of "Auto Solve" as "solve_direct"
Mon, 25 Oct 2010 09:29:43 +0200 blanchet make "sledgehammer_params" work on single-threaded platforms
Fri, 22 Oct 2010 18:31:45 +0200 blanchet tuning
Fri, 22 Oct 2010 18:24:10 +0200 blanchet handle timeouts (to prevent failure from other threads);
Mon, 25 Oct 2010 12:11:12 +0200 haftmann update keywords
Mon, 25 Oct 2010 10:45:22 +0200 krauss some partial_function examples
Mon, 25 Oct 2010 11:16:23 +0200 wenzelm added ML antiquotation @{assert};
Mon, 25 Oct 2010 11:01:00 +0200 wenzelm updated keywords;
Sat, 23 Oct 2010 23:42:04 +0200 krauss integrated partial_function into HOL-Plain
Sat, 23 Oct 2010 23:41:19 +0200 krauss first version of partial_function package
Sat, 23 Oct 2010 23:39:37 +0200 krauss Complete_Partial_Order.thy: complete partial orders over arbitrary chains, with fixpoint theorem
Mon, 25 Oct 2010 08:08:08 +0200 bulwahn merged
Fri, 22 Oct 2010 18:38:59 +0200 bulwahn splitting Hotel Key card example into specification and the two tests for counter example generation
Fri, 22 Oct 2010 18:38:59 +0200 bulwahn adding generator quickcheck
Fri, 22 Oct 2010 18:38:59 +0200 bulwahn restructuring values command and adding generator compilation
Fri, 22 Oct 2010 18:38:59 +0200 bulwahn moving general functions from core_data to predicate_compile_aux
Fri, 22 Oct 2010 18:38:59 +0200 bulwahn updating to new notation in commented examples
Sun, 24 Oct 2010 15:11:24 -0700 huffman merged
Sun, 24 Oct 2010 03:43:12 -0700 huffman use default names sprod/Rep_sprod/Abs_sprod from pcpodef instead of Sprod/Rep_Sprod/Abs_Sprod; similarly for ssum
Sat, 23 Oct 2010 19:56:33 -0700 huffman remove legacy comp_dbind option from domain package
Sat, 23 Oct 2010 11:04:26 -0700 huffman change fixrec parser to not accept theorem names with (unchecked) option
Sat, 23 Oct 2010 11:03:50 -0700 huffman tuned
Fri, 22 Oct 2010 15:49:18 -0700 huffman rename lemma surjective_pairing_Sprod2 to spair_sfst_ssnd
Fri, 22 Oct 2010 15:47:43 -0700 huffman add lemma strict3
Fri, 22 Oct 2010 11:24:52 -0700 huffman do proofs using Rep_Sprod_simps, Rep_Ssum_simps; remove unused lemmas
Fri, 22 Oct 2010 07:45:32 -0700 huffman make discrete_cpo a subclass of chfin; remove chfin instances for fun, cfun
Fri, 22 Oct 2010 07:44:34 -0700 huffman direct instantiation unit :: discrete_cpo
Fri, 22 Oct 2010 06:58:45 -0700 huffman remove finite_po class
Fri, 22 Oct 2010 06:08:51 -0700 huffman simplify proofs about flift; remove unneeded lemmas
Fri, 22 Oct 2010 05:54:54 -0700 huffman simplify proof
Thu, 21 Oct 2010 15:21:39 -0700 huffman minimize imports
Thu, 21 Oct 2010 15:19:07 -0700 huffman add type annotation to avoid warning
Thu, 21 Oct 2010 12:51:36 -0700 huffman simplify some proofs, convert to Isar style
Thu, 21 Oct 2010 12:03:49 -0700 huffman rename lemma spair_lemma to spair_Sprod
Thu, 21 Oct 2010 06:03:18 -0700 huffman pcpodef (open) 'a lift
Thu, 21 Oct 2010 05:44:38 -0700 huffman remove intro! attribute from {sinl,sinr}_defined
Thu, 21 Oct 2010 05:35:32 -0700 huffman simplify proofs of ssumE, sprodE
Sun, 24 Oct 2010 21:25:13 +0200 wenzelm merged
Sun, 24 Oct 2010 20:37:30 +0200 nipkow renamed nat_number
Sun, 24 Oct 2010 20:19:00 +0200 nipkow nat_number -> eval_nat_numeral
Fri, 22 Oct 2010 23:45:20 +0200 krauss some cleanup in Function_Lib
Fri, 22 Oct 2010 17:15:46 +0200 blanchet merged
Fri, 22 Oct 2010 16:45:55 +0200 blanchet compile
Fri, 22 Oct 2010 16:37:11 +0200 blanchet added SMT solver to Sledgehammer docs
Fri, 22 Oct 2010 16:11:43 +0200 blanchet more robust handling of "remote_" vs. non-"remote_" provers
Fri, 22 Oct 2010 15:02:27 +0200 blanchet generalized the relevance filter so that it takes the list of "irrelevant constants" as argument (since the ATP and SMT preprocessing are different)
Fri, 22 Oct 2010 14:47:43 +0200 blanchet replaced references with proper record that's threaded through
Fri, 22 Oct 2010 14:10:32 +0200 blanchet fixed signature of "is_smt_solver_installed";
Fri, 22 Oct 2010 13:57:54 +0200 blanchet renamed modules
Fri, 22 Oct 2010 13:54:51 +0200 blanchet renamed files
Fri, 22 Oct 2010 13:49:44 +0200 blanchet took out "smt"/"remote_smt" from default ATPs until they are properly implemented
Fri, 22 Oct 2010 13:48:21 +0200 blanchet remove more needless code ("run_smt_solvers");
Fri, 22 Oct 2010 12:15:31 +0200 blanchet got rid of duplicate functionality ("run_smt_solver_somehow");
Fri, 22 Oct 2010 11:58:33 +0200 blanchet bring ATPs and SMT solvers more in line with each other
Fri, 22 Oct 2010 11:11:34 +0200 blanchet make Sledgehammer minimizer fully work with SMT
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip