Thu, 09 Jun 2011 08:32:21 +0200 |
bulwahn |
removing unneccessary manual instantiations and dead definitions; hiding more constants and facts
|
changeset |
files
|
Thu, 09 Jun 2011 08:32:19 +0200 |
bulwahn |
adding a nicer error message for quickcheck_narrowing; hiding fact empty_def
|
changeset |
files
|
Thu, 09 Jun 2011 08:32:18 +0200 |
bulwahn |
adding narrowing engine for existentials
|
changeset |
files
|
Thu, 09 Jun 2011 08:32:18 +0200 |
bulwahn |
adapting Quickcheck_Narrowing: adding setup for characters; correcting import statement
|
changeset |
files
|
Thu, 09 Jun 2011 08:32:16 +0200 |
bulwahn |
adding theory Quickcheck_Narrowing to HOL-Main image
|
changeset |
files
|
Thu, 09 Jun 2011 08:32:15 +0200 |
bulwahn |
adapting IsaMakefile
|
changeset |
files
|
Thu, 09 Jun 2011 08:32:14 +0200 |
bulwahn |
moving Quickcheck_Narrowing from Library to base directory
|
changeset |
files
|
Thu, 09 Jun 2011 08:32:13 +0200 |
bulwahn |
compilation of Haskell in its own target for Quickcheck; passing options by arguments in Narrowing_Generators
|
changeset |
files
|
Thu, 09 Jun 2011 08:31:41 +0200 |
bulwahn |
local simp rule in List_Cset
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
tuning
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
compile
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
cleaner fact freshening, which also works in corner cases, e.g. if two backquoted facts have the same name (but have different variable indices)
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
added a really fully typed translation as a fallback for Metis, in rare cases where Metis correctly proves a theorem but has type-unsound steps in it (which is likelier to happen with some of the lighter translations)
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
improve sort inference in Metis proofs -- in some rare cases Metis steals Isabelle's variable names and the sorts must then be inferred as well
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
removed needless function that duplicated standard functionality, with a little unnecessary twist
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
removed more dead code
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
be a bit more liberal with respect to the universal sort -- it sometimes help
|
changeset |
files
|
Thu, 09 Jun 2011 00:16:28 +0200 |
blanchet |
renamed "untyped_aconv" to distinguish it clearly from the standard "aconv_untyped"
|
changeset |
files
|
Wed, 08 Jun 2011 22:13:49 +0200 |
wenzelm |
merged
|
changeset |
files
|
Wed, 08 Jun 2011 17:01:07 +0200 |
blanchet |
avoid duplicate facts, which confuse the minimizer output
|
changeset |
files
|
Wed, 08 Jun 2011 16:20:19 +0200 |
blanchet |
pass Metis facts and negated conjecture as facts, with (almost) correctly set localities, so that the correct encoding is used for nonmonotonic occurrences of infinite types
|
changeset |
files
|
Wed, 08 Jun 2011 16:20:18 +0200 |
blanchet |
restore comment about subtle issue
|
changeset |
files
|
Wed, 08 Jun 2011 16:20:18 +0200 |
blanchet |
made "query" type systes a bit more sound -- local facts, e.g. the negated conjecture, may make invalid the infinity check, e.g. if we are proving that there exists two values of an infinite type, we can use the negated conjecture that there is only one value to derive unsound proofs unless the type is properly encoded
|
changeset |
files
|
Wed, 08 Jun 2011 16:20:18 +0200 |
blanchet |
don't launch the automatic minimizer for zero facts
|
changeset |
files
|
Wed, 08 Jun 2011 16:20:18 +0200 |
blanchet |
don't generate unsound proof error for missing proofs
|
changeset |
files
|
Wed, 08 Jun 2011 16:20:18 +0200 |
blanchet |
renamed option to avoid talking about seconds, since this is now the default Isabelle unit
|
changeset |
files
|
Wed, 08 Jun 2011 16:20:18 +0200 |
blanchet |
fixed format selection logic for Waldmeister
|
changeset |
files
|
Wed, 08 Jun 2011 16:20:18 +0200 |
blanchet |
better default type system for Waldmeister, with fewer predicates (for types or type classes)
|
changeset |
files
|
Wed, 08 Jun 2011 22:06:05 +0200 |
wenzelm |
simplified directory structure;
|
changeset |
files
|
Wed, 08 Jun 2011 21:40:54 +0200 |
wenzelm |
simplified directory structure;
|
changeset |
files
|
Wed, 08 Jun 2011 21:29:49 +0200 |
wenzelm |
further jedit build option;
|
changeset |
files
|
Wed, 08 Jun 2011 20:58:51 +0200 |
wenzelm |
build jedit as part of regular startup script (in that case depending on jedit_build component);
|
changeset |
files
|
Wed, 08 Jun 2011 17:49:01 +0200 |
wenzelm |
updated headers;
|
changeset |
files
|
Wed, 08 Jun 2011 17:42:07 +0200 |
wenzelm |
moved sources -- eliminated Netbeans artifact of jedit package directory;
|
changeset |
files
|
Wed, 08 Jun 2011 17:32:31 +0200 |
wenzelm |
removed obsolete Netbeans project setup;
|
changeset |
files
|
Wed, 08 Jun 2011 17:11:00 +0200 |
wenzelm |
support fresh build of jars;
|
changeset |
files
|
Wed, 08 Jun 2011 16:19:22 +0200 |
wenzelm |
more jvmpath wrapping for Cygwin;
|
changeset |
files
|
Wed, 08 Jun 2011 15:56:57 +0200 |
wenzelm |
more robust exception pattern General.Subscript;
|
changeset |
files
|
Wed, 08 Jun 2011 15:39:55 +0200 |
wenzelm |
pervasive Output operations;
|
changeset |
files
|
Wed, 08 Jun 2011 15:25:44 +0200 |
wenzelm |
modernized Proof_Context;
|
changeset |
files
|
Wed, 08 Jun 2011 14:44:54 +0200 |
wenzelm |
standardized header;
|
changeset |
files
|
Wed, 08 Jun 2011 13:45:01 +0200 |
boehmes |
merged
|
changeset |
files
|
Wed, 08 Jun 2011 13:43:15 +0200 |
boehmes |
updated SMT certificates
|
changeset |
files
|
Wed, 08 Jun 2011 11:59:45 +0200 |
boehmes |
only collect substituions neither seen before nor derived in the same refinement step
|
changeset |
files
|
Wed, 08 Jun 2011 12:13:37 +0200 |
wenzelm |
updated imports (cf. 93b1183e43e5);
|
changeset |
files
|
Wed, 08 Jun 2011 10:24:07 +0200 |
wenzelm |
merged
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
new Metis version
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
removed yet another hack in "make_metis" script -- respect opacity of "Metis_Name.name"
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
exploit new semantics of "max_new_instances"
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
minor optimization
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
don't needlessly extensionalize
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
don't needlessly presimplify -- makes ATP problem preparation much faster
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
tuned
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
removed experimental code submitted by mistake
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
make sure that the message tail (timing + TPTP important message) is preserved upon automatic minimization
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
removed removed option from documentation
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
killed "explicit_apply" option in Sledgehammer -- the "smart" default is about as lightweight as "false" and just as complete as "true"
|
changeset |
files
|
Wed, 08 Jun 2011 08:47:43 +0200 |
blanchet |
slightly faster/cleaner accumulation of polymorphic consts
|
changeset |
files
|
Wed, 08 Jun 2011 00:01:20 +0200 |
krauss |
eliminated unnecessary tail-recursion and funny use of records as 'named arguments' for functions
|
changeset |
files
|
Wed, 08 Jun 2011 00:01:20 +0200 |
krauss |
more conventional variable naming
|
changeset |
files
|
Wed, 08 Jun 2011 00:01:20 +0200 |
krauss |
dropped outdated/speculative historical comments;
|
changeset |
files
|
Wed, 08 Jun 2011 00:01:20 +0200 |
krauss |
less redundant tags
|
changeset |
files
|
Wed, 08 Jun 2011 00:01:20 +0200 |
krauss |
removed generation of instantiated pattern set, which is never actually used
|
changeset |
files
|
Wed, 08 Jun 2011 00:01:20 +0200 |
krauss |
more precise type for obscure "prfx" field
|
changeset |
files
|
Tue, 07 Jun 2011 21:37:40 +0200 |
boehmes |
clarified (and slightly modified) the semantics of max_new_instances
|
changeset |
files
|
Tue, 07 Jun 2011 19:22:52 +0200 |
kleing |
use null_heap instead of %_. 0 to avoid printing problems
|
changeset |
files
|
Tue, 07 Jun 2011 14:38:42 +0200 |
blanchet |
prioritize more relevant facts for monomorphization
|
changeset |
files
|
Tue, 07 Jun 2011 14:17:35 +0200 |
blanchet |
more suitable implementation of "schematic_consts_of" for monomorphizer, for ATPs
|
changeset |
files
|
Tue, 07 Jun 2011 14:17:35 +0200 |
blanchet |
workaround current "max_new_instances" semantics
|
changeset |
files
|
Tue, 07 Jun 2011 14:17:35 +0200 |
blanchet |
fixed missing proof handling
|
changeset |
files
|
Tue, 07 Jun 2011 14:17:35 +0200 |
blanchet |
optimized the relevance filter a little bit
|
changeset |
files
|
Tue, 07 Jun 2011 14:06:12 +0200 |
bulwahn |
printing environment in mutabelle's log
|
changeset |
files
|
Tue, 07 Jun 2011 11:24:54 +0200 |
bulwahn |
merged
|
changeset |
files
|
Tue, 07 Jun 2011 11:24:16 +0200 |
bulwahn |
merged; manually merged IsaMakefile
|
changeset |
files
|
Tue, 07 Jun 2011 11:12:05 +0200 |
bulwahn |
splitting Cset into Cset and List_Cset
|
changeset |
files
|
Tue, 07 Jun 2011 11:11:01 +0200 |
bulwahn |
adding finitize_functions and processing of equivalences in existential compilation in quickcheck_narrowing
|
changeset |
files
|
Tue, 07 Jun 2011 11:10:58 +0200 |
bulwahn |
adding examples with existentials
|
changeset |
files
|
Tue, 07 Jun 2011 11:10:57 +0200 |
bulwahn |
renaming the formalisation of the birthday problem to a proper English name
|
changeset |
files
|
Tue, 07 Jun 2011 11:10:42 +0200 |
bulwahn |
adding compilation that allows existentials in Quickcheck_Narrowing
|
changeset |
files
|
Tue, 07 Jun 2011 11:13:52 +0200 |
blanchet |
move away from old SMT monomorphizer
|
changeset |
files
|
Tue, 07 Jun 2011 11:12:52 +0200 |
blanchet |
tuning
|
changeset |
files
|
Tue, 07 Jun 2011 11:05:09 +0200 |
blanchet |
merged
|
changeset |
files
|
Tue, 07 Jun 2011 11:04:17 +0200 |
blanchet |
use the proper prover name, e.g. metis_full_types, not metis (full_types), for minimizing
|
changeset |
files
|
Tue, 07 Jun 2011 10:46:09 +0200 |
blanchet |
removed "verbose" option -- there won't be any verbosity in there, according to Sascha (yeah)
|
changeset |
files
|
Tue, 07 Jun 2011 10:43:18 +0200 |
blanchet |
nicely thread monomorphism verbosity in Metis and Sledgehammer
|
changeset |
files
|
Tue, 07 Jun 2011 10:24:16 +0200 |
boehmes |
clarified meaning of monomorphization configuration option by renaming it
|
changeset |
files
|
Tue, 07 Jun 2011 08:58:23 +0200 |
blanchet |
documentation tweaks
|
changeset |
files
|
Tue, 07 Jun 2011 08:52:35 +0200 |
blanchet |
obsoleted "metisFT", and added "no_types" version of Metis as fallback to Sledgehammer after noticing how useful it can be
|
changeset |
files
|
Tue, 07 Jun 2011 07:57:24 +0200 |
blanchet |
fixed typo in legacy feature message
|
changeset |
files
|
Tue, 07 Jun 2011 07:45:12 +0200 |
blanchet |
use new monomorphization code
|
changeset |
files
|
Tue, 07 Jun 2011 07:44:54 +0200 |
blanchet |
added (currently unused) verbose configuration option
|
changeset |
files
|
Tue, 07 Jun 2011 07:06:24 +0200 |
blanchet |
renamed ML function
|
changeset |
files
|
Tue, 07 Jun 2011 07:04:53 +0200 |
blanchet |
renamed example theory to "ATP_Export", for consistency with its underlying "ATP_" modules
|
changeset |
files
|
Tue, 07 Jun 2011 06:58:52 +0200 |
blanchet |
pass props not thms to ATP translator
|
changeset |
files
|
Mon, 06 Jun 2011 23:46:02 +0200 |
blanchet |
slighly more reasonable Vampire slices (until new monomorphizer is used)
|
changeset |
files
|
Mon, 06 Jun 2011 23:43:28 +0200 |
blanchet |
removed confusing slicing logic
|
changeset |
files
|
Mon, 06 Jun 2011 23:26:40 +0200 |
blanchet |
suggest first reconstructor that timed out, not last (i.e. metis not metisFT in most cases)
|
changeset |
files
|
Mon, 06 Jun 2011 23:11:14 +0200 |
blanchet |
effectively reenable slices for SPASS and Vampire -- they were disabled by mistake
|
changeset |
files
|
Mon, 06 Jun 2011 22:03:58 +0200 |
blanchet |
minor: curly brackets, not square brackets
|
changeset |
files
|
Mon, 06 Jun 2011 21:58:29 +0200 |
blanchet |
document metis better in Sledgehammer docs
|
changeset |
files
|
Mon, 06 Jun 2011 21:02:24 +0200 |
blanchet |
updated Sledgehammer message
|
changeset |
files
|
Mon, 06 Jun 2011 20:56:06 +0200 |
blanchet |
removed old optimization that isn't one anyone
|
changeset |
files
|
Mon, 06 Jun 2011 20:56:06 +0200 |
blanchet |
generate less type information in polymorphic case
|
changeset |
files
|
Mon, 06 Jun 2011 20:56:06 +0200 |
blanchet |
Metis code cleanup
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:36 +0200 |
blanchet |
enable new Metis
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
made "explicit_apply"'s smart mode (more) complete
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
fall back in case path finder fails -- these errors are sometimes salvageable
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
compile
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
change var name as a workaround for rare issue in Metis's reconstruction code -- namely, "find_var" fails because "X = X" is wrongly mirrorred as "A = A"
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
marked "metisF" as legacy -- nobody uses it or needs it
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
more preparations towards hijacking Metis
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
remove more occurrences of "metisX", preparing for the D Day when it will silently hijack "metis" and "metisFT"
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
don't mention "metisX" so much in the docs -- it will go away soon
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
reintroduced metisFT in example
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
make "smart" mode of "explicit_apply" smarter, by also detecting the other kind of higher-order quantification, namely "bool"s
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
imported patch metis_reconstr_give_type_infer_a_chance
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
make "metisX"'s default more like old "metis"
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
whitespace tuning
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
tuned Metis examples
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
more through tests of new Metis
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
improved correctness of handling of higher-order occurrences of "Not" in new Metis (and probably in old Metis)
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
fixed type helper indices in new Metis
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
improved ATP clausifier so it can deal with "x => (y <=> z)"
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
avoid renumbering hypotheses
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
fixed reconstruction of new Skolem constants in new Metis
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
don't translate new Skolemizer assumptions in new Metis
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
tuning
|
changeset |
files
|
Mon, 06 Jun 2011 20:36:35 +0200 |
blanchet |
fixed detection of Skolem constants in type construction detection code
|
changeset |
files
|