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

clarified signature;


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

killed final stops in Sledgehammer and friends


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

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


# 369e4785 13-Dec-2015 wenzelm <none@none>

more general types Proof.method / context_tactic;
proper context for Method.insert_tac;
tuned;


# 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


# 63c273c7 01-Jun-2015 haftmann <none@none>

dropped dead config option


# 71c619a0 28-May-2015 blanchet <none@none>

took out Sledgehammer minimizer optimization that breaks things


# 62dbb4e4 03-May-2015 blanchet <none@none>

improved one-line preplaying (don't rely on 'using x by simp' to mean 'by (simp add: x)' and beware of inaccessible '(local.)this')


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

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


# a2f4658a 30-Sep-2014 blanchet <none@none>

don't affect other subgoals with 'auto' in one-liner proofs


# 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


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

going back to bc06471cb7b7 for silencing -- the bad side effects occurred only with 'smt', and the alternative silencing sometimes broke 'auto' etc.


# 85d53264 28-Aug-2014 blanchet <none@none>

moved skolem method


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

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


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

tuned method description


# 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


# 1ec574ba 16-Aug-2014 wenzelm <none@none>

modernized module name and setup;


# 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


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

faster minimization by not adding facts that are already in the simpset


# ddb4eee1 25-Jul-2014 blanchet <none@none>

added missing facts to proof method


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

fine-tuned methods


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


# 61286368 30-Jul-2014 blanchet <none@none>

tuned ML function name


# 76f116e0 24-Jun-2014 blanchet <none@none>

move method silencing code closer to the methods it is trying to silence, to reduce bad side-effects


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

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


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


# fceeffed 15-May-2014 blanchet <none@none>

new approach to silence proof methods, to avoid weird theory/context mismatches


# a088de98 13-May-2014 blanchet <none@none>

transfer theorems since 'silence_methods' may change the theory


# bfa2630b 04-May-2014 blanchet <none@none>

use right meson tactic for preplaying


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

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


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

simplified preplaying information


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

integrate SMT2 with Sledgehammer


# 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


# 89b0d620 13-Feb-2014 blanchet <none@none>

removed hint that is seldom useful in practice


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

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


# 3223eef9 03-Feb-2014 blanchet <none@none>

removed legacy 'metisFT' method


# 5a7cb477 03-Feb-2014 blanchet <none@none>

tuning


# 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