History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Tools/SMT/smt_config.ML
Revision Date Author Comments
# 7110473f 30-Oct-2018 fleury <Mathias.Fleury@mpi-inf.mpg.de>

add reconstruction by veriT in method smt


# 99e3d4c3 06-Dec-2017 wenzelm <none@none>

prefer control symbol antiquotations;


# 9a20f33d 01-Oct-2017 blanchet <none@none>

properly take quantifiers into account (cf. my Ph.D. thesis, Section 6.4.1) and offer three modes of completeness (for experiments mostly)


# f9beda92 29-Aug-2017 blanchet <none@none>

towards support for HO SMT-LIB


# 1d8a8be4 28-Jul-2017 blanchet <none@none>

introduced option for nat-as-int in SMT


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

tuned signature -- clarified modules;

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


# 61f869f4 30-May-2015 wenzelm <none@none>

tuned message;


# 4aa541f4 06-Apr-2015 wenzelm <none@none>

@{command_spec} is superseded by @{command_keyword};


# b8aa512a 29-Dec-2014 boehmes <none@none>

optionally display statistics for Z3 proof reconstruction


# 6bf1de71 29-Dec-2014 boehmes <none@none>

avoid more than one data slot per module


# a4bf9b76 29-Dec-2014 boehmes <none@none>

limit reconstruction time of Z3 proof steps to be able to detect long-running reconstruction steps


# 7ee8e540 03-Nov-2014 wenzelm <none@none>

eliminated unused int_only flag (see also c12484a27367);
just proper commands;


# 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


# b6e6a472 26-Mar-2014 wenzelm <none@none>

prefer Context_Position where a context is available;
prefer explicit Context_Position.is_visible -- avoid redundant message composition;
tuned signature;


# 7216e79c 18-Mar-2014 wenzelm <none@none>

clarifed module name;

--HG--
rename : src/Pure/Thy/thy_load.ML => src/Pure/PIDE/resources.ML
rename : src/Pure/Thy/thy_load.scala => src/Pure/PIDE/resources.scala
rename : src/Tools/jEdit/src/jedit_thy_load.scala => src/Tools/jEdit/src/jedit_resources.scala


# 9bc2d09b 02-Oct-2013 blanchet <none@none>

make SMT integration slacker w.r.t. bad apples (facts)


# 7d59a5d8 18-Jul-2013 wenzelm <none@none>

tuned signature;


# 59410e28 09-Apr-2013 wenzelm <none@none>

discontinued Toplevel.no_timing complication -- also recovers timing of diagnostic commands, e.g. 'find_theorems';
print timing as tracing, to keep it out of the way in Proof General;
no timing of control commands, especially relevant for Proof General;


# e26a601f 28-Mar-2013 boehmes <none@none>

new, simpler implementation of monomorphization;
old monomorphization code is still available as Legacy_Monomorphization;
modified SMT integration to use the new monomorphization code


# b5be22e7 03-Dec-2012 wenzelm <none@none>

synchronized read access to cache file -- avoid potential conflict with ongoing write (which is non-atomic);
clarified signature -- cache init is unsynchronized and hopefully used at most once per file;


# 3abd2838 30-May-2012 boehmes <none@none>

introduced option "z3_with_extensions" to control whether Z3's support for nonlinear arithmetic and datatypes should be enabled (including potential proof reconstruction failures)


# b24a20db 27-Mar-2012 blanchet <none@none>

renamed "smt_fixed" to "smt_read_only_certificates"


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


# b173aaef 29-Feb-2012 boehmes <none@none>

SMT fails if the chosen SMT solver is not installed


# 61c3b64e 29-Dec-2011 wenzelm <none@none>

comments;


# 247df2ed 02-May-2011 wenzelm <none@none>

added Attrib.setup_config_XXX conveniences, with implicit setup of the background theory;
proper name bindings;


# c15b6e59 01-Apr-2011 boehmes <none@none>

make configuration of (SMT) full monomorphization more flexible: turn boolean argument into a configuration option


# 79efc702 13-Mar-2011 wenzelm <none@none>

Path.print is the official way to show file-system paths to users -- note that Path.implode often indicates violation of the abstract datatype;


# 54cdd3ea 13-Feb-2011 boehmes <none@none>

limit the number of generated SMT monomorphization instances (in addition to the existing monomorphization limit which does not prevent seemingly infinite loops);
updated SMT certificate


# 436f6b2f 14-Feb-2011 boehmes <none@none>

more explicit errors to inform users about problems related to SMT solvers;
fall back to remote SMT solver (if local version does not exist);
extend the Z3 proof parser to accommodate for slight changes introduced by Z3 2.18


# 97038484 10-Jan-2011 boehmes <none@none>

be more precise: also merge option values


# bdde754c 10-Jan-2011 boehmes <none@none>

only print warning in a visible context (previously, the warning was printed more than once)


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

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


# dc8334f2 07-Jan-2011 boehmes <none@none>

shortened the warning about uninstalled SMT solvers (the additional hint might get obsolete without further notice)


# 75a79ce2 07-Jan-2011 boehmes <none@none>

made SML/NJ happy


# 5dd62dd8 06-Jan-2011 boehmes <none@none>

differentiate between local and remote SMT solvers (e.g., "z3" vs. "remote_z3");
turned individual SMT solvers into components;
made CVC3 the default SMT solver (Z3 is licensed as "non-commercial only");
tuned smt_filter interface


# a6d5970d 15-Dec-2010 boehmes <none@none>

added option to enable trigger inference;
better documentation of triggers and SMT available options


# 4b0c0402 15-Dec-2010 boehmes <none@none>

moved SMT classes and dictionary functions to SMT_Utils


# 681fd023 15-Dec-2010 boehmes <none@none>

added option to modify the random seed of SMT solvers


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


# 981e2ce7 17-Nov-2010 boehmes <none@none>

keep input and output files used to communicate with the SMT solver (for debugging purposes mainly)


# e7b46e12 12-Nov-2010 boehmes <none@none>

look for certificates relative to the theory


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