History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
Revision Date Author Comments
# eeea2b9e 25-Oct-2019 blanchet <none@none>

removed experimental encoding for Waldmeister


# a4bab154 04-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# 7110473f 30-Oct-2018 fleury <Mathias.Fleury@mpi-inf.mpg.de>

add reconstruction by veriT in method smt


# ef151f45 20-Jul-2018 blanchet <none@none>

don't lose facts that were introduced to deal with a theory or some preprocessing in the prover (e.g. the definition of 'abs' in an SMT proof)


# 8aec7217 01-Feb-2018 wenzelm <none@none>

tuned signature: more operations;


# 75c0bb14 13-Aug-2016 blanchet <none@none>

killed final stops in Sledgehammer and friends


# a4893486 16-Jul-2016 wenzelm <none@none>

tuned signature;


# 185dcd47 02-Apr-2016 wenzelm <none@none>

prefer infix operations;


# 08f53f20 01-Feb-2016 blanchet <none@none>

avoid error in Isar proof reconstruction if no ATP proof is available


# 19895c91 29-Jun-2015 blanchet <none@none>

removed chained facts from preplaying -- and careful about extra chained facts when removing 'proof -' and 'qed' from one-line Isar proofs


# 5091b5ae 03-Mar-2015 blanchet <none@none>

SPASS-Pirate is now called Pirate

--HG--
rename : src/HOL/Tools/ATP/scripts/remote_spass_pirate => src/HOL/Tools/ATP/scripts/remote_pirate


# 76c7446c 31-Oct-2014 wenzelm <none@none>

discontinued obsolete Output.urgent_message;


# 6260b828 12-Oct-2014 blanchet <none@none>

improved handling of extensionality in Isar proofs generated from LEO-II and Satallax


# f9be6fd2 02-Oct-2014 blanchet <none@none>

more precise lemma insertion


# 7da2f3ce 02-Oct-2014 blanchet <none@none>

insert lemmas closer to where they are needed, both for esthetics and (primarily) for correctness in case the lemma refers to a skolem


# 33cfb143 02-Oct-2014 blanchet <none@none>

eliminate duplicate hypotheses (which can arise due to (un)clausification)


# 78c3d543 02-Oct-2014 blanchet <none@none>

'moura' method is also useful for reconstructing skolemization of lambda-lifting of formulas for other provers than Z3


# 0b6cbc5a 15-Sep-2014 blanchet <none@none>

tuning


# f4d6dd0f 14-Sep-2014 blanchet <none@none>

removed accidental '@{print}'


# 8666297f 02-Sep-2014 steckerm <none@none>

Some work on the new waldmeister integration


# 63548199 28-Aug-2014 blanchet <none@none>

renamed 'skolem' to 'moura' (to suggest Z3-style skolemization); reintroduced 'fastforce' to the mix of tested proof methods


# 5b07dac6 28-Aug-2014 blanchet <none@none>

removed show stuttering


# 1bf7e2a5 28-Aug-2014 blanchet <none@none>

try 'skolem' method first for Z3


# 13c70a63 28-Aug-2014 blanchet <none@none>

added 'skolem' method, esp. for 'obtain's generated from Z3 proofs


# ac75f5e7 27-Aug-2014 blanchet <none@none>

renamed new SMT module from 'SMT2' to 'SMT'

--HG--
rename : src/HOL/SMT2.thy => src/HOL/SMT.thy
rename : src/HOL/Tools/SMT2/smt2_builtin.ML => src/HOL/Tools/SMT/smt_builtin.ML
rename : src/HOL/Tools/SMT2/smt2_config.ML => src/HOL/Tools/SMT/smt_config.ML
rename : src/HOL/Tools/SMT2/smt2_datatypes.ML => src/HOL/Tools/SMT/smt_datatypes.ML
rename : src/HOL/Tools/SMT2/smt2_failure.ML => src/HOL/Tools/SMT/smt_failure.ML
rename : src/HOL/Tools/SMT2/smt2_normalize.ML => src/HOL/Tools/SMT/smt_normalize.ML
rename : src/HOL/Tools/SMT2/smt2_real.ML => src/HOL/Tools/SMT/smt_real.ML
rename : src/HOL/Tools/SMT2/smt2_solver.ML => src/HOL/Tools/SMT/smt_solver.ML
rename : src/HOL/Tools/SMT2/smt2_systems.ML => src/HOL/Tools/SMT/smt_systems.ML
rename : src/HOL/Tools/SMT2/smt2_translate.ML => src/HOL/Tools/SMT/smt_translate.ML
rename : src/HOL/Tools/SMT2/smt2_util.ML => src/HOL/Tools/SMT/smt_util.ML
rename : src/HOL/Tools/SMT2/smtlib2.ML => src/HOL/Tools/SMT/smtlib.ML
rename : src/HOL/Tools/SMT2/smtlib2_interface.ML => src/HOL/Tools/SMT/smtlib_interface.ML
rename : src/HOL/Tools/SMT2/smtlib2_isar.ML => src/HOL/Tools/SMT/smtlib_isar.ML
rename : src/HOL/Tools/SMT2/smtlib2_proof.ML => src/HOL/Tools/SMT/smtlib_proof.ML
rename : src/HOL/Tools/SMT2/verit_isar.ML => src/HOL/Tools/SMT/verit_isar.ML
rename : src/HOL/Tools/SMT2/verit_proof.ML => src/HOL/Tools/SMT/verit_proof.ML
rename : src/HOL/Tools/SMT2/verit_proof_parse.ML => src/HOL/Tools/SMT/verit_proof_parse.ML
rename : src/HOL/Tools/SMT2/z3_new_interface.ML => src/HOL/Tools/SMT/z3_interface.ML
rename : src/HOL/Tools/SMT2/z3_new_isar.ML => src/HOL/Tools/SMT/z3_isar.ML
rename : src/HOL/Tools/SMT2/z3_new_proof.ML => src/HOL/Tools/SMT/z3_proof.ML
rename : src/HOL/Tools/SMT2/z3_new_real.ML => src/HOL/Tools/SMT/z3_real.ML
rename : src/HOL/Tools/SMT2/z3_new_replay.ML => src/HOL/Tools/SMT/z3_replay.ML
rename : src/HOL/Tools/SMT2/z3_new_replay_literals.ML => src/HOL/Tools/SMT/z3_replay_literals.ML
rename : src/HOL/Tools/SMT2/z3_new_replay_methods.ML => src/HOL/Tools/SMT/z3_replay_methods.ML
rename : src/HOL/Tools/SMT2/z3_new_replay_rules.ML => src/HOL/Tools/SMT/z3_replay_rules.ML
rename : src/HOL/Tools/SMT2/z3_new_replay_util.ML => src/HOL/Tools/SMT/z3_replay_util.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_prover_smt2.ML => src/HOL/Tools/Sledgehammer/sledgehammer_prover_smt.ML
rename : src/HOL/Word/Tools/smt2_word.ML => src/HOL/Word/Tools/smt_word.ML


# fbf4ecd4 05-Aug-2014 blanchet <none@none>

rationalize Skolem names


# eea37d65 05-Aug-2014 blanchet <none@none>

tuning


# f31ea233 05-Aug-2014 blanchet <none@none>

tuning


# 55792f6c 04-Aug-2014 blanchet <none@none>

deal with E definitions


# d0ae16b7 04-Aug-2014 blanchet <none@none>

cleaner 'compress' option


# 8dd03340 04-Aug-2014 blanchet <none@none>

tuned terminology (cf. 'isar_proofs' option)


# 12791f01 03-Aug-2014 blanchet <none@none>

rationalized sorting of facts -- so that preplaying (almost always) coincides with the real thing, preventing odd failures


# 29af0064 24-Jul-2014 blanchet <none@none>

refined filter for ATP steps to avoid 'have True' steps in E proofs


# 5a5724ad 24-Jul-2014 blanchet <none@none>

'shift_quantors' is not an E skolemization rule (cf. 3ab503b04bdb)


# 3d540b5c 01-Aug-2014 blanchet <none@none>

better duplicate detection


# 9abfd5af 01-Aug-2014 blanchet <none@none>

normalize conjectures vs. negated conjectures when comparing terms


# 504e120b 01-Aug-2014 blanchet <none@none>

tweaked 'clone' formula detection


# 66c99a97 01-Aug-2014 blanchet <none@none>

fine-tuned Isar reconstruction, esp. boolean simplifications


# 89efba68 01-Aug-2014 blanchet <none@none>

centralized boolean simplification so that e.g. LEO-II benefits from it


# 07e7301c 01-Aug-2014 blanchet <none@none>

better handling of variable names


# 23ce6ae4 01-Aug-2014 blanchet <none@none>

nicer generated variable names


# af295814 01-Aug-2014 blanchet <none@none>

tuning


# 5e9f3c95 01-Aug-2014 blanchet <none@none>

tuning


# a4c762db 01-Aug-2014 blanchet <none@none>

more precise handling of LEO-II skolemization


# f2d6b3bc 01-Aug-2014 blanchet <none@none>

beware of 'skolem' rules that do not skolemize (e.g. LEO-II)


# ac69d2cf 01-Aug-2014 blanchet <none@none>

added appropriate method for skolemization of Z3 steps to the mix


# c91b511e 01-Aug-2014 blanchet <none@none>

tentatively took out 'fastforce' from the set of tried methods -- it seems to be largely subsumed and is hard to silence


# 4a5e0afe 01-Aug-2014 blanchet <none@none>

tuning


# 16de9a98 01-Aug-2014 blanchet <none@none>

eliminated Sledgehammer's "min" subcommand (and lots of complications in the code)


# 1f0ff8fb 30-Jul-2014 fleury <none@none>

Skolemization for tmp_ite_elim rule in the SMT solver veriT.


# fa2cfdb9 30-Jul-2014 fleury <none@none>

Changing the role of rule "tmp_ite_elim" of the SMT solver veriT to Lemma.


# 4c1fa505 30-Jul-2014 fleury <none@none>

Whitespace and indentation correction.


# 688959b7 30-Jul-2014 fleury <none@none>

imported patch hilbert_choice_support


# f5c59070 30-Jul-2014 fleury <none@none>

veriT changes for lifted terms, and ite_elim rules.


# 8edb0caa 30-Jul-2014 fleury <none@none>

Subproofs for the SMT solver veriT.


# a40467dc 30-Jul-2014 fleury <none@none>

Basic support for the SMT prover veriT.


# fae19496 30-Jul-2014 fleury <none@none>

Skolemization support for leo-II and Zipperposition.


# b8f4c9ec 29-Jul-2014 blanchet <none@none>

also try 'metis' with 'full_types'


# 628399f0 24-Jun-2014 blanchet <none@none>

supports gradual skolemization (cf. Z3) by threading context through correctly


# 9dcaf59f 24-Jun-2014 blanchet <none@none>

given two one-liners, only show the best of the two


# 05a02815 24-Jun-2014 blanchet <none@none>

don't generate Isar proof skeleton for what amounts to a one-line proof


# 047b3f9c 12-Jun-2014 blanchet <none@none>

renamed Sledgehammer options


# c5b00bcc 02-Jun-2014 fleury <none@none>

basic setup for zipperposition prover


# de96180b 21-May-2014 blanchet <none@none>

properly reconstruct helpers in Z3 proofs


# 312fdfa6 21-May-2014 blanchet <none@none>

tuning


# 0798791c 16-May-2014 blanchet <none@none>

correctly add extra facts to lemmas (cf. conjecture and hypotheses) in Z3 Isar proofs


# 8589cd89 16-May-2014 blanchet <none@none>

use 'simp add:' syntax in Sledgehammer rather than 'using'


# 91badc4f 04-May-2014 blanchet <none@none>

added 'satx' to Sledgehammer's portfolio (cf. 'isar_try0')


# 940de23f 14-Mar-2014 blanchet <none@none>

consolidate consecutive steps that prove the same formula


# bf8eef3e 14-Mar-2014 blanchet <none@none>

undo rewrite rules (e.g. for 'fun_app') in Isar


# 2c88514c 14-Mar-2014 blanchet <none@none>

debugging stuff


# 00ff94c2 14-Mar-2014 blanchet <none@none>

more simplification of trivial steps


# 1a139c00 14-Mar-2014 blanchet <none@none>

tuning


# 7009730a 13-Mar-2014 blanchet <none@none>

tuning


# 8b8b6855 13-Mar-2014 blanchet <none@none>

simplified preplaying information


# f936bab5 13-Mar-2014 blanchet <none@none>

integrate SMT2 with Sledgehammer


# e8872587 06-Mar-2014 wenzelm <none@none>

tuned signature;


# cf3941c9 13-Feb-2014 blanchet <none@none>

avoid changing the state's context -- this results in transfer problems later with SMT, and hence preplay tactic failures


# 7f5432b9 04-Feb-2014 blanchet <none@none>

more generous Isar proof compression -- try to remove failing steps


# f9098ce8 04-Feb-2014 blanchet <none@none>

do a second phase of proof compression after minimization


# 477409cf 04-Feb-2014 blanchet <none@none>

tuned code


# a41de456 04-Feb-2014 blanchet <none@none>

