src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
Fri, 31 Jan 2014 18:43:16 +0100 blanchet moved code around
Fri, 31 Jan 2014 18:43:16 +0100 blanchet added 'algebra' to the mix
Fri, 31 Jan 2014 18:43:16 +0100 blanchet more informative trace
Fri, 31 Jan 2014 16:41:54 +0100 blanchet better tracing + syntactically correct 'metis' calls
Fri, 31 Jan 2014 16:26:43 +0100 blanchet tuned ML function names
Fri, 31 Jan 2014 16:10:39 +0100 blanchet tuning
Fri, 31 Jan 2014 16:07:20 +0100 blanchet moved ML code around
Fri, 31 Jan 2014 10:23:32 +0100 blanchet renamed many Sledgehammer ML files to clarify structure
Thu, 30 Jan 2014 14:37:53 +0100 blanchet renamed Sledgehammer options for symmetry between positive and negative versions
Thu, 19 Dec 2013 13:43:21 +0100 blanchet made timeouts in Sledgehammer not be 'option's -- simplified lots of code
Thu, 21 Nov 2013 12:29:29 +0100 blanchet fixed spying so that the envirnoment variables are queried at run-time not at build-time
Tue, 19 Nov 2013 18:34:04 +0100 blanchet tuning
Thu, 17 Oct 2013 01:34:34 +0200 blanchet added comment
Tue, 15 Oct 2013 15:31:18 +0200 blanchet use MePo with Auto Sledgehammer, because it's lighter than MaSh and always available
Fri, 04 Oct 2013 11:52:10 +0200 blanchet run fewer provers in "try" mode
Fri, 04 Oct 2013 11:28:28 +0200 blanchet count remote threads as well when balancing CPU usage -- otherwise jEdit users and other users of the "blocking" mode may have to wait for 2 * timeout if they e.g. have 4 cores and 5 provers (the typical situation)
Mon, 23 Sep 2013 14:53:43 +0200 blanchet added "spy" option to Sledgehammer
Fri, 20 Sep 2013 22:39:30 +0200 blanchet merged "isar_try0" and "isar_minimize" options
Fri, 20 Sep 2013 22:39:30 +0200 blanchet hardcoded obscure option
Fri, 20 Sep 2013 22:39:30 +0200 blanchet hard-coded an obscure option
Fri, 20 Sep 2013 22:39:30 +0200 blanchet use configuration mechanism for low-level tracing
Fri, 20 Sep 2013 22:39:30 +0200 blanchet took out Waldmeister from list of default provers -- it's usually just visual noise, and its integration in Sledgehammer leaves much to be desired
Fri, 20 Sep 2013 22:39:30 +0200 blanchet tuning (use a blacklist instead of a whitelist)
Thu, 22 Aug 2013 23:03:21 +0200 blanchet fixed subtle bug with "take" + thread overlord through
Thu, 22 Aug 2013 16:03:13 +0200 blanchet have kill_all also kill MaSh server + be paranoid about reloading after clear_state, to allow for easier experimentation
Sat, 17 Aug 2013 22:45:48 +0200 wenzelm prefer system option sledgehammer_timeout, with standard GUI in jEdit Plugin Options;
Sat, 17 Aug 2013 22:15:45 +0200 wenzelm some protocol to determine provers according to ML;
Sat, 17 Aug 2013 19:54:16 +0200 wenzelm always enable "minimize" to simplify interaction model;
Sat, 17 Aug 2013 19:13:28 +0200 wenzelm sledgehammer sendback always uses Markup.padding_command: sensible default for most practical applications -- old-style in-line replacement is superseded by auto mode or panel;
Sat, 17 Aug 2013 12:21:25 +0200 wenzelm eliminated pointless subgoal argument;
Sat, 17 Aug 2013 12:13:53 +0200 wenzelm more direct sledgehammer configuration via mode = Normal_Result and output_result;
Mon, 12 Aug 2013 17:57:51 +0200 wenzelm clarified Query_Operation.register: avoid hard-wired parallel policy;
Thu, 08 Aug 2013 14:24:21 +0200 wenzelm dockable window for Sledgehammer, based on asynchronous/parallel query operation;
Sat, 13 Jul 2013 21:02:41 +0200 wenzelm merged
Sat, 13 Jul 2013 00:50:49 +0200 wenzelm hybrid "auto" tool setup, for TTY (within theory) and PIDE (global print function);
Fri, 12 Jul 2013 23:45:05 +0200 wenzelm system options for Isabelle/HOL proof tools;
Fri, 12 Jul 2013 22:41:25 +0200 smolkas added sledgehammer parameters isar_try0 and isar_minimize and their negative aliases
Tue, 09 Jul 2013 18:45:06 +0200 smolkas completely rewrote SH compress; added two parameters for experimentation/fine grained control
Tue, 11 Jun 2013 16:13:19 -0400 smolkas make use of show_type_emphasis instead of using hack; make sure global configurations don't affect proof script creation
Tue, 21 May 2013 09:02:58 +0200 blanchet added compatibility alias
Thu, 16 May 2013 13:34:13 +0200 blanchet tuning -- renamed '_from_' to '_of_' in Sledgehammer
Wed, 15 May 2013 23:00:17 +0200 wenzelm merged;
Wed, 15 May 2013 22:30:24 +0200 wenzelm clarified preferences: "override" re-initialized on prover startup, and "default" sent to PG -- thus recover typical defaults like auto-quickcheck in PG 4.x;
Wed, 15 May 2013 20:22:46 +0200 wenzelm maintain ProofGeneral preferences within ProofGeneral module;
Wed, 15 May 2013 17:39:41 +0200 wenzelm just one ProofGeneral module;
Wed, 15 May 2013 17:43:42 +0200 blanchet renamed Sledgehammer functions with 'for' in their names to 'of'
Mon, 06 May 2013 11:03:08 +0200 smolkas added preplay tracing
Wed, 27 Mar 2013 17:58:07 +0100 wenzelm more robust access Toplevel.proof_of -- prefer warning via Toplevel.unknown_proof over hard crash (notably for skipped proofs);
Wed, 20 Feb 2013 14:10:51 +0100 blanchet minimize SMT proofs with E if Isar proofs are desired and Metis managed to preplay
Wed, 20 Feb 2013 09:58:28 +0100 blanchet fixed typo in option name
Wed, 20 Feb 2013 08:44:24 +0100 blanchet made "isar_proofs" a 3-way option, to provide a way to totally disable isar_proofs if desired
Wed, 20 Feb 2013 08:44:24 +0100 blanchet alias for people like me
Fri, 15 Feb 2013 09:17:26 +0100 blanchet killed legacy alias
Thu, 14 Feb 2013 22:49:22 +0100 smolkas renamed sledgehammer_shrink to sledgehammer_compress
Fri, 11 Jan 2013 14:35:28 +0100 smolkas tuned
Fri, 11 Jan 2013 13:57:51 +0100 smolkas set show_markup to false in order to avoid problems in jedit
Sat, 05 Jan 2013 22:31:30 +0100 blanchet nicer output
Sat, 05 Jan 2013 22:31:30 +0100 blanchet pass option to minimize
Fri, 04 Jan 2013 19:00:49 +0100 blanchet renamed "kill" subcommand to avoid clash with "kill" keyword (which confuses Proof General and results in strange syntax highlighting)
Wed, 19 Dec 2012 22:43:07 +0100 blanchet crank up default timeout for MaSh ATP learning
Sat, 15 Dec 2012 19:57:12 +0100 blanchet thread no timeout properly
Wed, 12 Dec 2012 00:24:06 +0100 blanchet adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)
Mon, 12 Nov 2012 14:11:51 +0100 blanchet create temp directory if not already created
Tue, 06 Nov 2012 15:15:33 +0100 blanchet renamed Sledgehammer option
Thu, 18 Oct 2012 15:05:17 +0200 blanchet renamed Isar-proof related options + changed semantics of Isar shrinking
Fri, 28 Sep 2012 09:12:50 +0200 blanchet tuned message
Fri, 14 Sep 2012 12:09:27 +0200 blanchet merged two commands
Thu, 26 Jul 2012 11:07:27 +0200 blanchet detect unknown options again
Mon, 23 Jul 2012 15:32:30 +0200 blanchet don't relearn old facts in Isar mode
Mon, 23 Jul 2012 15:32:30 +0200 blanchet took out CVC3 again -- there seems to be issues with the server version of CVC3 + minor tweaks
Fri, 20 Jul 2012 22:19:46 +0200 blanchet honor suggested MaSh weights
Fri, 20 Jul 2012 22:19:46 +0200 blanchet use CVC3 and Yices by default if they are available and there are enough cores
Fri, 20 Jul 2012 22:19:46 +0200 blanchet minimal maxes + tuning
Fri, 20 Jul 2012 22:19:46 +0200 blanchet learn from SMT proofs when they can be minimized by Metis
Fri, 20 Jul 2012 22:19:46 +0200 blanchet convenience
Fri, 20 Jul 2012 22:19:46 +0200 blanchet learning should honor the fact override and the chained facts
Fri, 20 Jul 2012 22:19:46 +0200 blanchet added "learn_from_atp" command to MaSh, for patient users
Fri, 20 Jul 2012 22:19:46 +0200 blanchet more MaSh docs
Fri, 20 Jul 2012 22:19:46 +0200 blanchet learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds
Fri, 20 Jul 2012 22:19:46 +0200 blanchet learn command in MaSh
Fri, 20 Jul 2012 22:19:45 +0200 blanchet renamed ML structures
Wed, 18 Jul 2012 08:44:05 +0200 blanchet optimize parent computation in MaSh + remove temporary files
Wed, 18 Jul 2012 08:44:04 +0200 blanchet learn from minimized ATP proofs
Wed, 18 Jul 2012 08:44:04 +0200 blanchet use async manager to manage MaSh learners to make sure they get killed cleanly
Wed, 18 Jul 2012 08:44:04 +0200 blanchet added option to control which fact filter is used
Wed, 18 Jul 2012 08:44:04 +0200 blanchet make tracing an option
Wed, 18 Jul 2012 08:44:03 +0200 blanchet more implementation work on MaSh
Wed, 18 Jul 2012 08:44:03 +0200 blanchet started implementing MaSh client-side I/O
Wed, 18 Jul 2012 08:44:03 +0200 blanchet renamed Sledgehammer options
Wed, 18 Jul 2012 08:44:03 +0200 blanchet more code rationalization in relevance filter
Wed, 11 Jul 2012 21:43:19 +0200 blanchet further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
Wed, 23 May 2012 13:28:20 +0200 blanchet lower the monomorphization thresholds for less scalable provers
Sat, 21 Apr 2012 11:15:49 +0200 blanchet swap out Satallax, pull in E-SInE again -- it's not clear yet how useful Satallax is after proof reconstruction, whereas E-SInE performed surprisingly well on latest evaluations
Wed, 21 Mar 2012 16:53:24 +0100 blanchet improve "remote_satallax" by exploiting unsat core
Tue, 20 Mar 2012 18:42:45 +0100 blanchet made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
Tue, 20 Mar 2012 00:44:30 +0100 blanchet added "dont_preplay" alias
Fri, 16 Mar 2012 18:20:12 +0100 wenzelm outer syntax command definitions based on formal command_spec derived from theory header declarations;
Thu, 15 Mar 2012 20:07:00 +0100 wenzelm prefer formally checked @{keyword} parser;
Mon, 06 Feb 2012 23:01:01 +0100 blanchet renamed type encoding
Sat, 04 Feb 2012 12:08:18 +0100 blanchet made option available to users (mostly for experiments)
Thu, 02 Feb 2012 12:42:05 +0100 blanchet include new SPASS by default if available
Mon, 23 Jan 2012 17:40:32 +0100 blanchet renamed two files to make room for a new file
Thu, 19 Jan 2012 21:37:12 +0100 blanchet renamed "sound" option to "strict"
Thu, 19 Jan 2012 21:37:12 +0100 blanchet lower timeout for preplay, now that we have more preplay methods
Thu, 01 Dec 2011 13:34:14 +0100 blanchet added "minimize" option for more control over automatic minimization
Thu, 01 Dec 2011 13:34:13 +0100 blanchet renamed "slicing" to "slice"
Wed, 16 Nov 2011 16:35:19 +0100 blanchet thread in additional options to minimizer
Wed, 16 Nov 2011 13:22:36 +0100 blanchet make metis reconstruction handling more flexible
Wed, 16 Nov 2011 09:42:27 +0100 blanchet parse lambda translation option in Metis
Fri, 23 Sep 2011 16:44:51 +0200 blanchet reintroduced E-SInE now that it's unexpectedly working again (thanks to Geoff)
Thu, 22 Sep 2011 19:42:06 +0200 blanchet take out remote E-SInE -- it's broken and Geoff says it might take quite a while before he gets to it, plus it's fairly obsolete in the meantime
Wed, 07 Sep 2011 13:50:17 +0200 blanchet parse new experimental '@' encodings
Wed, 07 Sep 2011 13:50:17 +0200 blanchet tuning
Wed, 07 Sep 2011 09:10:41 +0200 blanchet rationalize uniform encodings
Mon, 05 Sep 2011 14:42:31 +0200 blanchet fixed handling of "sledgehammer_params", so that "sledgehammer_params [e]" is really the same as "sledgehammer_params [provers = e]"
Fri, 02 Sep 2011 14:43:20 +0200 blanchet renamed "Metis_Tactics" to "Metis_Tactic", now that there is only one Metis tactic ("metisFT" is legacy)
Tue, 30 Aug 2011 16:07:45 +0200 blanchet extended simple types with polymorphism -- the implementation still needs some work though
Thu, 25 Aug 2011 14:25:07 +0200 blanchet rationalized option names -- mono becomes raw_mono and mangled becomes mono
Wed, 24 Aug 2011 11:17:33 +0200 blanchet more reliable "sledgehammer\_tac" reconstruction, by avoiding "insert_tac"
Mon, 22 Aug 2011 15:02:45 +0200 blanchet cleaner handling of polymorphic monotonicity inference
less more (0) -120 tip