History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Tools/Sledgehammer/sledgehammer.ML
Revision Date Author Comments
# 1d377dcc 21-Jan-2019 blanchet <none@none>

get rid of visibility in MaSh -- it slows it down more than it helps


# c1b7a107 13-Aug-2016 blanchet <none@none>

avoid loading MaSh file first time around for higher responsiveness of Sledgehammer


# 68473ab9 13-Aug-2016 blanchet <none@none>

optimization in MaSh parsing


# f02fe845 13-Aug-2016 blanchet <none@none>

tuned ML


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

killed final stops in Sledgehammer and friends


# 33d34f82 16-Jun-2016 blanchet <none@none>

be more careful before filtering out chained facts in Sledgehammer


# 9d709195 17-May-2016 blanchet <none@none>

proper consideration of chained facts in 'try0' minimization


# d56b4476 27-Mar-2016 blanchet <none@none>

a more generous hard timeout


# b09f23e4 27-Mar-2016 blanchet <none@none>

early warning when Sledgehammer finds a proof


# c8a3ab07 05-Mar-2016 wenzelm <none@none>

tuned signature -- clarified modules;

--HG--
rename : src/Pure/Concurrent/time_limit.ML => src/Pure/Concurrent/timeout.ML


# dccdabe3 03-Mar-2016 wenzelm <none@none>

clarified modules;
tuned signature;


# 456ff485 01-Feb-2016 blanchet <none@none>

preplaying of 'smt' and 'metis' more in sync with actual method


# 5cbf1a62 01-Feb-2016 blanchet <none@none>

preplaying of 'smt' and 'metis' more in sync with actual method


# a99a3743 05-Oct-2015 blanchet <none@none>

further improved fine point w.r.t. replaying in the presence of chained facts and a non-empty meta-quantifier prefix + avoid printing internal names in backquotes


# 0ef6756d 02-Oct-2015 blanchet <none@none>

further reduced dependency on legacy async thread manager


# b72de54b 02-Oct-2015 blanchet <none@none>

removed legacy asynchronous mode in Sledgehammer


# 3716e228 21-Sep-2015 wenzelm <none@none>

clarified markup;
tuned signature;


# 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


# 2147d9b6 22-Jun-2015 blanchet <none@none>

keep 'Pure.all' in goals when preplaying


# 2060d40b 22-Jun-2015 blanchet <none@none>

use right context for preplay, to avoid errors in fact lookup


# 34035ccd 04-Mar-2015 wenzelm <none@none>

tuned signature -- prefer qualified names;


# 3c4cd10c 29-Jan-2015 wenzelm <none@none>

more explicit indication of Async_Manager_Legacy as Proof General legacy;

--HG--
rename : src/HOL/Tools/Sledgehammer/async_manager.ML => src/HOL/Tools/Sledgehammer/async_manager_legacy.ML


# 986c7f6c 23-Dec-2014 wenzelm <none@none>

explicit message channels for "state", "information";
separate state_message_color;


# 13ddea91 26-Nov-2014 wenzelm <none@none>

renamed "pairself" to "apply2", in accordance to @{apply 2};


# c12ca051 07-Nov-2014 wenzelm <none@none>

plain value Keywords.keywords, which might be used outside theory for bootstrap purposes;
plain value Outer_Syntax within theory: parsing requires current theory context;
clarified name of Keyword.is_literal according to its semantics;
eliminated pointless type Keyword.T;
simplified @{command_spec};
clarified bootstrap keywords and syntax: take it as basis instead of side-branch;


# 514ac706 06-Nov-2014 wenzelm <none@none>

prefer explicit Keyword.keywords;


# d29594dd 03-Nov-2014 wenzelm <none@none>

eliminated obsolete Proof.goal_message -- print outcome more directly;


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

discontinued obsolete Output.urgent_message;


# 8b681e9f 30-Sep-2014 blanchet <none@none>

don't call 'hd' on a possibly empty list


# 9ce20114 04-Aug-2014 blanchet <none@none>

default on 'metis' for ATPs if preplaying is disabled


# 7163f726 03-Aug-2014 blanchet <none@none>

more informative preplay failures


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

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


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

honor 'dont_minimize' option when preplaying one-liner proof


# 16ad7b59 14-Jul-2014 blanchet <none@none>

record MaSh algorithm in spying data


# caf1efe8 01-Jul-2014 blanchet <none@none>

tuned message


# 1ea02303 26-Jun-2014 blanchet <none@none>

reintroduced MaSh hints, this time as persistent creatures


# 6ad544a8 26-Jun-2014 blanchet <none@none>

tuned output


# 4df9f9c4 26-Jun-2014 blanchet <none@none>

tuning


# 00e418b3 01-Aug-2014 blanchet <none@none>

export ML function


# 46945d2f 01-Aug-2014 blanchet <none@none>

restored a bit of laziness


# 1ff4ab0e 01-Aug-2014 blanchet <none@none>

further minimize one-liner


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

tuning


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

eliminated needlessly complex message tail


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

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


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

rationalized preplaying by eliminating (now superfluous) laziness


# 07041a99 16-Jun-2014 blanchet <none@none>

moved code around

--HG--
rename : src/HOL/Tools/Sledgehammer/sledgehammer_prover_waldmeister.ML => src/HOL/Tools/ATP/atp_waldmeister.ML


# 7cc77f8f 27-May-2014 blanchet <none@none>

optimized computation


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

properly reconstruct helpers in Z3 proofs


# 59db6ad2 21-May-2014 blanchet <none@none>

shorten Sledgehammer output, as suggested by Andrei Popescu


# 516d4157 21-May-2014 blanchet <none@none>

avoid markup-generating @{make_string}


# 52dd9fc9 27-Mar-2014 wenzelm <none@none>

clarified Isabelle/ML bootstrap, such that Execution does not require ML_Compiler;


# 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


# 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


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

tuning


# 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


# 1c693177 07-Dec-2010 blanchet <none@none>

pass constant arguments to the built-in check function, cf. d2b1fc1b8e19


# 1e323d7a 07-Dec-2010 boehmes <none@none>

centralized handling of built-in types and constants;
also store types and constants which are rewritten during preprocessing;
interfaces are identified by classes (supporting inheritance, at least on the level of built-in symbols);
removed term_eq in favor of type replacements: term-level occurrences of type bool are replaced by type term_bool (only for the translation)


# 1e36dea1 06-Dec-2010 blanchet <none@none>

handle "max_relevant" uniformly


# 2c6ad15f 06-Dec-2010 blanchet <none@none>

honor the default max relevant facts setting from the SMT solvers in Sledgehammer


# 707b76a1 06-Dec-2010 blanchet <none@none>

trust SMT filter's timeout -- nested timeouts seem to be at the origin of spontaneous Interrupt exceptions in some cases


# 6cdca956 06-Dec-2010 blanchet <none@none>

reraise interrupt exceptions


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

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


# ac8f79ef 26-Nov-2010 blanchet <none@none>

put facts found by SMT solver in alphabetical order and omit chained facts, as was done already for ATP proofs


# d579fd68 26-Nov-2010 blanchet <none@none>

adjust Sledgehammer/SMT fudge factor


# 51bbe234 25-Nov-2010 blanchet <none@none>

cosmetics


# 3021c7a9 25-Nov-2010 blanchet <none@none>

set Metis option on correct context, lest it be ignored


# b6668c77 24-Nov-2010 blanchet <none@none>

make "debug" mode of Sledgehammer/SMT more liberal


# 693dce2d 24-Nov-2010 blanchet <none@none>

more precise error handling in Sledgehammer/SMT for Z3 and remote SMT provers


# 44bf3323 23-Nov-2010 blanchet <none@none>

more precise error handling for Z3;
refactored some of the error handling code shared by ATP and SMT


# 964895f2 23-Nov-2010 blanchet <none@none>

use "Thm.transfer" in Sledgehammer to prevent theory merger issues in "SMT_Solver.smt_filter" later on


# 2c3aca6a 23-Nov-2010 blanchet <none@none>

try Metis to reconstruct SMT proofs, to increase success rate and reduce dependency on (often remote) SMT solvers or certificates


# 14e6bac1 19-Nov-2010 wenzelm <none@none>

renamed raw "explode" function to "raw_explode" to emphasize its meaning;


# f46b6402 15-Nov-2010 boehmes <none@none>

renamed SMT failure: Abnormal_Termination is indeed more appropriate than Solver_Crashed


# bccf10ef 15-Nov-2010 blanchet <none@none>

better error message


# d40d8ba7 15-Nov-2010 blanchet <none@none>

better error message


# bb58d249 15-Nov-2010 blanchet <none@none>

cosmetics


# 69cc8147 15-Nov-2010 blanchet <none@none>

interpret SMT_Failure.Solver_Crashed correctly


# 97b69cf7 15-Nov-2010 blanchet <none@none>

pick up SMT solver crashes and report them to the user/Mirabelle if desired


# 3166c63c 10-Nov-2010 blanchet <none@none>

make SML/NJ happy


# 4b0faf2e 08-Nov-2010 blanchet <none@none>

reduce the number of monomorphization iterations from 10 (the default) to 4, in the interest of faster SMT solving


# bf286a01 08-Nov-2010 blanchet <none@none>

compile -- 7550b2cba1cb broke the build


# b1d1d667 07-Nov-2010 boehmes <none@none>

better modularization: moved SMT configuration options and diagnostics as well as SMT failure and exception into separate structures (both of which are loaded first and consequently are available to other SMT structures)


# f0e8233f 07-Nov-2010 blanchet <none@none>

make sure the SMT solver runs several iterations by lowering the timeout at each iteration -- yields better results in practice


# 56e2c8ea 07-Nov-2010 blanchet <none@none>

always use a hard timeout in Mirabelle


# 1736d471 07-Nov-2010 blanchet <none@none>

don't pass too many facts on the first iteration of the SMT solver


# 8589ee0a 07-Nov-2010 blanchet <none@none>

catch TimeOut exception


# c5ff20f2 07-Nov-2010 blanchet <none@none>

ensure the SMT solver respects the timeout -- Mirabelle revealed cases where "smt_filter" apparently never returns


# 778b3ad1 07-Nov-2010 blanchet <none@none>

if SMT used as a filter in a loop fails at each iteration, returns the first error, not the last, since it is more informative -- the first error typically says "out of memory", whereas the last might well be "the SMT problem is unprovable", which should be no surprise if too many facts were removed


# c7dfdec9 06-Nov-2010 blanchet <none@none>

invoke SMT solver in a loop, with fewer and fewer facts, in case of error


# e2031cff 04-Nov-2010 blanchet <none@none>

cosmetics


# ab2ab2bb 04-Nov-2010 blanchet <none@none>

use the SMT integration's official list of built-ins


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

standardize on seconds for Nitpick and Sledgehammer timeouts


# 9d0210b4 28-Oct-2010 blanchet <none@none>

clear identification;
thread "Auto S/H" (vs. manual S/H) setting through SMT


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

adapted SMT solver error handling to reflect latest changes in "SMT_Solver"


# 68a022b8 26-Oct-2010 blanchet <none@none>

better list of irrelevant SMT constants


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

if "debug" is on, print list of relevant facts (poweruser request);
internal renaming


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

standardize on "fact" terminology (vs. "axiom" or "theorem") in Sledgehammer -- but keep "Axiom" in the lower-level "ATP_Problem" module


# fbc7a0f9 26-Oct-2010 boehmes <none@none>

capture out-of-memory warnings of Z3 and turn them into proper exceptions; be more precise about SMT solver run-time: return NONE instead of ~1


# 8eaee23c 26-Oct-2010 blanchet <none@none>

remove needless context argument;
prefer "Proof.context_of" to "#context o Proof.goal", since it considers any "using [[...]]"


# 3be283af 26-Oct-2010 blanchet <none@none>

tuning


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

proper error handling for SMT solvers in Sledgehammer


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

integrated "smt" proof method with Sledgehammer


# 93623054 25-Oct-2010 wenzelm <none@none>

renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;


# 1889b149 22-Oct-2010 blanchet <none@none>

tuning


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

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


# 0a9b4097 22-Oct-2010 blanchet <none@none>

generalized the relevance filter so that it takes the list of "irrelevant constants" as argument (since the ATP and SMT preprocessing are different)


# 34e96e6a 22-Oct-2010 blanchet <none@none>

replaced references with proper record that's threaded through


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

fixed signature of "is_smt_solver_installed";
renaming


# 11b9c001 22-Oct-2010 blanchet <none@none>

renamed modules


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

remove more needless code ("run_smt_solvers");
tuning


# 4092d4d5 21-Oct-2010 blanchet <none@none>

got rid of duplicate functionality ("run_smt_solver_somehow");
added minimization command to SMT solver message


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

bring ATPs and SMT solvers more in line with each other


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

make Sledgehammer minimizer fully work with SMT