split 'linarith' and 'presburger' (to avoid annoying warnings + to speed up reconstruction when 'presburger' is needed)


# da44b6aa 03-Feb-2014 blanchet <none@none>

rationalized lists of methods


# 22f66987 03-Feb-2014 blanchet <none@none>

extended method list


# fb11429b 03-Feb-2014 blanchet <none@none>

generate comments in Isar proofs


# 9a5b75f2 03-Feb-2014 blanchet <none@none>

renamed 'smt' option 'smt_proofs' to avoid clash with 'smt' prover


# 2946be22 03-Feb-2014 blanchet <none@none>

tuned behavior of 'smt' option


# 46915898 03-Feb-2014 blanchet <none@none>

proper fresh name generation


# af459cea 03-Feb-2014 blanchet <none@none>

tuned data structure


# b54f3e71 03-Feb-2014 blanchet <none@none>

tuned data structure


# 88ad28c0 03-Feb-2014 blanchet <none@none>

less aggressive evaluation


# 328c952e 03-Feb-2014 blanchet <none@none>

added a new version of 'metis' to the mix


# 37d29385 03-Feb-2014 blanchet <none@none>

implemented new 'try0_isar' semantics


# f0dd587a 03-Feb-2014 blanchet <none@none>

got rid of 'try0' step that is now redundant


# c0348805 03-Feb-2014 blanchet <none@none>

centralize more preplaying


# 714b0a4e 03-Feb-2014 blanchet <none@none>

centralize preplaying


# fcc30082 03-Feb-2014 blanchet <none@none>

tuned


# 62d265e3 03-Feb-2014 blanchet <none@none>

added 'smt' option to control generation of 'by smt' proofs


# 700f2e9d 03-Feb-2014 blanchet <none@none>

renamed ML file

--HG--
rename : src/HOL/Tools/Sledgehammer/sledgehammer_reconstructor.ML => src/HOL/Tools/Sledgehammer/sledgehammer_proof_methods.ML


# 70573b75 03-Feb-2014 blanchet <none@none>

tuning


# 94e4af3c 03-Feb-2014 blanchet <none@none>

merged 'reconstructors' and 'proof methods'


# c0b367e3 03-Feb-2014 blanchet <none@none>

tuning


# 58f3d3c0 02-Feb-2014 blanchet <none@none>

more data structure rationalization


# f7251444 02-Feb-2014 blanchet <none@none>

more data structure rationalization


# 28c29fd3 02-Feb-2014 blanchet <none@none>

rationalized threading of 'metis' arguments


# ac271564 02-Feb-2014 blanchet <none@none>

refactored data structure (step 3)


# a987912b 02-Feb-2014 blanchet <none@none>

unform treatment of preplay_timeout = 0 and > 0


# 0199bc1a 02-Feb-2014 blanchet <none@none>

use Skolem proof methods appropriately


# 47bd3a59 02-Feb-2014 blanchet <none@none>

simplified data structure -- eliminated distinction between 'first-class' and 'second-class' proof methods


# 348374bc 31-Jan-2014 blanchet <none@none>

generalized preplaying infrastructure to store various results for various methods


# 03de82be 31-Jan-2014 blanchet <none@none>

added a 'trace' option


# c24c8aaa 31-Jan-2014 blanchet <none@none>

moved code around


# 5c1d5f08 31-Jan-2014 blanchet <none@none>

added 'algebra' to the mix


# 6cacd6c0 31-Jan-2014 blanchet <none@none>

more informative trace


# eb41fa66 31-Jan-2014 blanchet <none@none>

better tracing + syntactically correct 'metis' calls


# 70b7915d 31-Jan-2014 blanchet <none@none>

tuned ML function names


# fed5d9bd 31-Jan-2014 blanchet <none@none>

tuning


# 945bedcb 31-Jan-2014 blanchet <none@none>

moved ML code around


# eb52da60 31-Jan-2014 blanchet <none@none>

renamed many Sledgehammer ML files to clarify structure

--HG--
rename : src/HOL/Tools/Sledgehammer/sledgehammer_run.ML => src/HOL/Tools/Sledgehammer/sledgehammer.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML => src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_annotate.ML => src/HOL/Tools/Sledgehammer/sledgehammer_isar_annotate.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_compress.ML => src/HOL/Tools/Sledgehammer/sledgehammer_isar_compress.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_minimize_isar.ML => src/HOL/Tools/Sledgehammer/sledgehammer_isar_minimize.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_preplay.ML => src/HOL/Tools/Sledgehammer/sledgehammer_isar_preplay.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_print.ML => src/HOL/Tools/Sledgehammer/sledgehammer_isar_print.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_proof.ML => src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_try0.ML => src/HOL/Tools/Sledgehammer/sledgehammer_isar_try0.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML => src/HOL/Tools/Sledgehammer/sledgehammer_prover_minimize.ML


# 2109d469 30-Jan-2014 blanchet <none@none>

renamed Sledgehammer options for symmetry between positive and negative versions


# 70e2710a 19-Dec-2013 blanchet <none@none>

made timeouts in Sledgehammer not be 'option's -- simplified lots of code


# 7a677357 20-Nov-2013 blanchet <none@none>

fixed spying so that the envirnoment variables are queried at run-time not at build-time


# 7ff3b5f2 19-Nov-2013 blanchet <none@none>

tuning


# baf36949 16-Oct-2013 blanchet <none@none>

added comment


# 6a7956b5 15-Oct-2013 blanchet <none@none>

use MePo with Auto Sledgehammer, because it's lighter than MaSh and always available


# 2f9705a4 04-Oct-2013 blanchet <none@none>

run fewer provers in "try" mode


# 91edd2e9 04-Oct-2013 blanchet <none@none>

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)


# 8c08106e 04-Oct-2013 blanchet <none@none>

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)


# be10b5cc 23-Sep-2013 blanchet <none@none>

added "spy" option to Sledgehammer


# 3c5d67b1 20-Sep-2013 blanchet <none@none>

merged "isar_try0" and "isar_minimize" options


# d558d966 20-Sep-2013 blanchet <none@none>

hardcoded obscure option


# 30fb6f57 20-Sep-2013 blanchet <none@none>

hard-coded an obscure option


# 96f42bd1 20-Sep-2013 blanchet <none@none>

use configuration mechanism for low-level tracing


# e3d74f5a 20-Sep-2013 blanchet <none@none>

took out Waldmeister from list of default provers -- it's usually just visual noise, and its integration in Sledgehammer leaves much to be desired


# fff567a1 20-Sep-2013 blanchet <none@none>

tuning (use a blacklist instead of a whitelist)


# e762273c 22-Aug-2013 blanchet <none@none>

fixed subtle bug with "take" + thread overlord through


