History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML
Revision Date Author Comments
# 438cc573 20-Aug-2019 wenzelm <none@none>

clarified signature;


# 4bad625f 03-Jun-2019 wenzelm <none@none>

clarified signature;


# 038835b6 11-Jan-2018 wenzelm <none@none>

uniform use of Standard ML op-infix -- eliminated warnings;


# a7ccdf43 10-Jan-2018 nipkow <none@none>

ran isabelle update_op on all sources


# 51bb5ca6 06-Jun-2017 wenzelm <none@none>

discontinued obsolete print mode;


# 56cc5262 30-Nov-2015 blanchet <none@none>

avoid 'hence' and 'thus' in generated proofs


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


# 5e0c92af 29-Sep-2014 blanchet <none@none>

make sure no '__' suffixes make it until Isar proof


# 9c7aa39b 29-Sep-2014 blanchet <none@none>

rename skolem symbols in the negative case as well


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

use 'thesis' only if it expands to the right thing (it won't after an 'unfolding', for example)


# 944e83de 28-Aug-2014 blanchet <none@none>

generate 'thesis' variable in Sledgehammer Isar proofs


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

three-line 'obtain' format for generated Isar proofs


# 159b1272 27-Aug-2014 blanchet <none@none>

reintroduced two-line-per-inference Isar proof format


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

tuned skolemization


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

rationalize Skolem names


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

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


# 373e2f6e 25-Jul-2014 blanchet <none@none>

more robustness in Isar proof construction


# a59965f9 24-Jul-2014 blanchet <none@none>

introduce fact chaining also under first step


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

better handling of variable names


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

nicer generated variable names


# 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


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

basic setup for zipperposition prover


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


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

integrate SMT2 with Sledgehammer


# 71a89b87 03-Feb-2014 blanchet <none@none>

don't lose additional outcomes


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

generate comments in Isar proofs


# 0b0225ca 03-Feb-2014 blanchet <none@none>

refactor relabeling code


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

tuned data structure


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

tuned data structure


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

more flexible compression, choosing whichever proof method works


# 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


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

merged 'reconstructors' and 'proof methods'


# 2bd828a3 03-Feb-2014 blanchet <none@none>

added 'smt' as a proof method


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

tuning


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

more data structure rationalization


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

rationalized threading of 'metis' arguments


# 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


# 02e01d58 31-Jan-2014 blanchet <none@none>

tuning


# 270a8909 31-Jan-2014 blanchet <none@none>

more concise Isar output


# 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