# 1db1f4c7 22-Oct-2010 blanchet <none@none>

generalization of the Sledgehammer minimizer, to make it possible to handle SMT solvers as well


# 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 ..."


# d86baa55 16-Sep-2010 blanchet <none@none>

rename "Metis_Clauses" to "Metis_Translate" for consistency with "Sledgehammer_Translate"

--HG--
rename : src/HOL/Tools/Sledgehammer/metis_clauses.ML => src/HOL/Tools/Sledgehammer/metis_translate.ML


# a4a148d4 16-Sep-2010 blanchet <none@none>

move SPASS's Flotter hack to "Sledgehammer_Reconstruct"


# b1fc4845 16-Sep-2010 blanchet <none@none>

skip some "important" messages


# 5bfe22d9 16-Sep-2010 blanchet <none@none>

refactoring: move ATP proof and error extraction code to "ATP_Proof" module


# 186f4197 16-Sep-2010 blanchet <none@none>

use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs


# acf1190a 16-Sep-2010 blanchet <none@none>

factored out TSTP/SPASS/Vampire proof parsing;
from "Sledgehammer_Reconstructo" to a new module "ATP_Proof"


# 60986191 14-Sep-2010 blanchet <none@none>

finish support for E 1.2 proof reconstruction;
this involves picking up the axiom and conjecture names specified using a "file" annotation in the TSTP file, since we cannot rely anymore on formula numbers (E 1.2 adds a strange offset)


# 457efa51 14-Sep-2010 blanchet <none@none>

clarify message


# f2fad0c9 14-Sep-2010 blanchet <none@none>

use same hack as in "Async_Manager" to work around Proof General bug


# 4c134944 14-Sep-2010 blanchet <none@none>

handle relevance filter corner cases more gracefully;
e.g. the minimizer selects 15 facts but "max_relevant = 14"


# 7ab0dafa 14-Sep-2010 blanchet <none@none>

Sledgehammer should be called in "prove" mode;
otherwise the proof text won't fit into the proof document


# 06279c2b 13-Sep-2010 blanchet <none@none>

tuning


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

tuning


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

implemented Auto Sledgehammer


# 62f95125 09-Sep-2010 blanchet <none@none>

more precise error messages when Vampire is interrupted or SPASS runs into an internal bug


# ae1f86fe 09-Sep-2010 blanchet <none@none>

better error reporting when the Sledgehammer minimizer is interrupted


# 93226bb2 06-Sep-2010 blanchet <none@none>

use Future.fork rather than Thread.fork, so that the thread is part of the global thread management


# 00768c9e 06-Sep-2010 wenzelm <none@none>

some results of concurrency code inspection;


# a837a32a 02-Sep-2010 blanchet <none@none>

show the number of facts for each prover in "verbose" mode


# 9d0f2737 02-Sep-2010 blanchet <none@none>

make sure "Unknown ATP" errors reach the users -- i.e. don't generate them from a thread


# ef752320 02-Sep-2010 blanchet <none@none>

If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user


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

show real CPU time


# 14a59fde 01-Sep-2010 blanchet <none@none>

factor out code shared by all ATPs so that it's run only once


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

handle all whitespace, not just ASCII 32


# 2504321e 01-Sep-2010 blanchet <none@none>

speed up SPASS hack + output time information in "blocking" mode


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

minor refactoring


# 035d5dfa 01-Sep-2010 blanchet <none@none>

translate the axioms to FOF once and for all ATPs


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

run relevance filter in a thread, to avoid blocking


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

only kill ATP threads in nonblocking mode


# 502ede9f 01-Sep-2010 blanchet <none@none>

share the relevance filter among the provers


# 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


# 879a8326 31-Aug-2010 blanchet <none@none>

rename sledgehammer config attributes


# 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


# 69934840 30-Aug-2010 blanchet <none@none>

remove useless var


# 34a4355e 30-Aug-2010 blanchet <none@none>

remove needless parameter


# f33285ae 26-Aug-2010 blanchet <none@none>

improve SPASS hack, when a clause comes from several facts


# 0737a633 26-Aug-2010 blanchet <none@none>

consider "locality" when assigning weights to facts


# 6245c17e 25-Aug-2010 blanchet <none@none>

renaming


# 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"


# 433b4150 24-Aug-2010 blanchet <none@none>

make sure that "undo_ascii_of" is the inverse of "ascii_of", also for non-printable characters -- and avoid those in ``-style facts


# be951c03 24-Aug-2010 blanchet <none@none>

clean handling of whether a fact is chained or not;
more elegant and reliable than encoding it in the name


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

weed out junk in relevance filter


# fe59c4c4 22-Aug-2010 blanchet <none@none>

be more generous towards SPASS's -SOS mode


# b0a48d28 22-Aug-2010 blanchet <none@none>

prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
the disjunctive view of "conjecture" is nonstandard but taken by E, SPASS, Vampire, etc.


# 780ac17f 19-Aug-2010 blanchet <none@none>

tuning


# b1f5cb20 19-Aug-2010 blanchet <none@none>

no spurious trailing "\n" at the end of Sledgehammer's output


# 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


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

improve SPASS clause numbering hack


# 781ea295 16-Aug-2010 blanchet <none@none>

more debug output


# 8493de05 09-Aug-2010 blanchet <none@none>

prevent ATP thread for staying around for 1 minute if an exception occurred earlier;
this is a workaround for what could be a misfeature of "Async_Manager", which I'd rather not touch


# 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


# 52314483 09-Aug-2010 blanchet <none@none>

reintroduced old code that removed axioms from the conjecture assumptions, ported to FOF


# 3e58b9bc 09-Aug-2010 blanchet <none@none>

fix embarrassing bug in elim rule handling, introduced during the port to FOF


# 8cd67f76 04-Aug-2010 blanchet <none@none>

fix bug in Nitpick's "equationalize" function (the prems were ignored) + make it do some basic extensionalization


# 8ca17258 29-Jul-2010 blanchet <none@none>

don't choke on synonyms when parsing SPASS's Flotter output + renamings;
the output format isn't documented so it was hard to guess that a single clause could be associated with several names...


# f78a86f3 29-Jul-2010 blanchet <none@none>

fix bug in the newly introduced "bound concealing" code


# 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


# 6bffdf24 29-Jul-2010 blanchet <none@none>

handle schematic vars the same way in Sledgehammer as in Metis, to avoid unreplayable proofs


# 64a835a2 29-Jul-2010 blanchet <none@none>

speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"


# b2451d37 29-Jul-2010 blanchet <none@none>

work around atomization failures


# 62dd96e3 29-Jul-2010 blanchet <none@none>

perform the presimplification done by Metis.make_nnf in Sledgehammer again, to deal with "If" and similar constructs


# a66df725 29-Jul-2010 blanchet <none@none>

fix bug with "=" vs. "fequal" introduced by last change (dddb8ba3a1ce)


# f72671b0 29-Jul-2010 blanchet <none@none>

generate correct names for "$true" and "$false";
this was lost somewhere in the non-clausification


# c41a6765 29-Jul-2010 blanchet <none@none>

don't assume canonical rule format


# 7ab2cc25 29-Jul-2010 blanchet <none@none>

avoid "clause" and "cnf" terminology where it no longer makes sense


# 67e38df5 29-Jul-2010 blanchet <none@none>

"axiom_clauses" -> "axioms" (these are no longer clauses)


# bfadabe5 29-Jul-2010 blanchet <none@none>

remove the "extra_clauses" business introduced in 19a5f1c8a844;
it isn't working reliably because of:
* relevance_override
* it is ignored anyway by TPTP generator
A better solution would/will be to ensure monotonicity: extra axioms not used in an ATP proof shouldn't make the rest of the problem provable


# 4ed00612 28-Jul-2010 blanchet <none@none>

handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on


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

minor refactoring


# d1cad83e 28-Jul-2010 blanchet <none@none>

fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses


# db077e64 28-Jul-2010 blanchet <none@none>

revive "e" and "remote_e"'s fact extraction so that it works with E 1.2 as well;
we can no longer just count the formulas, because for some reason E's numbering either no longer starts at 1 or it doesn't increment by 1 at each step


# 5c51681a 28-Jul-2010 blanchet <none@none>

renaming


# 85f0e925 27-Jul-2010 blanchet <none@none>

improve detection of installed SPASS


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

minor refactoring


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

more refactoring


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

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


# 3f2e18c0 27-Jul-2010 blanchet <none@none>

rename

--HG--
rename : src/HOL/Tools/ATP_Manager/atp_manager.ML => src/HOL/Tools/Sledgehammer/sledgehammer.ML