# d7f79e47 22-Aug-2013 blanchet <none@none>

have kill_all also kill MaSh server + be paranoid about reloading after clear_state, to allow for easier experimentation


# 0122820d 17-Aug-2013 wenzelm <none@none>

prefer system option sledgehammer_timeout, with standard GUI in jEdit Plugin Options;


# 70b5ba3c 17-Aug-2013 wenzelm <none@none>

some protocol to determine provers according to ML;


# c6e889d9 17-Aug-2013 wenzelm <none@none>

always enable "minimize" to simplify interaction model;
override params more directly -- they are no longer echoed in minimize command;


# e19e4dd4 17-Aug-2013 wenzelm <none@none>

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;
back to Normal mode: with output_result it is sufficient to determine TTY vs. PIDE operation;


# 5caf3769 16-Aug-2013 wenzelm <none@none>

eliminated pointless subgoal argument;


# a461805e 16-Aug-2013 wenzelm <none@none>

more direct sledgehammer configuration via mode = Normal_Result and output_result;
retain standard sledgehammer parallelization policies;


# 5e3dc32f 12-Aug-2013 wenzelm <none@none>

clarified Query_Operation.register: avoid hard-wired parallel policy;
sledgehammer: more conventional parallel exception handling -- print just one interrupt;


# 686da4bc 08-Aug-2013 wenzelm <none@none>

dockable window for Sledgehammer, based on asynchronous/parallel query operation;


# 68670fb3 12-Jul-2013 wenzelm <none@none>

hybrid "auto" tool setup, for TTY (within theory) and PIDE (global print function);


# e46f39e8 12-Jul-2013 wenzelm <none@none>

system options for Isabelle/HOL proof tools;


# 44a9ccdf 12-Jul-2013 smolkas <none@none>

added sledgehammer parameters isar_try0 and isar_minimize and their negative aliases


# 142db0d1 09-Jul-2013 smolkas <none@none>

completely rewrote SH compress; added two parameters for experimentation/fine grained control


# c56cbeb4 11-Jun-2013 smolkas <none@none>

make use of show_type_emphasis instead of using hack; make sure global configurations don't affect proof script creation


# 240dfa4c 21-May-2013 blanchet <none@none>

added compatibility alias


# e232176f 16-May-2013 blanchet <none@none>

tuning -- renamed '_from_' to '_of_' in Sledgehammer


# c71d3769 15-May-2013 wenzelm <none@none>

clarified preferences: "override" re-initialized on prover startup, and "default" sent to PG -- thus recover typical defaults like auto-quickcheck in PG 4.x;


# 42c02b01 15-May-2013 wenzelm <none@none>

maintain ProofGeneral preferences within ProofGeneral module;
initialize Isabelle/Pure preferences within normal user space (with antiquotations);
tuned;


# 801d585a 15-May-2013 blanchet <none@none>

renamed Sledgehammer functions with 'for' in their names to 'of'


# cb7d30c4 15-May-2013 wenzelm <none@none>

just one ProofGeneral module;

--HG--
rename : src/Pure/ProofGeneral/proof_general_emacs.ML => src/Pure/ProofGeneral/proof_general.ML


# 323241a5 06-May-2013 smolkas <none@none>

added preplay tracing


# a9f74476 27-Mar-2013 wenzelm <none@none>

more robust access Toplevel.proof_of -- prefer warning via Toplevel.unknown_proof over hard crash (notably for skipped proofs);


# 982d7cae 20-Feb-2013 blanchet <none@none>

minimize SMT proofs with E if Isar proofs are desired and Metis managed to preplay


# 594b835f 20-Feb-2013 blanchet <none@none>

fixed typo in option name


# 24cd411a 20-Feb-2013 blanchet <none@none>

made "isar_proofs" a 3-way option, to provide a way to totally disable isar_proofs if desired


# 5be3a0be 20-Feb-2013 blanchet <none@none>

alias for people like me


# 826b00b6 15-Feb-2013 blanchet <none@none>

killed legacy alias


# 583ed312 14-Feb-2013 smolkas <none@none>

renamed sledgehammer_shrink to sledgehammer_compress

--HG--
rename : src/HOL/Tools/Sledgehammer/sledgehammer_shrink.ML => src/HOL/Tools/Sledgehammer/sledgehammer_compress.ML


# 05efe995 11-Jan-2013 smolkas <none@none>

tuned


# e75a80fd 11-Jan-2013 smolkas <none@none>

set show_markup to false in order to avoid problems in jedit


# 5d18cfa7 05-Jan-2013 blanchet <none@none>

nicer output


# 70700972 05-Jan-2013 blanchet <none@none>

pass option to minimize


# b0c1a438 04-Jan-2013 blanchet <none@none>

renamed "kill" subcommand to avoid clash with "kill" keyword (which confuses Proof General and results in strange syntax highlighting)


# ee1dd9f3 19-Dec-2012 blanchet <none@none>

crank up default timeout for MaSh ATP learning


# 74412286 15-Dec-2012 blanchet <none@none>

thread no timeout properly


# f99d6679 11-Dec-2012 blanchet <none@none>

adopt the neutral "prover" terminology for MaSh rather than the ambiguous/wrong ATP terminology (which sometimes excludes SMT solvers)


# 2a322b89 12-Nov-2012 blanchet <none@none>

create temp directory if not already created


# 33afc4e3 06-Nov-2012 blanchet <none@none>

renamed Sledgehammer option


# 59bd790a 18-Oct-2012 blanchet <none@none>

renamed Isar-proof related options + changed semantics of Isar shrinking


# 111003cb 28-Sep-2012 blanchet <none@none>

tuned message


# a296c798 13-Sep-2012 blanchet <none@none>

merged two commands


# 0d360337 26-Jul-2012 blanchet <none@none>

detect unknown options again


# c053a937 23-Jul-2012 blanchet <none@none>

don't relearn old facts in Isar mode


# b49eff54 23-Jul-2012 blanchet <none@none>

took out CVC3 again -- there seems to be issues with the server version of CVC3 + minor tweaks


# 84aa75b1 20-Jul-2012 blanchet <none@none>

honor suggested MaSh weights


# 92803e9b 20-Jul-2012 blanchet <none@none>

use CVC3 and Yices by default if they are available and there are enough cores


# caae738e 20-Jul-2012 blanchet <none@none>

minimal maxes + tuning


# 279df876 20-Jul-2012 blanchet <none@none>

learn from SMT proofs when they can be minimized by Metis


# 63710e18 20-Jul-2012 blanchet <none@none>

convenience


# 9e4601f2 20-Jul-2012 blanchet <none@none>

learning should honor the fact override and the chained facts


