Sun, 13 Mar 2011 19:16:19 +0100 wenzelm cleanup of former settings GHC_PATH, EXEC_GHC, EXEC_OCAML, EXEC_SWIPL, EXEC_YAP -- discontinued implicit detection;
Sun, 13 Mar 2011 17:35:35 +0100 wenzelm some cleanup of old-style settings;
Sun, 13 Mar 2011 17:28:14 +0100 wenzelm clarified ISABELLE_CSDP setting (formerly CSDP_EXE);
Sun, 13 Mar 2011 16:52:59 +0100 wenzelm more conventional Mutabelle settings -- similar to Mirabelle;
Sun, 13 Mar 2011 16:38:54 +0100 wenzelm more basic use of Path.position/File.read;
Sun, 13 Mar 2011 16:38:14 +0100 wenzelm prefer qualified ISABELLE_NEOS_SERVER;
Sun, 13 Mar 2011 16:30:02 +0100 wenzelm proper File.shell_path;
Sun, 13 Mar 2011 16:14:14 +0100 wenzelm more conventional variable name;
Sun, 13 Mar 2011 16:01:00 +0100 wenzelm Path.print is the official way to show file-system paths to users -- note that Path.implode often indicates violation of the abstract datatype;
Sun, 13 Mar 2011 15:16:37 +0100 wenzelm fixed document;
Sun, 13 Mar 2011 15:13:53 +0100 wenzelm isatest: test more external code;
Sun, 13 Mar 2011 15:10:00 +0100 wenzelm tuned headers;
Sun, 13 Mar 2011 14:51:38 +0100 wenzelm allow spaces in executable names;
Sun, 13 Mar 2011 13:57:20 +0100 wenzelm tuned;
Sun, 13 Mar 2011 13:53:54 +0100 wenzelm tuned headers;
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn adapting example file to renaming of the quickcheck tester
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn renaming tester from lazy_exhaustive to narrowing
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn minor corrections for renaming; moved postprocessing of terms to Quickcheck_Common
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn renaming example file correctly
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn adapting Main file generation for Quickcheck_Narrowing
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn adapting Quickcheck_Narrowing and example file to new names
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn renaming LSC_Examples theory to Quickcheck_Narrowing
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn renaming lazysmallcheck ML file to Quickcheck_Narrowing
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn renaming LSC to Quickcheck_Narrowing
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn adaptions in generators using the common functions
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn adding file quickcheck_common to carry common functions of all quickcheck generators
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn adapting record package to renaming of quickcheck's structures
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn moving and renaming lazysmallcheck to narrowing which reflects the characteristical behaviour better
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn correcting dependencies in IsaMakefile
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn renaming signatures and structures; correcting header
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn adapting Quickcheck theory after moving ML files
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn moving quickcheck_generators.ML to Quickcheck directory and renaming it random_generators.ML
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn moving exhaustive_generators.ML to Quickcheck directory
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn correcting dependencies after renaming
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn replacing naming of small by exhaustive
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn renaming smallvalue_generators.ML to exhaustive_generators.ML
Fri, 11 Mar 2011 15:21:13 +0100 bulwahn renaming constants in Quickcheck_Exhaustive theory
Fri, 11 Mar 2011 15:21:12 +0100 bulwahn renaming Smallcheck to Quickcheck_Exhaustive
Fri, 11 Mar 2011 10:37:45 +0100 bulwahn only testing theory LSC_Examples when GHC is installed on the machine
Fri, 11 Mar 2011 10:37:43 +0100 bulwahn increasing timeout of example for counterexample generation
Fri, 11 Mar 2011 10:37:42 +0100 bulwahn adding termination proofs to series functions in LSC; commenting out momentarily unused term refinement functions in LSC
Fri, 11 Mar 2011 10:37:41 +0100 bulwahn adding lazysmallcheck example theory to HOL-ex session
Fri, 11 Mar 2011 10:37:40 +0100 bulwahn adding serial instance of finite_4 in lazysmallcheck; changing code equations for implies
Fri, 11 Mar 2011 10:37:38 +0100 bulwahn replacing strings in generated Code resolves the changing names of Typerep in lazysmallcheck prototype
Fri, 11 Mar 2011 10:37:37 +0100 bulwahn changing invocation of ghc from interactive mode to compilation increases the performance of lazysmallcheck by a factor of twenty; changing Integer type to Int reduces by another 50 percent
Fri, 11 Mar 2011 10:37:37 +0100 bulwahn adding an example theory for Lazysmallcheck prototype
Fri, 11 Mar 2011 10:37:36 +0100 bulwahn adding Lazysmallcheck prototype to HOL-Library
Fri, 11 Mar 2011 10:37:35 +0100 bulwahn adding files for prototype of lazysmallcheck
Fri, 11 Mar 2011 08:58:29 +0100 bulwahn removing debug message in quickcheck's postprocessor
Fri, 11 Mar 2011 08:13:00 +0100 bulwahn fixing postprocessing; adding a configuration to enable and disable pretty presentation of quickcheck's counterexample
Fri, 11 Mar 2011 08:12:59 +0100 bulwahn 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 bulwahn improving term postprocessing for counterexample presentation in quickcheck
Fri, 11 Mar 2011 08:12:55 +0100 bulwahn tuned
Wed, 09 Mar 2011 21:40:38 +0100 boehmes finished and tested Z3 proof reconstruction for injective functions;
Wed, 09 Mar 2011 10:28:01 +0100 blanchet improved formula for specialization, to prevent needless specializations -- and removed dead code
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
Fri, 04 Mar 2011 17:39:30 +0100 berghofe spark_end now joins proofs of VCs before writing *.prv file.
Fri, 04 Mar 2011 11:43:20 +0100 krauss clarified
Fri, 04 Mar 2011 11:52:54 +0100 krauss produce helpful mira summary for more errors
Fri, 04 Mar 2011 00:09:47 +0100 wenzelm eliminated prems;
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;
Thu, 03 Mar 2011 21:43:06 +0100 wenzelm tuned proofs -- eliminated prems;
Thu, 03 Mar 2011 18:43:15 +0100 wenzelm merged
Thu, 03 Mar 2011 14:38:31 +0100 blanchet merged
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
Thu, 03 Mar 2011 18:42:12 +0100 wenzelm simplified Thy_Info.check_file -- discontinued load path;
Thu, 03 Mar 2011 18:10:28 +0100 wenzelm discontinued legacy load path;
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;
Thu, 03 Mar 2011 15:46:02 +0100 wenzelm modernized imports;
Thu, 03 Mar 2011 15:36:54 +0100 wenzelm observe standard header format;
Thu, 03 Mar 2011 15:19:20 +0100 wenzelm removed spurious 'unused_thms' (cf. 1a65b780bd56);
Thu, 03 Mar 2011 15:18:05 +0100 wenzelm isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
Thu, 03 Mar 2011 11:36:10 +0100 berghofe merged
Thu, 03 Mar 2011 11:15:50 +0100 berghofe merged
Thu, 03 Mar 2011 11:01:42 +0100 berghofe - Made sure that sort_defs is aware of constants introduced by add_type_def
Thu, 03 Mar 2011 11:20:48 +0100 blanchet mention new Nitpick options
Thu, 03 Mar 2011 11:20:48 +0100 blanchet simplify "need" option's syntax
Thu, 03 Mar 2011 11:20:48 +0100 blanchet renamed "preconstr" option "need"
Thu, 03 Mar 2011 10:55:41 +0100 hoelzl finally remove upper_bound_finite_set
Thu, 03 Mar 2011 15:59:44 +1100 kleing separate settings for afp test
Wed, 02 Mar 2011 15:51:22 +0100 blanchet added missing spaces in output
Wed, 02 Mar 2011 14:50:16 +0100 blanchet lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
Wed, 02 Mar 2011 13:09:57 +0100 blanchet unfold definitions in "preconstrs" option
Wed, 02 Mar 2011 13:09:57 +0100 blanchet robust handling of types occurring in "eval" and "preconstr" options but not in the goal
Wed, 02 Mar 2011 13:09:57 +0100 blanchet make "preconstr" option more robust -- shouldn't throw exceptions
Tue, 01 Mar 2011 10:40:14 +0000 paulson merged
Mon, 28 Feb 2011 15:06:55 +0000 paulson merged
Mon, 28 Feb 2011 15:06:36 +0000 paulson declare ext [intro]: Extensionality now available by default
Mon, 28 Feb 2011 22:12:09 +0100 boehmes merged
Mon, 28 Feb 2011 22:10:57 +0100 boehmes removed dependency on Dense_Linear_Order
Mon, 28 Feb 2011 19:06:24 +0100 bulwahn adding function Quickcheck.test_terms to provide checking a batch of terms
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
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)
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"
Mon, 28 Feb 2011 17:53:10 +0100 blanchet if "total_consts" is set, report cex's as quasi-genuine
Mon, 28 Feb 2011 17:53:10 +0100 blanchet document new "total_consts" option
Mon, 28 Feb 2011 17:53:10 +0100 blanchet added "total_consts" option
Sat, 26 Feb 2011 20:40:45 +0100 nipkow added a few lemmas by Andreas Lochbihler
Sat, 26 Feb 2011 20:16:44 +0100 nipkow Corrected HOLCF/FOCUS dependency
Sat, 26 Feb 2011 17:44:42 +0100 nipkow Added material by David Trachtenherz
Sat, 26 Feb 2011 16:16:36 +0100 nipkow corrected HOLCF dependency on Nat_Infinity
Fri, 25 Feb 2011 22:07:56 +0100 nipkow got rid of lemma upper_bound_finite_set
Fri, 25 Feb 2011 20:08:00 +0100 nipkow merged
Fri, 25 Feb 2011 20:07:48 +0100 nipkow Some cleaning up
Fri, 25 Feb 2011 17:11:24 +0100 krauss updated generated files
Fri, 25 Feb 2011 17:11:05 +0100 krauss fixed manual (rule no longer exists)
Fri, 25 Feb 2011 16:59:48 +0100 krauss removed support for tail-recursion from function package (now implemented by partial_function)
Fri, 25 Feb 2011 16:57:44 +0100 krauss reactivate time measurement (partly reverting c27b0b37041a);
Fri, 25 Feb 2011 16:57:43 +0100 krauss generalize find_theorems filters to work on raw propositions, too
Fri, 25 Feb 2011 14:25:52 +0100 nipkow merged
Fri, 25 Feb 2011 14:25:41 +0100 nipkow added simp lemma nth_Cons_pos to List
Fri, 25 Feb 2011 12:16:18 +0100 noschinl Refactor find_theorems to provide a more general filter_facts method
Fri, 25 Feb 2011 08:46:52 +0100 krauss removed dead code/unused exports/speculative generality
Thu, 24 Feb 2011 21:54:28 +0100 krauss recdef -> fun(ction)
Thu, 24 Feb 2011 20:52:05 +0100 krauss removed unused lemma
Thu, 24 Feb 2011 17:54:36 +0100 krauss recdef -> fun(ction);
Thu, 24 Feb 2011 17:38:05 +0100 krauss eliminated clones of List.upto
Wed, 23 Feb 2011 17:40:28 +0100 noschinl fix non-exhaustive pattern match in find_theorems
Wed, 23 Feb 2011 11:42:01 +0100 hoelzl merged
Wed, 23 Feb 2011 11:40:18 +0100 hoelzl add lemma KL_divergence_vimage, mutual_information_generic
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip