src/HOL/SMT.thy
Wed, 30 Sep 2020 18:37:22 +0200 desharna Effectively disable timeout for smt method/tactic
Sun, 06 Jan 2019 15:04:34 +0100 wenzelm isabelle update -u path_cartouches;
Tue, 30 Oct 2018 16:24:04 +0100 fleury add reconstruction by veriT in method smt
Tue, 30 Oct 2018 16:24:01 +0100 fleury split SMT reconstruction into library
Mon, 24 Sep 2018 14:30:09 +0200 nipkow Prefix form of infix with * on either side no longer needs special treatment
Wed, 11 Apr 2018 10:59:13 +0200 boehmes avoid adding unnecessary quantified lemmas when embedding natural number terms into integer terms: quantified lemmas can cause Z3 to produce complex proofs that are hard to replay in Isabelle
Wed, 10 Jan 2018 15:25:09 +0100 nipkow ran isabelle update_op on all sources
Sun, 26 Nov 2017 21:08:32 +0100 wenzelm more symbols;
Sun, 08 Oct 2017 22:28:22 +0200 haftmann euclidean rings need no normalization
Wed, 30 Aug 2017 23:36:21 +0200 blanchet added options to make veriT more complete
Tue, 29 Aug 2017 18:30:23 +0200 blanchet towards support for HO SMT-LIB
Thu, 03 Aug 2017 23:43:17 +0200 blanchet pass option recommended by Andy Reynolds to CVC4 1.5 (released) or better
Fri, 28 Jul 2017 15:36:32 +0100 blanchet introduced option for nat-as-int in SMT
Mon, 07 Dec 2015 10:38:04 +0100 wenzelm isabelle update_cartouches -c -t;
Tue, 10 Nov 2015 23:41:20 +0100 wenzelm recovered from a9c0572109af;
Tue, 10 Nov 2015 17:49:54 +0100 fleury fixing premises in veriT proof reconstruction
Sat, 18 Jul 2015 22:58:50 +0200 wenzelm isabelle update_cartouches;
Sat, 25 Apr 2015 09:48:06 +0200 blanchet made CVC4 support work also without unsat cores
Wed, 08 Apr 2015 18:47:38 +0200 blanchet updated SMT module and Sledgehammer to fully open source Z3
Fri, 16 Jan 2015 23:23:31 +0100 boehmes more efficient Z3 proof reconstruction for rewrite steps with conjunctions and disjunctions, similar to Old_SMT
Mon, 24 Nov 2014 12:35:13 +0100 blanchet added one more CVC4 option that helps Judgment Day (10 theory version)
Mon, 24 Nov 2014 12:35:13 +0100 blanchet added Z3 reconstruction rule suggested by F. Maric
Mon, 24 Nov 2014 12:35:13 +0100 blanchet one more CVC4 option that helps
Mon, 24 Nov 2014 12:35:13 +0100 blanchet renamed 'veriT' to 'verit', to stick to all-lowercase rule for prover names
Thu, 20 Nov 2014 17:29:18 +0100 blanchet added CVC4 option that helps on JD
Thu, 20 Nov 2014 17:29:18 +0100 blanchet removed explicit '--quant-cf' option to CVC4, now that it's the default
Wed, 19 Nov 2014 10:31:15 +0100 blanchet parse CVC4 unsat cores
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Fri, 24 Oct 2014 15:07:51 +0200 hoelzl use NO_MATCH-simproc for distribution rules in field_simps, otherwise field_simps on '(a / (c + d)) * (e + f)' can be non-terminating
Mon, 06 Oct 2014 19:19:16 +0200 blanchet strengthened 'moura' method
Mon, 29 Sep 2014 14:32:30 +0200 blanchet made 'moura' tactic more powerful
Thu, 25 Sep 2014 13:30:57 +0200 blanchet added useful options to CVC4
Wed, 17 Sep 2014 16:53:39 +0200 blanchet added interface for CVC4 extensions
Thu, 28 Aug 2014 16:58:26 +0200 blanchet tuned method description
Thu, 28 Aug 2014 00:40:38 +0200 blanchet renamed new SMT module from 'SMT2' to 'SMT'
Sat, 16 Aug 2014 18:31:47 +0200 wenzelm updated to named_theorems;
Thu, 12 Jun 2014 01:00:49 +0200 blanchet reduces Sledgehammer dependencies
Thu, 12 Jun 2014 01:00:49 +0200 blanchet tuning
Thu, 12 Jun 2014 01:00:49 +0200 blanchet use 'ctr_sugar' abstraction in SMT(2)
Wed, 11 Jun 2014 11:28:46 +0200 blanchet fixed unsoundness in SMT(2) as oracle: don't register typedef Abs_x as constructor unless it is known to be injective
Thu, 13 Mar 2014 13:18:13 +0100 blanchet moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
Tue, 11 Mar 2014 15:34:38 +0100 blanchet full path
Sun, 19 Jan 2014 22:38:17 +0100 boehmes removed obsolete remote_cvc3 and remote_z3
Mon, 13 Jan 2014 20:20:44 +0100 wenzelm activation of Z3 via "z3_non_commercial" system option (without requiring restart);
Mon, 03 Dec 2012 16:07:28 +0100 wenzelm synchronized read access to cache file -- avoid potential conflict with ongoing write (which is non-atomic);
Wed, 22 Aug 2012 23:22:57 +0200 wenzelm prefer ML_file over old uses;
Mon, 23 Apr 2012 21:44:36 +0200 wenzelm more standard method setup;
Tue, 27 Mar 2012 16:59:13 +0300 blanchet renamed "smt_fixed" to "smt_read_only_certificates"
Thu, 15 Mar 2012 22:08:53 +0100 wenzelm declare command keywords via theory header, including strict checking outside Pure;
Mon, 07 Nov 2011 17:54:35 +0100 boehmes replace higher-order matching against schematic theorem with dedicated reconstruction method
Thu, 25 Aug 2011 11:15:31 +0200 boehmes improved completeness and efficiency of Z3 proof reconstruction, especially by an improved handling of Skolemization
Tue, 09 Aug 2011 09:05:21 +0200 blanchet load lambda-lifting structure earlier, so it can be used in Metis
Wed, 20 Jul 2011 12:23:20 +0200 boehmes generalized lambda-lifting such that it is less specifically tailored for SMT (it does not anymore dependent on any SMT-specific code)
Wed, 20 Jul 2011 09:23:12 +0200 boehmes moved lambda-lifting on terms into a separate structure (for better re-use in tools other than SMT)
Wed, 20 Jul 2011 09:23:09 +0200 boehmes removed old (unused) SMT monomorphizer
Tue, 07 Jun 2011 10:24:16 +0200 boehmes clarified meaning of monomorphization configuration option by renaming it
Mon, 14 Feb 2011 12:25:26 +0100 boehmes limit the number of generated SMT monomorphization instances (in addition to the existing monomorphization limit which does not prevent seemingly infinite loops);
Mon, 17 Jan 2011 17:45:52 +0100 boehmes made Z3 the default SMT solver again
Fri, 07 Jan 2011 17:58:51 +0100 boehmes tuned text
Fri, 07 Jan 2011 15:39:13 +0100 boehmes added hints about licensing restrictions and how to enable Z3
less more (0) -60 tip