Fri, 11 Mar 2011 08:12:59 +0100 renaming dest_plain_fun to dest_fun_upds and adding handling of undefined for postprocessing of quickcheck
bulwahn [Fri, 11 Mar 2011 08:12:59 +0100] rev 41902
renaming dest_plain_fun to dest_fun_upds and adding handling of undefined for postprocessing of quickcheck
Fri, 11 Mar 2011 08:12:58 +0100 improving term postprocessing for counterexample presentation in quickcheck
bulwahn [Fri, 11 Mar 2011 08:12:58 +0100] rev 41901
improving term postprocessing for counterexample presentation in quickcheck
Fri, 11 Mar 2011 08:12:55 +0100 tuned
bulwahn [Fri, 11 Mar 2011 08:12:55 +0100] rev 41900
tuned
Wed, 09 Mar 2011 21:40:38 +0100 finished and tested Z3 proof reconstruction for injective functions;
boehmes [Wed, 09 Mar 2011 21:40:38 +0100] rev 41899
finished and tested Z3 proof reconstruction for injective functions; only treat variables as atomic, and especially abstract constants (Isabelle's interpretation of these constants is most likely not known to Z3 and thus irrelevant for the proof)
Wed, 09 Mar 2011 10:28:01 +0100 improved formula for specialization, to prevent needless specializations -- and removed dead code
blanchet [Wed, 09 Mar 2011 10:28:01 +0100] rev 41898
improved formula for specialization, to prevent needless specializations -- and removed dead code
Wed, 09 Mar 2011 10:25:29 +0100 perform no arity check in debug mode so that we get to see the Kodkod problem
blanchet [Wed, 09 Mar 2011 10:25:29 +0100] rev 41897
perform no arity check in debug mode so that we get to see the Kodkod problem
Fri, 04 Mar 2011 17:39:30 +0100 spark_end now joins proofs of VCs before writing *.prv file.
berghofe [Fri, 04 Mar 2011 17:39:30 +0100] rev 41896
spark_end now joins proofs of VCs before writing *.prv file.
Fri, 04 Mar 2011 11:43:20 +0100 clarified
krauss [Fri, 04 Mar 2011 11:43:20 +0100] rev 41895
clarified
Fri, 04 Mar 2011 11:52:54 +0100 produce helpful mira summary for more errors
krauss [Fri, 04 Mar 2011 11:52:54 +0100] rev 41894
produce helpful mira summary for more errors
Fri, 04 Mar 2011 00:09:47 +0100 eliminated prems;
wenzelm [Fri, 04 Mar 2011 00:09:47 +0100] rev 41893
eliminated prems;
Thu, 03 Mar 2011 22:06:15 +0100 eliminated UNITY_Examples.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 3dec57ec3473;
wenzelm [Thu, 03 Mar 2011 22:06:15 +0100] rev 41892
eliminated UNITY_Examples.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 3dec57ec3473;
Thu, 03 Mar 2011 21:43:06 +0100 tuned proofs -- eliminated prems;
wenzelm [Thu, 03 Mar 2011 21:43:06 +0100] rev 41891
tuned proofs -- eliminated prems;
Thu, 03 Mar 2011 18:43:15 +0100 merged
wenzelm [Thu, 03 Mar 2011 18:43:15 +0100] rev 41890
merged
Thu, 03 Mar 2011 14:38:31 +0100 merged
blanchet [Thu, 03 Mar 2011 14:38:31 +0100] rev 41889
merged
Thu, 03 Mar 2011 14:25:15 +0100 don't forget to look for constants appearing only in "need" option -- otherwise we get exceptions in "the_name" later on
blanchet [Thu, 03 Mar 2011 14:25:15 +0100] rev 41888
don't forget to look for constants appearing only in "need" option -- otherwise we get exceptions in "the_name" later on
Thu, 03 Mar 2011 18:42:12 +0100 simplified Thy_Info.check_file -- discontinued load path;
wenzelm [Thu, 03 Mar 2011 18:42:12 +0100] rev 41887
simplified Thy_Info.check_file -- discontinued load path;
Thu, 03 Mar 2011 18:10:28 +0100 discontinued legacy load path;
wenzelm [Thu, 03 Mar 2011 18:10:28 +0100] rev 41886
discontinued legacy load path;
Thu, 03 Mar 2011 15:56:17 +0100 re-interpret ProofGeneralPgip.changecwd as Thy_Load.set_master_path, presuming that this is close to the intended semantics;
wenzelm [Thu, 03 Mar 2011 15:56:17 +0100] rev 41885
re-interpret ProofGeneralPgip.changecwd as Thy_Load.set_master_path, presuming that this is close to the intended semantics;
Thu, 03 Mar 2011 15:46:02 +0100 modernized imports;
wenzelm [Thu, 03 Mar 2011 15:46:02 +0100] rev 41884
modernized imports;
Thu, 03 Mar 2011 15:36:54 +0100 observe standard header format;
wenzelm [Thu, 03 Mar 2011 15:36:54 +0100] rev 41883
observe standard header format;
Thu, 03 Mar 2011 15:19:20 +0100 removed spurious 'unused_thms' (cf. 1a65b780bd56);
wenzelm [Thu, 03 Mar 2011 15:19:20 +0100] rev 41882
removed spurious 'unused_thms' (cf. 1a65b780bd56);
Thu, 03 Mar 2011 15:18:05 +0100 isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
wenzelm [Thu, 03 Mar 2011 15:18:05 +0100] rev 41881
isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
Thu, 03 Mar 2011 11:36:10 +0100 merged
berghofe [Thu, 03 Mar 2011 11:36:10 +0100] rev 41880
merged
Thu, 03 Mar 2011 11:15:50 +0100 merged
berghofe [Thu, 03 Mar 2011 11:15:50 +0100] rev 41879
merged
Thu, 03 Mar 2011 11:01:42 +0100 - Made sure that sort_defs is aware of constants introduced by add_type_def
berghofe [Thu, 03 Mar 2011 11:01:42 +0100] rev 41878
- Made sure that sort_defs is aware of constants introduced by add_type_def - add_def now compares Isabelle types rather than SPARK types to ensure that type abbreviations are taken into account
Thu, 03 Mar 2011 11:20:48 +0100 mention new Nitpick options
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41877
mention new Nitpick options
Thu, 03 Mar 2011 11:20:48 +0100 simplify "need" option's syntax
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41876
simplify "need" option's syntax
Thu, 03 Mar 2011 11:20:48 +0100 renamed "preconstr" option "need"
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41875
renamed "preconstr" option "need"
Thu, 03 Mar 2011 10:55:41 +0100 finally remove upper_bound_finite_set
hoelzl [Thu, 03 Mar 2011 10:55:41 +0100] rev 41874
finally remove upper_bound_finite_set
Thu, 03 Mar 2011 15:59:44 +1100 separate settings for afp test
kleing [Thu, 03 Mar 2011 15:59:44 +1100] rev 41873
separate settings for afp test
Wed, 02 Mar 2011 15:51:22 +0100 added missing spaces in output
blanchet [Wed, 02 Mar 2011 15:51:22 +0100] rev 41872
added missing spaces in output
Wed, 02 Mar 2011 14:50:16 +0100 lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
blanchet [Wed, 02 Mar 2011 14:50:16 +0100] rev 41871
lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
Wed, 02 Mar 2011 13:09:57 +0100 unfold definitions in "preconstrs" option
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41870
unfold definitions in "preconstrs" option
Wed, 02 Mar 2011 13:09:57 +0100 robust handling of types occurring in "eval" and "preconstr" options but not in the goal
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41869
robust handling of types occurring in "eval" and "preconstr" options but not in the goal
Wed, 02 Mar 2011 13:09:57 +0100 make "preconstr" option more robust -- shouldn't throw exceptions
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41868
make "preconstr" option more robust -- shouldn't throw exceptions
Tue, 01 Mar 2011 10:40:14 +0000 merged
paulson [Tue, 01 Mar 2011 10:40:14 +0000] rev 41867
merged
Mon, 28 Feb 2011 15:06:55 +0000 merged
paulson [Mon, 28 Feb 2011 15:06:55 +0000] rev 41866
merged
Mon, 28 Feb 2011 15:06:36 +0000 declare ext [intro]: Extensionality now available by default
paulson [Mon, 28 Feb 2011 15:06:36 +0000] rev 41865
declare ext [intro]: Extensionality now available by default
Mon, 28 Feb 2011 22:12:09 +0100 merged
boehmes [Mon, 28 Feb 2011 22:12:09 +0100] rev 41864
merged
Mon, 28 Feb 2011 22:10:57 +0100 removed dependency on Dense_Linear_Order
boehmes [Mon, 28 Feb 2011 22:10:57 +0100] rev 41863
removed dependency on Dense_Linear_Order
Mon, 28 Feb 2011 19:06:24 +0100 adding function Quickcheck.test_terms to provide checking a batch of terms
bulwahn [Mon, 28 Feb 2011 19:06:24 +0100] rev 41862
adding function Quickcheck.test_terms to provide checking a batch of terms
Mon, 28 Feb 2011 19:06:23 +0100 adding a function to compile a batch of terms for quickcheck with one code generation invocation
bulwahn [Mon, 28 Feb 2011 19:06:23 +0100] rev 41861
adding a function to compile a batch of terms for quickcheck with one code generation invocation
Mon, 28 Feb 2011 17:53:10 +0100 improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41860
improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
Mon, 28 Feb 2011 17:53:10 +0100 made "fixed_is_special_eligible_arg" smarter w.r.t. pairs, and fixed previous unintended behavior because "andalso" ties more tightly than "orelse"
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41859
made "fixed_is_special_eligible_arg" smarter w.r.t. pairs, and fixed previous unintended behavior because "andalso" ties more tightly than "orelse"
Mon, 28 Feb 2011 17:53:10 +0100 if "total_consts" is set, report cex's as quasi-genuine
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41858
if "total_consts" is set, report cex's as quasi-genuine
Mon, 28 Feb 2011 17:53:10 +0100 document new "total_consts" option
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41857
document new "total_consts" option
Mon, 28 Feb 2011 17:53:10 +0100 added "total_consts" option
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41856
added "total_consts" option
Sat, 26 Feb 2011 20:40:45 +0100 added a few lemmas by Andreas Lochbihler
nipkow [Sat, 26 Feb 2011 20:40:45 +0100] rev 41855
added a few lemmas by Andreas Lochbihler
Sat, 26 Feb 2011 20:16:44 +0100 Corrected HOLCF/FOCUS dependency
nipkow [Sat, 26 Feb 2011 20:16:44 +0100] rev 41854
Corrected HOLCF/FOCUS dependency
Sat, 26 Feb 2011 17:44:42 +0100 Added material by David Trachtenherz
nipkow [Sat, 26 Feb 2011 17:44:42 +0100] rev 41853
Added material by David Trachtenherz
Sat, 26 Feb 2011 16:16:36 +0100 corrected HOLCF dependency on Nat_Infinity
nipkow [Sat, 26 Feb 2011 16:16:36 +0100] rev 41852
corrected HOLCF dependency on Nat_Infinity
Fri, 25 Feb 2011 22:07:56 +0100 got rid of lemma upper_bound_finite_set
nipkow [Fri, 25 Feb 2011 22:07:56 +0100] rev 41851
got rid of lemma upper_bound_finite_set
Fri, 25 Feb 2011 20:08:00 +0100 merged
nipkow [Fri, 25 Feb 2011 20:08:00 +0100] rev 41850
merged
Fri, 25 Feb 2011 20:07:48 +0100 Some cleaning up
nipkow [Fri, 25 Feb 2011 20:07:48 +0100] rev 41849
Some cleaning up
Fri, 25 Feb 2011 17:11:24 +0100 updated generated files
krauss [Fri, 25 Feb 2011 17:11:24 +0100] rev 41848
updated generated files
Fri, 25 Feb 2011 17:11:05 +0100 fixed manual (rule no longer exists)
krauss [Fri, 25 Feb 2011 17:11:05 +0100] rev 41847
fixed manual (rule no longer exists)
Fri, 25 Feb 2011 16:59:48 +0100 removed support for tail-recursion from function package (now implemented by partial_function)
krauss [Fri, 25 Feb 2011 16:59:48 +0100] rev 41846
removed support for tail-recursion from function package (now implemented by partial_function)
Fri, 25 Feb 2011 16:57:44 +0100 reactivate time measurement (partly reverting c27b0b37041a);
krauss [Fri, 25 Feb 2011 16:57:44 +0100] rev 41845
reactivate time measurement (partly reverting c27b0b37041a); export pretty_theorem, to display both internal or external facts
Fri, 25 Feb 2011 16:57:43 +0100 generalize find_theorems filters to work on raw propositions, too
krauss [Fri, 25 Feb 2011 16:57:43 +0100] rev 41844
generalize find_theorems filters to work on raw propositions, too
Fri, 25 Feb 2011 14:25:52 +0100 merged
nipkow [Fri, 25 Feb 2011 14:25:52 +0100] rev 41843
merged
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip