Wed, 09 Mar 2011 10:28:01 +0100 |
blanchet |
improved formula for specialization, to prevent needless specializations -- and removed dead code
|
changeset |
files
|
Wed, 09 Mar 2011 10:25:29 +0100 |
blanchet |
perform no arity check in debug mode so that we get to see the Kodkod problem
|
changeset |
files
|
Fri, 04 Mar 2011 17:39:30 +0100 |
berghofe |
spark_end now joins proofs of VCs before writing *.prv file.
|
changeset |
files
|
Fri, 04 Mar 2011 11:43:20 +0100 |
krauss |
clarified
|
changeset |
files
|
Fri, 04 Mar 2011 11:52:54 +0100 |
krauss |
produce helpful mira summary for more errors
|
changeset |
files
|
Fri, 04 Mar 2011 00:09:47 +0100 |
wenzelm |
eliminated prems;
|
changeset |
files
|
Thu, 03 Mar 2011 22:06:15 +0100 |
wenzelm |
eliminated UNITY_Examples.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 3dec57ec3473;
|
changeset |
files
|
Thu, 03 Mar 2011 21:43:06 +0100 |
wenzelm |
tuned proofs -- eliminated prems;
|
changeset |
files
|
Thu, 03 Mar 2011 18:43:15 +0100 |
wenzelm |
merged
|
changeset |
files
|
Thu, 03 Mar 2011 14:38:31 +0100 |
blanchet |
merged
|
changeset |
files
|
Thu, 03 Mar 2011 14:25:15 +0100 |
blanchet |
don't forget to look for constants appearing only in "need" option -- otherwise we get exceptions in "the_name" later on
|
changeset |
files
|
Thu, 03 Mar 2011 18:42:12 +0100 |
wenzelm |
simplified Thy_Info.check_file -- discontinued load path;
|
changeset |
files
|
Thu, 03 Mar 2011 18:10:28 +0100 |
wenzelm |
discontinued legacy load path;
|
changeset |
files
|
Thu, 03 Mar 2011 15:56:17 +0100 |
wenzelm |
re-interpret ProofGeneralPgip.changecwd as Thy_Load.set_master_path, presuming that this is close to the intended semantics;
|
changeset |
files
|
Thu, 03 Mar 2011 15:46:02 +0100 |
wenzelm |
modernized imports;
|
changeset |
files
|
Thu, 03 Mar 2011 15:36:54 +0100 |
wenzelm |
observe standard header format;
|
changeset |
files
|
Thu, 03 Mar 2011 15:19:20 +0100 |
wenzelm |
removed spurious 'unused_thms' (cf. 1a65b780bd56);
|
changeset |
files
|
Thu, 03 Mar 2011 15:18:05 +0100 |
wenzelm |
isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
|
changeset |
files
|
Thu, 03 Mar 2011 11:36:10 +0100 |
berghofe |
merged
|
changeset |
files
|
Thu, 03 Mar 2011 11:15:50 +0100 |
berghofe |
merged
|
changeset |
files
|
Thu, 03 Mar 2011 11:01:42 +0100 |
berghofe |
- Made sure that sort_defs is aware of constants introduced by add_type_def
|
changeset |
files
|
Thu, 03 Mar 2011 11:20:48 +0100 |
blanchet |
mention new Nitpick options
|
changeset |
files
|
Thu, 03 Mar 2011 11:20:48 +0100 |
blanchet |
simplify "need" option's syntax
|
changeset |
files
|
Thu, 03 Mar 2011 11:20:48 +0100 |
blanchet |
renamed "preconstr" option "need"
|
changeset |
files
|
Thu, 03 Mar 2011 10:55:41 +0100 |
hoelzl |
finally remove upper_bound_finite_set
|
changeset |
files
|
Thu, 03 Mar 2011 15:59:44 +1100 |
kleing |
separate settings for afp test
|
changeset |
files
|
Wed, 02 Mar 2011 15:51:22 +0100 |
blanchet |
added missing spaces in output
|
changeset |
files
|
Wed, 02 Mar 2011 14:50:16 +0100 |
blanchet |
lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
|
changeset |
files
|
Wed, 02 Mar 2011 13:09:57 +0100 |
blanchet |
unfold definitions in "preconstrs" option
|
changeset |
files
|
Wed, 02 Mar 2011 13:09:57 +0100 |
blanchet |
robust handling of types occurring in "eval" and "preconstr" options but not in the goal
|
changeset |
files
|
Wed, 02 Mar 2011 13:09:57 +0100 |
blanchet |
make "preconstr" option more robust -- shouldn't throw exceptions
|
changeset |
files
|
Tue, 01 Mar 2011 10:40:14 +0000 |
paulson |
merged
|
changeset |
files
|
Mon, 28 Feb 2011 15:06:55 +0000 |
paulson |
merged
|
changeset |
files
|
Mon, 28 Feb 2011 15:06:36 +0000 |
paulson |
declare ext [intro]: Extensionality now available by default
|
changeset |
files
|
Mon, 28 Feb 2011 22:12:09 +0100 |
boehmes |
merged
|
changeset |
files
|
Mon, 28 Feb 2011 22:10:57 +0100 |
boehmes |
removed dependency on Dense_Linear_Order
|
changeset |
files
|
Mon, 28 Feb 2011 19:06:24 +0100 |
bulwahn |
adding function Quickcheck.test_terms to provide checking a batch of terms
|
changeset |
files
|
Mon, 28 Feb 2011 19:06:23 +0100 |
bulwahn |
adding a function to compile a batch of terms for quickcheck with one code generation invocation
|
changeset |
files
|
Mon, 28 Feb 2011 17:53:10 +0100 |
blanchet |
improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
|
changeset |
files
|
Mon, 28 Feb 2011 17:53:10 +0100 |
blanchet |
made "fixed_is_special_eligible_arg" smarter w.r.t. pairs, and fixed previous unintended behavior because "andalso" ties more tightly than "orelse"
|
changeset |
files
|
Mon, 28 Feb 2011 17:53:10 +0100 |
blanchet |
if "total_consts" is set, report cex's as quasi-genuine
|
changeset |
files
|
Mon, 28 Feb 2011 17:53:10 +0100 |
blanchet |
document new "total_consts" option
|
changeset |
files
|
Mon, 28 Feb 2011 17:53:10 +0100 |
blanchet |
added "total_consts" option
|
changeset |
files
|
Sat, 26 Feb 2011 20:40:45 +0100 |
nipkow |
added a few lemmas by Andreas Lochbihler
|
changeset |
files
|
Sat, 26 Feb 2011 20:16:44 +0100 |
nipkow |
Corrected HOLCF/FOCUS dependency
|
changeset |
files
|
Sat, 26 Feb 2011 17:44:42 +0100 |
nipkow |
Added material by David Trachtenherz
|
changeset |
files
|
Sat, 26 Feb 2011 16:16:36 +0100 |
nipkow |
corrected HOLCF dependency on Nat_Infinity
|
changeset |
files
|
Fri, 25 Feb 2011 22:07:56 +0100 |
nipkow |
got rid of lemma upper_bound_finite_set
|
changeset |
files
|
Fri, 25 Feb 2011 20:08:00 +0100 |
nipkow |
merged
|
changeset |
files
|
Fri, 25 Feb 2011 20:07:48 +0100 |
nipkow |
Some cleaning up
|
changeset |
files
|
Fri, 25 Feb 2011 17:11:24 +0100 |
krauss |
updated generated files
|
changeset |
files
|
Fri, 25 Feb 2011 17:11:05 +0100 |
krauss |
fixed manual (rule no longer exists)
|
changeset |
files
|
Fri, 25 Feb 2011 16:59:48 +0100 |
krauss |
removed support for tail-recursion from function package (now implemented by partial_function)
|
changeset |
files
|
Fri, 25 Feb 2011 16:57:44 +0100 |
krauss |
reactivate time measurement (partly reverting c27b0b37041a);
|
changeset |
files
|
Fri, 25 Feb 2011 16:57:43 +0100 |
krauss |
generalize find_theorems filters to work on raw propositions, too
|
changeset |
files
|
Fri, 25 Feb 2011 14:25:52 +0100 |
nipkow |
merged
|
changeset |
files
|
Fri, 25 Feb 2011 14:25:41 +0100 |
nipkow |
added simp lemma nth_Cons_pos to List
|
changeset |
files
|
Fri, 25 Feb 2011 12:16:18 +0100 |
noschinl |
Refactor find_theorems to provide a more general filter_facts method
|
changeset |
files
|
Fri, 25 Feb 2011 08:46:52 +0100 |
krauss |
removed dead code/unused exports/speculative generality
|
changeset |
files
|
Thu, 24 Feb 2011 21:54:28 +0100 |
krauss |
recdef -> fun(ction)
|
changeset |
files
|