src/HOL/Tools/Quickcheck/quickcheck_common.ML
Wed, 03 Sep 2014 00:06:17 +0200 blanchet ported Quickcheck to support new datatypes better
Mon, 01 Sep 2014 16:17:46 +0200 blanchet renamed modules defining old datatypes, as a step towards having 'datatype_new' take 'datatype's place
Tue, 19 Aug 2014 09:39:11 +0200 blanchet reduced dependency on 'Datatype' theory and ML module
Thu, 03 Apr 2014 10:51:22 +0200 blanchet use same idiom as used for datatype 'size' function to name constants and theorems emerging from various type interpretations -- reduces the chances of name clashes on theory merges
Wed, 27 Mar 2013 14:50:30 +0100 wenzelm clarified Skip_Proof.cheat_tac: more standard tactic;
Fri, 15 Feb 2013 08:31:31 +0100 haftmann two target language numeral types: integer and natural, as replacement for code_numeral;
Thu, 14 Feb 2013 15:27:10 +0100 haftmann reform of predicate compiler / quickcheck theories:
Sun, 11 Nov 2012 19:56:02 +0100 haftmann dropped dead code;
Mon, 16 Jul 2012 21:20:56 +0200 wenzelm more direct Sorts.has_instance;
Fri, 30 Mar 2012 08:19:31 +0200 bulwahn refine bindings in quickcheck_common: do not conceal and do not declare as simps
Sat, 25 Feb 2012 09:07:53 +0100 bulwahn slightly changing the enumeration scheme
Tue, 21 Feb 2012 20:43:58 +0100 wenzelm made SML/NJ happy;
Tue, 21 Feb 2012 12:20:33 +0100 bulwahn subtype preprocessing in Quickcheck;
Tue, 14 Feb 2012 17:58:51 +0100 bulwahn adding abort_potential functionality in quickcheck
Wed, 25 Jan 2012 15:19:04 +0100 bulwahn generalizing check if size matters because it is different for random and exhaustive testing
Tue, 24 Jan 2012 09:13:24 +0100 bulwahn adding some rules to quickcheck's preprocessing
Mon, 23 Jan 2012 14:06:19 +0100 bulwahn adding fun_eq_iff to the preprocessing
Tue, 20 Dec 2011 17:22:31 +0100 bulwahn generalize ensure_sort_datatype to ensure_sort in quickcheck_common to allow generators for abstract types;
Tue, 20 Dec 2011 14:43:41 +0100 bulwahn tuned
Mon, 12 Dec 2011 17:22:48 +0100 bulwahn tuned quickcheck's response
Fri, 09 Dec 2011 12:21:01 +0100 bulwahn tuned quickcheck's response
Mon, 05 Dec 2011 12:36:22 +0100 bulwahn making the default behaviour of quickcheck a little bit less verbose;
Mon, 05 Dec 2011 12:36:20 +0100 bulwahn random reporting compilation returns if counterexample is genuine or potentially spurious, and takes genuine_only option as argument
Mon, 05 Dec 2011 12:36:06 +0100 bulwahn exhaustive returns if a counterexample is genuine or potentially spurious in the presence of assumptions more correctly
Mon, 05 Dec 2011 12:36:00 +0100 bulwahn renaming potential flag to genuine_only flag with an inverse semantics
Mon, 05 Dec 2011 12:35:06 +0100 bulwahn outputing the potentially spurious counterexample and continue search
Mon, 05 Dec 2011 12:35:05 +0100 bulwahn dynamic genuine_flag in compilation of random and exhaustive
Mon, 05 Dec 2011 12:35:04 +0100 bulwahn indicating where the restart should occur; making safe_if dynamic
Thu, 01 Dec 2011 22:14:35 +0100 bulwahn compilations return genuine flag to quickcheck framework
Thu, 01 Dec 2011 22:14:35 +0100 bulwahn the simple exhaustive compilation also indicates if counterexample is potentially spurious;
Thu, 01 Dec 2011 22:14:35 +0100 bulwahn quickcheck's compilation returns if it is genuine counterexample or a counterexample due to a match exception
Thu, 01 Dec 2011 22:14:35 +0100 bulwahn removing exception handling now that is caught at some other point;
Thu, 01 Dec 2011 22:14:35 +0100 bulwahn quickcheck random can also find potential counterexamples;
Wed, 30 Nov 2011 09:21:18 +0100 bulwahn quickcheck does not show evaluation terms of equations if they are simply free variables to avoid duplicated output; tuned
Wed, 30 Nov 2011 09:21:15 +0100 bulwahn adding more verbose messages to exhaustive quickcheck
Fri, 25 Nov 2011 19:07:26 +0100 krauss removed obsolete uses of Local_Theory.restore -- package composition P1 #> P2 no longer requires them due to 57def0b39696: P2 finds the results of P1 in the auxiliary context
Sat, 19 Nov 2011 21:18:38 +0100 wenzelm added ML antiquotation @{attributes};
Thu, 10 Nov 2011 17:26:15 +0100 bulwahn adding a minimalistic preprocessing rewriting common boolean operators; tuned
Wed, 09 Nov 2011 11:35:09 +0100 bulwahn more precise messages with the tester's name in quickcheck; tuned
Wed, 09 Nov 2011 11:34:59 +0100 bulwahn quickcheck fails with code generator errors only if one tester is invoked
Wed, 09 Nov 2011 11:34:57 +0100 bulwahn removing extra arguments
Wed, 09 Nov 2011 11:34:55 +0100 bulwahn removing deactivated timeout handling; catching compilation errors and only outputing an urgent message to enable parallel sucessful quickcheck compilations and runs to present their result
Wed, 09 Nov 2011 11:34:53 +0100 bulwahn tuned
Mon, 17 Oct 2011 10:19:01 +0200 bulwahn moving some common functions from quickcheck to the more HOL-specific quickcheck_common; renamed inductive_SML's configurations to more canonical names; adds automatically left and right hand sides of equations as evaluation terms
Thu, 22 Sep 2011 07:26:53 +0200 bulwahn adding post-processing of terms to narrowing-based Quickcheck
Wed, 17 Aug 2011 18:05:31 +0200 wenzelm modernized signature of Term.absfree/absdummy;
Fri, 13 May 2011 22:55:00 +0200 wenzelm proper Proof.context for classical tactics;
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Fri, 08 Apr 2011 14:20:57 +0200 wenzelm discontinued special treatment of structure Mixfix;
Tue, 05 Apr 2011 08:53:52 +0200 bulwahn generalizing ensure_sort_datatype for bounded_forall instances
Mon, 04 Apr 2011 14:44:11 +0200 bulwahn refactoring generator definition in quickcheck and removing clone
Fri, 01 Apr 2011 13:49:38 +0200 bulwahn adding an exhaustive validator for quickcheck's batch validating; moving strip_imp; minimal setup for bounded_forall
Wed, 30 Mar 2011 09:44:16 +0200 bulwahn generalizing compilation scheme of quickcheck generators to multiple arguments; changing random and exhaustive tester to use one code invocation for polymorphic instances with multiple cardinalities
Fri, 25 Mar 2011 11:19:00 +0100 bulwahn fixed postprocessing for term presentation in quickcheck; tuned spacing
Sun, 13 Mar 2011 13:53:54 +0100 wenzelm tuned headers;
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 adding file quickcheck_common to carry common functions of all quickcheck generators
less more (0) tip