Wed, 31 Oct 2012 11:23:21 +0100 |
blanchet |
soft SMT timeout
|
file |
diff |
annotate
|
Wed, 15 Feb 2012 23:19:30 +0100 |
wenzelm |
renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in conformance with similar operations in structure Term and Logic;
|
file |
diff |
annotate
|
Tue, 14 Feb 2012 19:18:57 +0100 |
wenzelm |
normalized aliases;
|
file |
diff |
annotate
|
Mon, 07 Nov 2011 17:54:38 +0100 |
boehmes |
try different alternatives in discharging extra assumptions when schematic theorems obtained from lambda-lifting can be instantiated in different ways
|
file |
diff |
annotate
|
Mon, 07 Nov 2011 17:54:35 +0100 |
boehmes |
replace higher-order matching against schematic theorem with dedicated reconstruction method
|
file |
diff |
annotate
|
Fri, 28 Oct 2011 23:41:16 +0200 |
wenzelm |
tuned Named_Thms: proper binding;
|
file |
diff |
annotate
|
Mon, 12 Sep 2011 07:55:43 +0200 |
nipkow |
new fastforce replacing fastsimp - less confusing name
|
file |
diff |
annotate
|
Thu, 25 Aug 2011 11:15:31 +0200 |
boehmes |
improved completeness and efficiency of Z3 proof reconstruction, especially by an improved handling of Skolemization
|
file |
diff |
annotate
|
Mon, 08 Aug 2011 17:23:15 +0200 |
wenzelm |
misc tuning -- eliminated old-fashioned rep_thm;
|
file |
diff |
annotate
|
Mon, 18 Jul 2011 18:52:52 +0200 |
boehmes |
allow rules with premises to be declared as z3_rule (to circumvent incompleteness of Z3 proof reconstruction)
|
file |
diff |
annotate
|
Thu, 26 May 2011 22:02:40 +0200 |
boehmes |
iteratively deepen abstractions to avoid rare Z3 proof reconstruction failures, e.g. when pulling if-then-else from below uninterpreted constants (suggested by Jasmin Christian Blanchette)
|
file |
diff |
annotate
|
Fri, 13 May 2011 22:55:00 +0200 |
wenzelm |
proper Proof.context for classical tactics;
|
file |
diff |
annotate
|
Sat, 16 Apr 2011 16:15:37 +0200 |
wenzelm |
modernized structure Proof_Context;
|
file |
diff |
annotate
|
Fri, 08 Apr 2011 19:04:08 +0200 |
boehmes |
corrected order of steps in Z3 proof reconstruction for elimination of unused quantified variables: first try to eliminate unused variables, then skip over used variables
|
file |
diff |
annotate
|
Fri, 01 Apr 2011 15:49:19 +0200 |
boehmes |
save reflexivity steps in discharging Z3 Skolemization hypotheses
|
file |
diff |
annotate
|
Fri, 01 Apr 2011 12:16:41 +0200 |
boehmes |
re-implemented proof reconstruction for Z3 skolemization: do not explicitly construct definitions for Skolem constants, and let higher-order resolution do most of the work in the end
|
file |
diff |
annotate
|
Wed, 09 Mar 2011 21:40:38 +0100 |
boehmes |
finished and tested Z3 proof reconstruction for injective functions;
|
file |
diff |
annotate
|
Mon, 03 Jan 2011 16:22:08 +0100 |
boehmes |
re-implemented support for datatypes (including records and typedefs);
|
file |
diff |
annotate
|
Mon, 20 Dec 2010 22:02:57 +0100 |
boehmes |
avoid ML structure aliases (especially single-letter abbreviations)
|
file |
diff |
annotate
|
Wed, 15 Dec 2010 16:29:56 +0100 |
boehmes |
the functions term_of and prop_of are also needed in earlier stages, not only for Z3 proof reconstruction, so they really belong in SMT_Utils
|
file |
diff |
annotate
|
Wed, 15 Dec 2010 10:12:48 +0100 |
boehmes |
fixed proof reconstruction for lambda-lifted problems (which broke when the lambda-lifting code was changed to operate on terms instead of on theorems)
|
file |
diff |
annotate
|
Wed, 15 Dec 2010 10:12:48 +0100 |
boehmes |
adapted the Z3 proof parser to recent changes in Z3's proof format;
|
file |
diff |
annotate
|
Wed, 15 Dec 2010 10:12:44 +0100 |
boehmes |
re-implemented eta-expansion, lambda-lifting, and explicit application on terms (exploiting the control over the term structure);
|
file |
diff |
annotate
|
Wed, 24 Nov 2010 10:39:58 +0100 |
boehmes |
be more precise: only treat constant 'distinct' applied to an explicit list as built-in
|
file |
diff |
annotate
|
Wed, 24 Nov 2010 08:51:48 +0100 |
boehmes |
be more liberal in reconstructing congruences from Z3 (sometimes the symmetric version of a premise is needed)
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 23:37:00 +0100 |
boehmes |
added support for quantifier weight annotations
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 15:45:43 +0100 |
boehmes |
share and use more utility functions;
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 15:45:42 +0100 |
boehmes |
added prove reconstruction for injective functions;
|
file |
diff |
annotate
|
Wed, 17 Nov 2010 08:14:56 +0100 |
boehmes |
use the const antiquotation for constants (this checks that the constant is declared, whereas the more general term antiquotation treats undeclared names as free variable)
|
file |
diff |
annotate
|
Fri, 12 Nov 2010 15:56:11 +0100 |
boehmes |
preliminary support for newer versions of Z3
|
file |
diff |
annotate
|
Mon, 08 Nov 2010 12:13:44 +0100 |
boehmes |
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)
|
file |
diff |
annotate
|
Fri, 29 Oct 2010 18:17:04 +0200 |
boehmes |
introduced SMT.distinct as a representation of the solvers' built-in predicate; check that SMT.distinct is always applied to an explicit list
|
file |
diff |
annotate
|
Tue, 26 Oct 2010 11:49:23 +0200 |
boehmes |
added a mode to only filter assumptions used in a Z3 proof (in which no proof reconstruction is performed)
|
file |
diff |
annotate
|
Tue, 26 Oct 2010 11:45:12 +0200 |
boehmes |
joined setup of SMT solvers in one place; turned Z3-specific options into SMT options (renamed configuration options from z3_* to smt_*); more detailed SMT exception; improved SMT filter interface
|
file |
diff |
annotate
|
Tue, 26 Oct 2010 11:39:26 +0200 |
boehmes |
keep track of theorems initially given to SMT (even if they are rewritten); provide interface to filter theorems necessary for SMT proofs
|
file |
diff |
annotate
|
Mon, 20 Sep 2010 16:05:25 +0200 |
wenzelm |
renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
|
file |
diff |
annotate
|
Wed, 01 Sep 2010 15:33:59 +0200 |
haftmann |
replaced Table.map' by Table.map
|
file |
diff |
annotate
|
Fri, 27 Aug 2010 10:56:46 +0200 |
haftmann |
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
|
file |
diff |
annotate
|
Wed, 26 May 2010 17:52:32 +0200 |
boehmes |
try logical and theory abstraction before full abstraction (avoids warnings of linarith)
|
file |
diff |
annotate
|
Sat, 15 May 2010 17:59:06 +0200 |
wenzelm |
incorporated further conversions and conversionals, after some minor tuning;
|
file |
diff |
annotate
|
Wed, 12 May 2010 23:54:04 +0200 |
boehmes |
layered SMT setup, adapted SMT clients, added further tests, made Z3 proof abstraction configurable
|
file |
diff |
annotate
|
Wed, 12 May 2010 23:54:02 +0200 |
boehmes |
integrated SMT into the HOL image
|
file |
diff |
annotate
|