# 4e48e0a3 20-Jul-2012 blanchet <none@none>

added "learn_from_atp" command to MaSh, for patient users


# 71baadff 20-Jul-2012 blanchet <none@none>

more MaSh docs


# 833017c5 20-Jul-2012 blanchet <none@none>

learn on explicit "min" command but do the learning in a thread, since it may take a couple of seconds


# 48ae61a7 20-Jul-2012 blanchet <none@none>

learn command in MaSh


# 7b5f817b 20-Jul-2012 blanchet <none@none>

renamed ML structures


# 8352d0ae 18-Jul-2012 blanchet <none@none>

optimize parent computation in MaSh + remove temporary files


# 57033d31 18-Jul-2012 blanchet <none@none>

learn from minimized ATP proofs


# 45add41e 18-Jul-2012 blanchet <none@none>

use async manager to manage MaSh learners to make sure they get killed cleanly


# 8531f3b7 18-Jul-2012 blanchet <none@none>

added option to control which fact filter is used


# 750cae58 18-Jul-2012 blanchet <none@none>

make tracing an option


# ae019a7f 18-Jul-2012 blanchet <none@none>

more implementation work on MaSh


# 7b7189a4 18-Jul-2012 blanchet <none@none>

started implementing MaSh client-side I/O


# c8c44f09 18-Jul-2012 blanchet <none@none>

renamed Sledgehammer options


# 928cadab 18-Jul-2012 blanchet <none@none>

more code rationalization in relevance filter


# a74b00cb 11-Jul-2012 blanchet <none@none>

further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)


# e91f0eee 23-May-2012 blanchet <none@none>

lower the monomorphization thresholds for less scalable provers


# 3857c267 21-Apr-2012 blanchet <none@none>

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


# 75fbec2e 21-Mar-2012 blanchet <none@none>

improve "remote_satallax" by exploiting unsat core


# b1a2301c 20-Mar-2012 blanchet <none@none>

made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release


# 8d633043 19-Mar-2012 blanchet <none@none>

added "dont_preplay" alias


# 150d8520 16-Mar-2012 wenzelm <none@none>

outer syntax command definitions based on formal command_spec derived from theory header declarations;


# de9fb383 15-Mar-2012 wenzelm <none@none>

prefer formally checked @{keyword} parser;


# 1879ce1b 06-Feb-2012 blanchet <none@none>

renamed type encoding


# 91817e9b 03-Feb-2012 blanchet <none@none>

made option available to users (mostly for experiments)


# 2e4d0d30 01-Feb-2012 blanchet <none@none>

include new SPASS by default if available


# 678bfbab 23-Jan-2012 blanchet <none@none>

renamed two files to make room for a new file

--HG--
rename : src/HOL/Tools/ATP/atp_translate.ML => src/HOL/Tools/ATP/atp_problem_generate.ML
rename : src/HOL/Tools/ATP/atp_reconstruct.ML => src/HOL/Tools/ATP/atp_proof_reconstruct.ML
rename : src/HOL/Tools/ATP/atp_redirect.ML => src/HOL/Tools/ATP/atp_proof_redirect.ML
rename : src/HOL/Tools/Metis/metis_translate.ML => src/HOL/Tools/Metis/metis_generate.ML


# 37b1d92a 19-Jan-2012 blanchet <none@none>

renamed "sound" option to "strict"


# 04546773 19-Jan-2012 blanchet <none@none>

lower timeout for preplay, now that we have more preplay methods


# 5ad5d53e 01-Dec-2011 blanchet <none@none>

added "minimize" option for more control over automatic minimization


# 6dda2ef1 01-Dec-2011 blanchet <none@none>

renamed "slicing" to "slice"


# 572708e4 16-Nov-2011 blanchet <none@none>

thread in additional options to minimizer


# 56883261 16-Nov-2011 blanchet <none@none>

make metis reconstruction handling more flexible


# 752baf74 16-Nov-2011 blanchet <none@none>

parse lambda translation option in Metis


# 532d01ea 23-Sep-2011 blanchet <none@none>

reintroduced E-SInE now that it's unexpectedly working again (thanks to Geoff)


# dbc3b669 22-Sep-2011 blanchet <none@none>

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


# 1f31c211 07-Sep-2011 blanchet <none@none>

parse new experimental '@' encodings


# 9ef818d4 07-Sep-2011 blanchet <none@none>

tuning


# d5c90015 07-Sep-2011 blanchet <none@none>

rationalize uniform encodings


# 04567399 05-Sep-2011 blanchet <none@none>

fixed handling of "sledgehammer_params", so that "sledgehammer_params [e]" is really the same as "sledgehammer_params [provers = e]"


# 79752fb0 02-Sep-2011 blanchet <none@none>

renamed "Metis_Tactics" to "Metis_Tactic", now that there is only one Metis tactic ("metisFT" is legacy)

--HG--
rename : src/HOL/Tools/Metis/metis_tactics.ML => src/HOL/Tools/Metis/metis_tactic.ML


# 874972d6 30-Aug-2011 blanchet <none@none>

extended simple types with polymorphism -- the implementation still needs some work though


# 6dbce3bd 25-Aug-2011 blanchet <none@none>

rationalized option names -- mono becomes raw_mono and mangled becomes mono


# ad5d36d9 24-Aug-2011 blanchet <none@none>

more reliable "sledgehammer\_tac" reconstruction, by avoiding "insert_tac"


# de0c7814 22-Aug-2011 blanchet <none@none>

cleaner handling of polymorphic monotonicity inference


# 5a6754e8 09-Aug-2011 blanchet <none@none>

renamed E wrappers for consistency with CASC conventions


# 4bb2ac36 26-Jul-2011 blanchet <none@none>

renamed "preds" encodings to "guards"


# 94ac38d9 01-Jul-2011 blanchet <none@none>

renamed "type_sys" to "type_enc", which is more accurate


# 14befe8d 27-Jun-2011 blanchet <none@none>

added "sound" option to force Sledgehammer to be pedantically sound


# 59caf625 27-Jun-2011 blanchet <none@none>

removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway


# 3693f5b3 09-Jun-2011 blanchet <none@none>

removed "atp" and "atps" aliases, which users should have forgotten by now if they ever used them


# 2987e870 09-Jun-2011 blanchet <none@none>

fewer monomorphic instances are necessary, thanks to Sascha's new monomorphizer -- backed up by Judgment Day


# 2259fd65 08-Jun-2011 blanchet <none@none>

killed "explicit_apply" option in Sledgehammer -- the "smart" default is about as lightweight as "false" and just as complete as "true"


# a9d607d7 31-May-2011 blanchet <none@none>

parse optional type system specification


# 47a925bb 31-May-2011 blanchet <none@none>

first step in sharing more code between ATP and Metis translation

--HG--
rename : src/HOL/Tools/Sledgehammer/sledgehammer_atp_reconstruct.ML => src/HOL/Tools/ATP/atp_reconstruct.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML => src/HOL/Tools/ATP/atp_translate.ML


# f1c4bd91 30-May-2011 blanchet <none@none>

made "explicit_apply" smarter -- no need to force explicit applications in minimizer on all constants, better do it more fine granularly


# 2fd7dac8 30-May-2011 blanchet <none@none>

fixed syntax of min options


# aa6c0a43 30-May-2011 blanchet <none@none>

minimize with Metis if possible


# d955103d 27-May-2011 blanchet <none@none>

try both "metis" and (on failure) "metisFT" in replay


# 88ed198e 27-May-2011 blanchet <none@none>

prioritize try and auto try's tools, with fast ones first, with a slight preference for provers vs. counterexample generators


# ccd855c0 27-May-2011 blanchet <none@none>

handle non-auto try case of Sledgehammer better


# af064218 27-May-2011 blanchet <none@none>

added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods


# 3e4271be 27-May-2011 blanchet <none@none>

renamed "Auto_Tools" "Try"

--HG--
rename : src/Tools/auto_tools.ML => src/Tools/try.ML


# 1f5d8ddb 27-May-2011 blanchet <none@none>

renamed "metis_timeout" to "preplay_timeout" and continued implementation


# 64a1dcc6 27-May-2011 blanchet <none@none>

shorten minimizer command further, exploiting until-now-undocumented syntax


# 2b3d2c60 27-May-2011 blanchet <none@none>

added syntax for specifying Metis timeout (currently used only by SMT solvers)


# 98c977b9 27-May-2011 blanchet <none@none>

reintroduced Waldmeister but limit the number of remote threads created


# e9d92762 27-May-2011 blanchet <none@none>

renamed "minimize" to "min" to make Sledgehammer output a little bit more concise


# 8538fde4 27-May-2011 blanchet <none@none>

take out Waldmeister from default for now -- success rate too low on Judgment Day


# 235523f1 27-May-2011 blanchet <none@none>

always run Sledgehammer synchronously in the jEdit interface (until the multithreading support for Proof General is ported)


# a6ca43c6 22-May-2011 blanchet <none@none>

improved Waldmeister support -- even run it by default on unit equational goals


# 68cbed9b 13-May-2011 blanchet <none@none>

reduce the number of mono iterations to prevent the mono code from going berserk


# bd96d2a2 13-May-2011 blanchet <none@none>

added convenience syntax


# e4da3e95 12-May-2011 blanchet <none@none>

renamed "max_mono_instances" to "max_new_mono_instances" and changed its semantics accordingly


# e63aa543 12-May-2011 blanchet <none@none>

ensure that Auto Sledgehammer is run with full type information


# 499db001 12-May-2011 blanchet <none@none>

added "max_mono_instances" option to Sledgehammer and renamed old "monomorphize_limit" option


# 78a03012 04-May-2011 blanchet <none@none>

smoother handling of ! and ? in type system names


# ff6987bc 02-May-2011 blanchet <none@none>

use strings to encode type systems in ATP module, to reduce the amount of out-of-place information and also to make it easier to print the type system used


# e065c20f 01-May-2011 blanchet <none@none>

restructured type systems some more -- the old naming schemes had "argshg diff |less" and "tagshg diff |less" as equivalent and didn't support a monomorphic version of "tags"


# 2e6f3ec7 01-May-2011 blanchet <none@none>

use ! for mildly unsound and !! for very unsound encodings


# d4905648 01-May-2011 blanchet <none@none>

implement the new ATP type system in Sledgehammer


# a68b7a8f 01-May-2011 blanchet <none@none>

make sure the minimizer monomorphizes when it should


# d274cdde 01-May-2011 blanchet <none@none>

added (without implementation yet) new type encodings for Sledgehammer/ATP


# 52982fc5 21-Apr-2011 blanchet <none@none>

tuning


# 24fe4587 21-Apr-2011 blanchet <none@none>

cleanup: get rid of "may_slice" arguments without changing semantics


# e8264200 21-Apr-2011 blanchet <none@none>

implemented general slicing for ATPs, especially E 1.2w and above


# 6d2612c8 16-Apr-2011 wenzelm <none@none>

modernized structure Proof_Context;


# 1aac892e 05-Apr-2011 blanchet <none@none>

renamed "const_args" option value to "args"


# 199d07be 05-Apr-2011 blanchet <none@none>

killed unimplemented type encoding "preds"


# d0b3dd85 04-Apr-2011 blanchet <none@none>

if "monomorphize" is enabled, mangle the type information in the names by default


# 4e0b77b1 31-Mar-2011 blanchet <none@none>

added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default


# e46718bc 08-Feb-2011 blanchet <none@none>

available_provers ~> supported_provers (for clarity)


# ef2d6500 08-Jan-2011 wenzelm <none@none>

misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;


# 3e91f867 17-Dec-2010 blanchet <none@none>

convenient syntax for setting provers -- useful for debugging, not for general consumption and hence not documented


# 9de777b9 16-Dec-2010 blanchet <none@none>

make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive


# e07fbc0b 15-Dec-2010 blanchet <none@none>

make "full_types" take precedence over "type_sys"


# 59669977 15-Dec-2010 blanchet <none@none>

implemented partially-typed "tags" type encoding


# 31d6abde 15-Dec-2010 blanchet <none@none>

implemented new type system encoding "overload_args", which is more lightweight than "const_args" (the unsound default) and hopefully almost as sound


# c8db1b11 15-Dec-2010 blanchet <none@none>

added "type_sys" option to Sledgehammer


# c7c67363 08-Dec-2010 blanchet <none@none>

split "Sledgehammer" module into two parts, to resolve forthcoming dependency problems

--HG--
rename : src/HOL/Tools/Sledgehammer/sledgehammer.ML => src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
rename : src/HOL/Tools/Sledgehammer/sledgehammer.ML => src/HOL/Tools/Sledgehammer/sledgehammer_run.ML


# 82f13fa9 03-Dec-2010 blanchet <none@none>

replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us


# 644aabca 03-Dec-2010 blanchet <none@none>

run synchronous Auto Tools in parallel


# 2bcc030f 18-Nov-2010 blanchet <none@none>

enabled SMT solver in Sledgehammer by default


# cdd76953 10-Nov-2010 wenzelm <none@none>

use official/portable Multithreading.max_threads_value, which is also subject to user preferences (NB: Thread.numProcessors is apt to lead to surprises like very high numbers for systems with hyperthreading);


# fce219e4 03-Nov-2010 blanchet <none@none>

use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
updated docs


# 020b02b6 03-Nov-2010 blanchet <none@none>

standardize on seconds for Nitpick and Sledgehammer timeouts


# beb1bdb2 26-Oct-2010 blanchet <none@none>

integrated "smt" proof method with Sledgehammer


# 2b947a1e 26-Oct-2010 blanchet <none@none>

tuning


# e39575ea 26-Oct-2010 blanchet <none@none>

make SML/NJ happy


# 9b0b8dcf 25-Oct-2010 blanchet <none@none>

make "sledgehammer_params" work on single-threaded platforms


# 5a563fce 22-Oct-2010 blanchet <none@none>

more robust handling of "remote_" vs. non-"remote_" provers


# 3b4fd903 22-Oct-2010 blanchet <none@none>

fixed signature of "is_smt_solver_installed";
renaming


# b0757fd0 22-Oct-2010 blanchet <none@none>

took out "smt"/"remote_smt" from default ATPs until they are properly implemented


# 43992c32 22-Oct-2010 blanchet <none@none>

make Sledgehammer minimizer fully work with SMT


# b19da212 21-Oct-2010 blanchet <none@none>

first step in adding support for an SMT backend to Sledgehammer


# e51bc677 21-Oct-2010 blanchet <none@none>

use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."


# eb1f6702 13-Sep-2010 blanchet <none@none>

use 30 s instead of 60 s as the default Sledgehammer timeout;
very few proofs are lost this way (esp. thanks to the parallel use of provers, cf. Boehme & Nipkow 2010), and this is much more tolerable for users


# c1e800ce 10-Sep-2010 blanchet <none@none>

tuning


# 8a52405a 11-Sep-2010 blanchet <none@none>

finished renaming "Auto_Counterexample" to "Auto_Tools"


# 19ff77cf 11-Sep-2010 blanchet <none@none>

implemented Auto Sledgehammer


# cab0aee2 01-Sep-2010 blanchet <none@none>

got rid of the "theory_relevant" option;
instead, have fudge factors that behave more smoothly for all provers


# 0df9f4dc 01-Sep-2010 blanchet <none@none>

generalize theorem argument parsing syntax


# 3c56c5f7 31-Aug-2010 blanchet <none@none>

finished renaming


# b85821b1 31-Aug-2010 blanchet <none@none>

added "expect" feature of Nitpick to Sledgehammer, for regression testing


# fa05f58c 31-Aug-2010 blanchet <none@none>

added "blocking" option to Sledgehammer to run in synchronous mode;
sometimes useful, e.g. for testing


# 6e6390ba 31-Aug-2010 blanchet <none@none>

add a penalty for being higher-order


# 01e73533 30-Aug-2010 blanchet <none@none>

make Sledgehammer's relevance filter somewhat slacker


# 5a249478 25-Aug-2010 blanchet <none@none>

reorganize options regarding to the relevance threshold and decay


# e914d6ff 25-Aug-2010 blanchet <none@none>

make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
"max_relevant" is more reliable than "max_relevant_per_iter";
also made sure that the option is monotone -- larger values should lead to more axioms -- which wasn't always the case before;
SOS for Vampire makes a difference of about 3% (i.e. 3% more proofs are found)


# 36d6a1a2 25-Aug-2010 blanchet <none@none>

get rid of "defs_relevant" feature;
nobody uses it and it works poorly


# 6dbcf8ce 25-Aug-2010 blanchet <none@none>

renamed "relevance_convergence" to "relevance_decay"


# ac50c74a 23-Aug-2010 blanchet <none@none>

invert semantics of "relevance_convergence", to make it more intuitive


# f2d120d1 23-Aug-2010 blanchet <none@none>

if no facts were selected on first iteration, try again with a lower threshold


# d0717f2d 18-Aug-2010 blanchet <none@none>

get rid of "minimize_timeout", now that there's an automatic adaptive timeout mechanism in "minimize"


# 93202b28 18-Aug-2010 blanchet <none@none>

added "max_relevant_per_iter" option to Sledgehammer


# 9aaf659f 08-Aug-2010 blanchet <none@none>

move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)

--HG--
rename : src/HOL/Tools/Sledgehammer/sledgehammer_fact_minimizer.ML => src/HOL/Tools/Sledgehammer/sledgehammer_fact_minimize.ML


# 65ac7ddf 29-Jul-2010 blanchet <none@none>

use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
this replaces the previous, somewhat messy solution of adding "extra" clauses


# 977daf9f 28-Jul-2010 blanchet <none@none>

minor refactoring


# 706bb890 28-Jul-2010 blanchet <none@none>

minor refactoring


# b308172d 27-Jul-2010 blanchet <none@none>

minor refactoring


# fb6f46bb 27-Jul-2010 blanchet <none@none>

rename "ATP_Manager" ML module to "Sledgehammer";
more refactoring to come


# e0e5093e 21-Jul-2010 blanchet <none@none>

renamings + only need second component of name pool to reconstruct proofs


# 7ec282ba 28-Jun-2010 blanchet <none@none>

always perform "inline" skolemization, polymorphism or not, Skolem cache or not


# d3a567ff 28-Jun-2010 blanchet <none@none>

always perform relevance filtering on original formulas


# 3df81eb1 25-Jun-2010 blanchet <none@none>

factor out thread creation


# 13912498 25-Jun-2010 blanchet <none@none>

got rid of "respect_no_atp" option, which even I don't use


# 28ffd341 25-Jun-2010 blanchet <none@none>

renamed "Sledgehammer_Fact_Preprocessor" to "Clausifier";
the new name reflects that it's not used only by Sledgehammer (but also by "meson" and "metis") and that it doesn't only clausify facts (but also goals)

--HG--
rename : src/HOL/Tools/Sledgehammer/sledgehammer_fact_preprocessor.ML => src/HOL/Tools/Sledgehammer/clausifier.ML


# 8cc15bec 25-Jun-2010 blanchet <none@none>

further reduce dependencies on "sledgehammer_fact_filter.ML"


# 831a6abc 23-Jun-2010 blanchet <none@none>

killed legacy "neg_clausify" and "clausify"


# 78449191 22-Jun-2010 blanchet <none@none>

removed Sledgehammer's support for the DFG syntax;
this removes 350 buggy lines from Sledgehammer. SPASS 3.5 and above support the TPTP syntax.


# eb75e9ae 11-Jun-2010 blanchet <none@none>

proper polymorphic Skolemization of uncached facts + synchronization of caching and relevance filter


# 562fda8f 05-Jun-2010 blanchet <none@none>

totally bypass Sledgehammer's relevance filter when facts are given using the "(fact1 ... factn)" syntax;
faster and more reliable


# 391e8b7c 04-Jun-2010 blanchet <none@none>

made "clausify" attribute a legacy feature;
seems to have ever only been a debugging feature


# 7394b636 04-Jun-2010 blanchet <none@none>

made "neg_clausify" a legacy feature


# e9152624 04-Jun-2010 blanchet <none@none>

kill active Sledgehammer threads when running minimize, to avoid confusing the user with too much output


# 771d26e8 28-May-2010 blanchet <none@none>

make sure chained facts appear in Isar proofs generated by Sledgehammer -- otherwise the proof won't work


# 7a6b0131 17-May-2010 wenzelm <none@none>

prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
eliminated old-style structure aliases K = Keyword, P = Parse;


# 92b34500 14-May-2010 blanchet <none@none>

renamed options


# e3ae2868 14-May-2010 blanchet <none@none>

renamed two Sledgehammer options


# e8c1430c 14-May-2010 blanchet <none@none>

delect installed ATPs dynamically, _not_ at image built time


# 1e17f9ae 01-May-2010 krauss <none@none>

made sml/nj happy about Sledgehammer and Nitpick (cf. 6f11c9b1fb3e, 3c2438efe224)


# 5408a7f3 28-Apr-2010 blanchet <none@none>

remove Sledgehammer's "sorts" option to annotate variables with sorts in proof;
what we need is smarter type annotations for variables _and_ constants


# c31dba68 27-Apr-2010 blanchet <none@none>

make Sledgehammer more friendly if no subgoal is left


# a1e85a74 27-Apr-2010 blanchet <none@none>

remove "higher_order" option from Sledgehammer -- the "smart" default is good enough


# 372a3b70 26-Apr-2010 blanchet <none@none>

rename options


# 78eff798 25-Apr-2010 blanchet <none@none>

cosmetics


# 23f7b381 25-Apr-2010 blanchet <none@none>

move "neg_clausify" method and "clausify" attribute to "sledgehammer_isar.ML"


# 9f19bd3c 23-Apr-2010 blanchet <none@none>

remove some bloat


# c63aa835 23-Apr-2010 blanchet <none@none>

renamed module "ATP_Wrapper" to "ATP_Systems"


# 057278ac 23-Apr-2010 blanchet <none@none>

move the minimizer to the Sledgehammer directory

--HG--
rename : src/HOL/Tools/ATP_Manager/atp_minimal.ML => src/HOL/Tools/Sledgehammer/sledgehammer_fact_minimizer.ML


# 0f99daf9 23-Apr-2010 blanchet <none@none>

move some sledgehammer stuff out of "atp_manager.ML"


# 37dab216 23-Apr-2010 blanchet <none@none>

move the Sledgehammer menu options to "sledgehammer_isar.ML"


# 2e022e8a 22-Apr-2010 blanchet <none@none>

remove hack that is no longer necessary now that "ATP_Wrapper" properly detects which ATPs are installed


# ce4a26b7 21-Apr-2010 blanchet <none@none>

pass relevant options from "sledgehammer" to "sledgehammer minimize";
one nice side effect of this change is that the "sledgehammer minimize" syntax now only occurs in "sledgehammer_isar.ML", instead of being spread across two files


# cec4748e 20-Apr-2010 blanchet <none@none>

added "explicit_apply" option to Sledgehammer, to control whether an explicit apply function should be used as much or as little as possible (replaces a previous global variable)


# 6e1436fe 19-Apr-2010 blanchet <none@none>

make Sledgehammer's minimizer also minimize Isar proofs


# b2d11c91 19-Apr-2010 blanchet <none@none>

rename Sledgehammer "theory_const" option to "theory_relevant", now that I understand better what it does


# 0fcdd178 16-Apr-2010 blanchet <none@none>

by default, don't try to start ATPs that aren't installed


# f38ad5c5 16-Apr-2010 blanchet <none@none>

fiddle with Sledgehammer option syntax


# 6af6bd76 16-Apr-2010 blanchet <none@none>

Sledgehammer: the empty set of fact () should mean nothing, not unchanged


# f3a1400d 14-Apr-2010 blanchet <none@none>

added "overlord" option (to get easy access to output files for debugging) + systematically use "raw_goal" rather than an inconsistent mixture


# 2c77148c 14-Apr-2010 blanchet <none@none>

make Sledgehammer "minimize" output less confusing + round up (not down) time limits to nearest second


# 87d19471 14-Apr-2010 blanchet <none@none>

make Sledgehammer's "timeout" option work for "minimize"


# 5ca7353b 14-Apr-2010 blanchet <none@none>

fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
and added "atp" as alias for "atps"


# a5f9c697 29-Mar-2010 blanchet <none@none>

added "modulus" and "sorts" options to control Sledgehammer's Isar proof output


# f5482a19 29-Mar-2010 blanchet <none@none>

make Sledgehammer output "by" vs. "apply", "qed" vs. "next", and any necessary "prefer"


# 4ec65078 28-Mar-2010 blanchet <none@none>

made "theory_const" a Sledgehammer option;
by default, it's true for SPASS and false for the others. This eliminates the need for the "spass_no_tc" ATP, which can be obtained by passing "no_theory_const" instead.


# 54f0c16f 28-Mar-2010 blanchet <none@none>

added "respect_no_atp" and "convergence" options to Sledgehammer;
these were previously hard-coded in "sledgehammer_fact_filter.ML"


# faaf4307 28-Mar-2010 blanchet <none@none>

make SML/NJ happy


# ec5fb72d 25-Mar-2010 blanchet <none@none>

make Mirabelle happy again


# 5473633f 24-Mar-2010 blanchet <none@none>

revert debugging output that shouldn't have been submitted in the first place


# 2256a154 23-Mar-2010 blanchet <none@none>

honor the newly introduced Sledgehammer parameters and fixed the parsing;
e.g. the prover "e_isar" (formely "e_full") is gone, instead do sledgehammer [atps = e, isar_proof] to get the same effect


# 99c65b33 23-Mar-2010 blanchet <none@none>

added a syntax for specifying facts to Sledgehammer;
e.g., sledgehammer (add: foo del: bar)
which tells the relevance filter to include "foo" but omit "bar".


# ce60b8a2 23-Mar-2010 blanchet <none@none>

added options to Sledgehammer;
syntax: sledgehammer [options] goal_no, where "[options]" and "goal_no" are optional


# 2a925c70 22-Mar-2010 blanchet <none@none>

make "sledgehammer" and "atp_minimize" improper commands


# 538e54e9 19-Mar-2010 blanchet <none@none>

move the Sledgehammer Isar commands together into one file;
this will make easier to add options and reorganize them later