Mon, 04 Apr 2011 14:44:11 +0200 refactoring generator definition in quickcheck and removing clone
bulwahn [Mon, 04 Apr 2011 14:44:11 +0200] rev 42214
refactoring generator definition in quickcheck and removing clone
Mon, 04 Apr 2011 14:37:20 +0200 use the proper contexts/simpsets/etc. in the TPTP proof method
blanchet [Mon, 04 Apr 2011 14:37:20 +0200] rev 42213
use the proper contexts/simpsets/etc. in the TPTP proof method
Mon, 04 Apr 2011 13:41:56 +0200 merged
blanchet [Mon, 04 Apr 2011 13:41:56 +0200] rev 42212
merged
Mon, 04 Apr 2011 13:27:34 +0200 make sure that Nitpick problem generation for cardinality 50 doesn't cause problems for lower cardinality by specifying the "batch_size" option
blanchet [Mon, 04 Apr 2011 13:27:34 +0200] rev 42211
make sure that Nitpick problem generation for cardinality 50 doesn't cause problems for lower cardinality by specifying the "batch_size" option
Mon, 04 Apr 2011 12:40:00 +0100 merged
paulson [Mon, 04 Apr 2011 12:40:00 +0100] rev 42210
merged
Mon, 04 Apr 2011 12:39:14 +0100 Deletion of all semicolons, because they interfere with Proof General
paulson [Mon, 04 Apr 2011 12:39:14 +0100] rev 42209
Deletion of all semicolons, because they interfere with Proof General
Mon, 04 Apr 2011 09:32:50 +0200 raised timeouts further, for SML/NJ -- because of variations in machines/compilers, fixed timeouts can merely prevent non-termination, not enforce particular performance characteristics.
krauss [Mon, 04 Apr 2011 09:32:50 +0200] rev 42208
raised timeouts further, for SML/NJ -- because of variations in machines/compilers, fixed timeouts can merely prevent non-termination, not enforce particular performance characteristics.
Sun, 03 Apr 2011 11:40:32 +0200 tuned proofs
haftmann [Sun, 03 Apr 2011 11:40:32 +0200] rev 42207
tuned proofs
Sat, 02 Apr 2011 18:07:29 +0200 tuned proof
haftmann [Sat, 02 Apr 2011 18:07:29 +0200] rev 42206
tuned proof
Mon, 04 Apr 2011 15:51:45 +0200 direct pretty printing of parsetrees -- prevent diagnostic output from crashing due to undeclared entities;
wenzelm [Mon, 04 Apr 2011 15:51:45 +0200] rev 42205
direct pretty printing of parsetrees -- prevent diagnostic output from crashing due to undeclared entities;
Sun, 03 Apr 2011 21:59:33 +0200 added Position.reports convenience;
wenzelm [Sun, 03 Apr 2011 21:59:33 +0200] rev 42204
added Position.reports convenience; modernized Syntax.trrule constructors; modernized Sign.add_trrules/del_trrules: internal arguments; modernized Isar_Cmd.translations/no_translations: external arguments; explicit syntax categories class_name/type_name, with reports via type_context; eliminated former class_name/type_name ast translations; tuned signatures;
Sun, 03 Apr 2011 18:17:21 +0200 show more tooltip/sub-expression markup;
wenzelm [Sun, 03 Apr 2011 18:17:21 +0200] rev 42203
show more tooltip/sub-expression markup;
Sun, 03 Apr 2011 17:35:16 +0200 show tooltip/sub-expression for entity markup;
wenzelm [Sun, 03 Apr 2011 17:35:16 +0200] rev 42202
show tooltip/sub-expression for entity markup;
Fri, 01 Apr 2011 18:29:10 +0200 merged
wenzelm [Fri, 01 Apr 2011 18:29:10 +0200] rev 42201
merged
Fri, 01 Apr 2011 17:20:56 +0200 remove unnecessary prob_preserving
hoelzl [Fri, 01 Apr 2011 17:20:56 +0200] rev 42200
remove unnecessary prob_preserving
Fri, 01 Apr 2011 17:20:33 +0200 add prob_space_vimage
hoelzl [Fri, 01 Apr 2011 17:20:33 +0200] rev 42199
add prob_space_vimage
Fri, 01 Apr 2011 17:16:08 +0200 use Unsynchronized.change convenience, which also emphasizes the raw access to these references (which happen to be local here);
wenzelm [Fri, 01 Apr 2011 17:16:08 +0200] rev 42198
use Unsynchronized.change convenience, which also emphasizes the raw access to these references (which happen to be local here);
Fri, 01 Apr 2011 16:29:58 +0200 fixed accidental redefinition
krauss [Fri, 01 Apr 2011 16:29:58 +0200] rev 42197
fixed accidental redefinition
Fri, 01 Apr 2011 15:49:19 +0200 save reflexivity steps in discharging Z3 Skolemization hypotheses
boehmes [Fri, 01 Apr 2011 15:49:19 +0200] rev 42196
save reflexivity steps in discharging Z3 Skolemization hypotheses
Fri, 01 Apr 2011 13:49:38 +0200 adding an exhaustive validator for quickcheck's batch validating; moving strip_imp; minimal setup for bounded_forall
bulwahn [Fri, 01 Apr 2011 13:49:38 +0200] rev 42195
adding an exhaustive validator for quickcheck's batch validating; moving strip_imp; minimal setup for bounded_forall
Fri, 01 Apr 2011 13:49:36 +0200 adding general interface for batch validators in quickcheck
bulwahn [Fri, 01 Apr 2011 13:49:36 +0200] rev 42194
adding general interface for batch validators in quickcheck
Fri, 01 Apr 2011 13:21:21 +0200 remove workaround 8f25605e646c, which is no longer necessary thanks to 173b0f488428
blanchet [Fri, 01 Apr 2011 13:21:21 +0200] rev 42193
remove workaround 8f25605e646c, which is no longer necessary thanks to 173b0f488428
Fri, 01 Apr 2011 12:19:54 +0200 scheduler for judgement day
krauss [Fri, 01 Apr 2011 12:19:54 +0200] rev 42192
scheduler for judgement day
Fri, 01 Apr 2011 12:16:41 +0200 re-implemented proof reconstruction for Z3 skolemization: do not explicitly construct definitions for Skolem constants, and let higher-order resolution do most of the work in the end
boehmes [Fri, 01 Apr 2011 12:16:41 +0200] rev 42191
re-implemented proof reconstruction for Z3 skolemization: do not explicitly construct definitions for Skolem constants, and let higher-order resolution do most of the work in the end
Fri, 01 Apr 2011 11:54:51 +0200 make configuration of (SMT) full monomorphization more flexible: turn boolean argument into a configuration option
boehmes [Fri, 01 Apr 2011 11:54:51 +0200] rev 42190
make configuration of (SMT) full monomorphization more flexible: turn boolean argument into a configuration option
Fri, 01 Apr 2011 10:18:20 +0200 merged
bulwahn [Fri, 01 Apr 2011 10:18:20 +0200] rev 42189
merged
Fri, 01 Apr 2011 09:20:59 +0200 adding time profiling in quickcheck's batch testing for further diagnosis in IsaCoSy
bulwahn [Fri, 01 Apr 2011 09:20:59 +0200] rev 42188
adding time profiling in quickcheck's batch testing for further diagnosis in IsaCoSy
Fri, 01 Apr 2011 09:48:01 +0200 raised timeouts further, for SML/NJ
krauss [Fri, 01 Apr 2011 09:48:01 +0200] rev 42187
raised timeouts further, for SML/NJ
Fri, 01 Apr 2011 09:29:58 +0200 adapted parsing of session timing (cf. e86b10c68f0b)
krauss [Fri, 01 Apr 2011 09:29:58 +0200] rev 42186
adapted parsing of session timing (cf. e86b10c68f0b)
Thu, 31 Mar 2011 17:15:13 +0200 merged
bulwahn [Thu, 31 Mar 2011 17:15:13 +0200] rev 42185
merged
Thu, 31 Mar 2011 11:17:52 +0200 adapting Quickcheck_Narrowing (overseen in 234ec7011e5d); commenting out some examples temporarily
bulwahn [Thu, 31 Mar 2011 11:17:52 +0200] rev 42184
adapting Quickcheck_Narrowing (overseen in 234ec7011e5d); commenting out some examples temporarily
Thu, 31 Mar 2011 14:02:03 +0200 provide a flag controlling whether all provided facts should be instantiated, possibly inventing new types (which does not work well with Sledgehammer)
boehmes [Thu, 31 Mar 2011 14:02:03 +0200] rev 42183
provide a flag controlling whether all provided facts should be instantiated, possibly inventing new types (which does not work well with Sledgehammer)
Thu, 31 Mar 2011 11:16:54 +0200 start monomorphization process with subgoal, not entire goal, to avoid needless instances (and only print monomorphization messages in debug mode)
blanchet [Thu, 31 Mar 2011 11:16:54 +0200] rev 42182
start monomorphization process with subgoal, not entire goal, to avoid needless instances (and only print monomorphization messages in debug mode)
Thu, 31 Mar 2011 11:16:53 +0200 temporary workaround: filter out spurious monomorphic instances
blanchet [Thu, 31 Mar 2011 11:16:53 +0200] rev 42181
temporary workaround: filter out spurious monomorphic instances
Thu, 31 Mar 2011 11:16:52 +0200 added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default
blanchet [Thu, 31 Mar 2011 11:16:52 +0200] rev 42180
added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default
Thu, 31 Mar 2011 11:16:51 +0200 added support for "dest:" to "try"
blanchet [Thu, 31 Mar 2011 11:16:51 +0200] rev 42179
added support for "dest:" to "try"
Thu, 31 Mar 2011 09:43:36 +0200 corrected infix precedence for boolean operators in Haskell
haftmann [Thu, 31 Mar 2011 09:43:36 +0200] rev 42178
corrected infix precedence for boolean operators in Haskell
Thu, 31 Mar 2011 08:28:03 +0200 merged
bulwahn [Thu, 31 Mar 2011 08:28:03 +0200] rev 42177
merged
Wed, 30 Mar 2011 19:09:57 +0200 removing dead code in exhaustive_generators
bulwahn [Wed, 30 Mar 2011 19:09:57 +0200] rev 42176
removing dead code in exhaustive_generators
Wed, 30 Mar 2011 19:09:56 +0200 removing junk that should not have been committed
bulwahn [Wed, 30 Mar 2011 19:09:56 +0200] rev 42175
removing junk that should not have been committed
Wed, 30 Mar 2011 23:26:40 +0200 modernized specifications;
wenzelm [Wed, 30 Mar 2011 23:26:40 +0200] rev 42174
modernized specifications;
Wed, 30 Mar 2011 22:53:18 +0200 accomodate autofix discipline of non-body context;
wenzelm [Wed, 30 Mar 2011 22:53:18 +0200] rev 42173
accomodate autofix discipline of non-body context;
Wed, 30 Mar 2011 22:45:10 +0200 session timing: show pseudo-speedup factor;
wenzelm [Wed, 30 Mar 2011 22:45:10 +0200] rev 42172
session timing: show pseudo-speedup factor;
Wed, 30 Mar 2011 22:06:25 +0200 visualize skolem and hilite (undeclared frees);
wenzelm [Wed, 30 Mar 2011 22:06:25 +0200] rev 42171
visualize skolem and hilite (undeclared frees); tuned colors;
Wed, 30 Mar 2011 22:03:50 +0200 more informative markup_free;
wenzelm [Wed, 30 Mar 2011 22:03:50 +0200] rev 42170
more informative markup_free;
Wed, 30 Mar 2011 21:07:48 +0200 inline lemmas instead of accidental physical addressing -- explicit is better than implicit;
wenzelm [Wed, 30 Mar 2011 21:07:48 +0200] rev 42169
inline lemmas instead of accidental physical addressing -- explicit is better than implicit;
Wed, 30 Mar 2011 20:21:40 +0200 tuned white space and indentation;
wenzelm [Wed, 30 Mar 2011 20:21:40 +0200] rev 42168
tuned white space and indentation; observe strict line length limitation (80-100 chars);
Wed, 30 Mar 2011 20:19:21 +0200 actually check list comprehension examples;
wenzelm [Wed, 30 Mar 2011 20:19:21 +0200] rev 42167
actually check list comprehension examples;
Wed, 30 Mar 2011 17:54:10 +0200 products of probability measures are probability measures
hoelzl [Wed, 30 Mar 2011 17:54:10 +0200] rev 42166
products of probability measures are probability measures
Wed, 30 Mar 2011 17:54:01 +0200 real multiplication is continuous
hoelzl [Wed, 30 Mar 2011 17:54:01 +0200] rev 42165
real multiplication is continuous
Wed, 30 Mar 2011 17:53:56 +0200 add lebesgue_real_affine
hoelzl [Wed, 30 Mar 2011 17:53:56 +0200] rev 42164
add lebesgue_real_affine
Wed, 30 Mar 2011 11:32:52 +0200 renewing specifications in HOL: replacing types by type_synonym
bulwahn [Wed, 30 Mar 2011 11:32:52 +0200] rev 42163
renewing specifications in HOL: replacing types by type_synonym
Wed, 30 Mar 2011 11:32:51 +0200 moved TimeLimit.timeLimit closure to limit time of compilation and execution to avoid the strange, occasional occuring message Exception trace for exception - Interrupt -- probably due to race conditions of a fast execution within the TimeLimit.timelimit closure
bulwahn [Wed, 30 Mar 2011 11:32:51 +0200] rev 42162
moved TimeLimit.timeLimit closure to limit time of compilation and execution to avoid the strange, occasional occuring message Exception trace for exception - Interrupt -- probably due to race conditions of a fast execution within the TimeLimit.timelimit closure
Wed, 30 Mar 2011 10:31:02 +0200 adding a regression test for SML_Quickcheck; putting SML_Quickcheck back in shape
bulwahn [Wed, 30 Mar 2011 10:31:02 +0200] rev 42161
adding a regression test for SML_Quickcheck; putting SML_Quickcheck back in shape
Wed, 30 Mar 2011 09:44:17 +0200 NEWS
bulwahn [Wed, 30 Mar 2011 09:44:17 +0200] rev 42160
NEWS
Wed, 30 Mar 2011 09:44:16 +0200 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
bulwahn [Wed, 30 Mar 2011 09:44:16 +0200] rev 42159
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
Tue, 29 Mar 2011 23:46:46 +0200 merged
wenzelm [Tue, 29 Mar 2011 23:46:46 +0200] rev 42158
merged
Tue, 29 Mar 2011 22:06:53 +0200 added missing smlnj target
krauss [Tue, 29 Mar 2011 22:06:53 +0200] rev 42157
added missing smlnj target
Tue, 29 Mar 2011 23:27:38 +0200 modernized specifications -- less axioms;
wenzelm [Tue, 29 Mar 2011 23:27:38 +0200] rev 42156
modernized specifications -- less axioms;
Tue, 29 Mar 2011 23:15:25 +0200 modernized specifications -- some attempts to avoid wild axiomatizations;
wenzelm [Tue, 29 Mar 2011 23:15:25 +0200] rev 42155
modernized specifications -- some attempts to avoid wild axiomatizations; comp: retain infix \<circ> to retain type "o" from FOL; tuned proofs;
Tue, 29 Mar 2011 22:36:56 +0200 tuned proofs;
wenzelm [Tue, 29 Mar 2011 22:36:56 +0200] rev 42154
tuned proofs;
Tue, 29 Mar 2011 21:48:01 +0200 use shared copy of hoare_syntax.ML;
wenzelm [Tue, 29 Mar 2011 21:48:01 +0200] rev 42153
use shared copy of hoare_syntax.ML; misc tuning;
Tue, 29 Mar 2011 21:11:02 +0200 Hoare syntax: standard abstraction syntax admits source positions;
wenzelm [Tue, 29 Mar 2011 21:11:02 +0200] rev 42152
Hoare syntax: standard abstraction syntax admits source positions; re-unified some clones (!);
Tue, 29 Mar 2011 17:47:11 +0200 tuned headers;
wenzelm [Tue, 29 Mar 2011 17:47:11 +0200] rev 42151
tuned headers;
Tue, 29 Mar 2011 17:30:26 +0200 tuned headers;
wenzelm [Tue, 29 Mar 2011 17:30:26 +0200] rev 42150
tuned headers;
Tue, 29 Mar 2011 14:27:44 +0200 NEWS
hoelzl [Tue, 29 Mar 2011 14:27:44 +0200] rev 42149
NEWS
Tue, 29 Mar 2011 14:27:42 +0200 rename Probability_Space to Probability_Measure
hoelzl [Tue, 29 Mar 2011 14:27:42 +0200] rev 42148
rename Probability_Space to Probability_Measure
Tue, 29 Mar 2011 14:27:41 +0200 add infinite product measure
hoelzl [Tue, 29 Mar 2011 14:27:41 +0200] rev 42147
add infinite product measure
Tue, 29 Mar 2011 14:27:39 +0200 split Product_Measure into Binary_Product_Measure and Finite_Product_Measure
hoelzl [Tue, 29 Mar 2011 14:27:39 +0200] rev 42146
split Product_Measure into Binary_Product_Measure and Finite_Product_Measure
Tue, 29 Mar 2011 14:27:31 +0200 proved caratheodory_empty_continuous
hoelzl [Tue, 29 Mar 2011 14:27:31 +0200] rev 42145
proved caratheodory_empty_continuous
Mon, 28 Mar 2011 23:49:53 +0200 list comprehension: strip positions where the translation cannot handle them right now;
wenzelm [Mon, 28 Mar 2011 23:49:53 +0200] rev 42144
list comprehension: strip positions where the translation cannot handle them right now;
Mon, 28 Mar 2011 22:44:14 +0200 address serious problem of type inference (introduced in 6f085332c7d3): _type_constraint_ needs type scheme A --> A with proper scope of parameters, otherwise term "(f :: _ => _) :: 'c => 'c" will get type "'a => 'b", for example;
wenzelm [Mon, 28 Mar 2011 22:44:14 +0200] rev 42143
address serious problem of type inference (introduced in 6f085332c7d3): _type_constraint_ needs type scheme A --> A with proper scope of parameters, otherwise term "(f :: _ => _) :: 'c => 'c" will get type "'a => 'b", for example;
Mon, 28 Mar 2011 17:33:16 +0200 raised various timeouts to accommodate sluggish SML/NJ
krauss [Mon, 28 Mar 2011 17:33:16 +0200] rev 42142
raised various timeouts to accommodate sluggish SML/NJ
Mon, 28 Mar 2011 10:25:28 +0200 changing values_timeout from a static option to a dynamic option as required for testing with SML/NJ
bulwahn [Mon, 28 Mar 2011 10:25:28 +0200] rev 42141
changing values_timeout from a static option to a dynamic option as required for testing with SML/NJ
Mon, 28 Mar 2011 09:22:22 +0200 keep smlnj HOL images around
krauss [Mon, 28 Mar 2011 09:22:22 +0200] rev 42140
keep smlnj HOL images around
Sun, 27 Mar 2011 21:44:10 +0200 merged
wenzelm [Sun, 27 Mar 2011 21:44:10 +0200] rev 42139
merged
Sun, 27 Mar 2011 17:32:25 +0200 added make target 'smlnj' to refer to what can/should be tested using smlnj -- allows the use of "isabelle makeall smlnj";
krauss [Sun, 27 Mar 2011 17:32:25 +0200] rev 42138
added make target 'smlnj' to refer to what can/should be tested using smlnj -- allows the use of "isabelle makeall smlnj"; adapted test configuration SML_makeall
Sun, 27 Mar 2011 16:56:16 +0200 avoid *** in normal output, which usually marks errors in logs
krauss [Sun, 27 Mar 2011 16:56:16 +0200] rev 42137
avoid *** in normal output, which usually marks errors in logs
Sun, 27 Mar 2011 21:19:23 +0200 added Markup.Name and Markup.Kind convenience;
wenzelm [Sun, 27 Mar 2011 21:19:23 +0200] rev 42136
added Markup.Name and Markup.Kind convenience; token_style for entity kind markup;
Sun, 27 Mar 2011 20:55:01 +0200 decode_term: some context-sensitive markup;
wenzelm [Sun, 27 Mar 2011 20:55:01 +0200] rev 42135
decode_term: some context-sensitive markup; more informative Markup.entity and Name_Space.markup_entry; Markup.const: use "constant" to make it coincide with name space kind;
Sun, 27 Mar 2011 19:51:51 +0200 tuned signatures;
wenzelm [Sun, 27 Mar 2011 19:51:51 +0200] rev 42134
tuned signatures;
Sun, 27 Mar 2011 19:27:31 +0200 decode_term: more precise reports;
wenzelm [Sun, 27 Mar 2011 19:27:31 +0200] rev 42133
decode_term: more precise reports;
Sun, 27 Mar 2011 18:12:18 +0200 adhoc token style for free/bound;
wenzelm [Sun, 27 Mar 2011 18:12:18 +0200] rev 42132
adhoc token style for free/bound;
Sun, 27 Mar 2011 17:55:11 +0200 decode_term/disambig: report resolved term variables for the unique (!) result;
wenzelm [Sun, 27 Mar 2011 17:55:11 +0200] rev 42131
decode_term/disambig: report resolved term variables for the unique (!) result;
Sun, 27 Mar 2011 15:01:47 +0200 removed unclear comments stemming from ed24ba6f69aa;
wenzelm [Sun, 27 Mar 2011 15:01:47 +0200] rev 42130
removed unclear comments stemming from ed24ba6f69aa;
Sat, 26 Mar 2011 21:45:29 +0100 present theory content as future, depending on intermediate proof state futures -- potential to reduce memory requirements and improve parallelization;
wenzelm [Sat, 26 Mar 2011 21:45:29 +0100] rev 42129
present theory content as future, depending on intermediate proof state futures -- potential to reduce memory requirements and improve parallelization;
Sat, 26 Mar 2011 21:28:04 +0100 added Future.cond_forks convenience;
wenzelm [Sat, 26 Mar 2011 21:28:04 +0100] rev 42128
added Future.cond_forks convenience;
Sat, 26 Mar 2011 18:31:39 +0100 Isabelle_System.create_tmp_path/with_tmp_file: optional extension;
wenzelm [Sat, 26 Mar 2011 18:31:39 +0100] rev 42127
Isabelle_System.create_tmp_path/with_tmp_file: optional extension; thread-safe versions of Present.display_graph, Present.isabelle_browser, Present.drafts -- using Isabelle_System.with_tmp_dir;
Sat, 26 Mar 2011 19:16:30 +0100 tuned;
wenzelm [Sat, 26 Mar 2011 19:16:30 +0100] rev 42126
tuned;
Sat, 26 Mar 2011 19:16:20 +0100 more direct loose_bvar1;
wenzelm [Sat, 26 Mar 2011 19:16:20 +0100] rev 42125
more direct loose_bvar1; tuned; slight re-unification of clone (cf. 47f8bfe0f597);
Sat, 26 Mar 2011 16:21:41 +0100 suppress Mercurial backup files;
wenzelm [Sat, 26 Mar 2011 16:21:41 +0100] rev 42124
suppress Mercurial backup files; uniform treatment of tool filtering in bash/perl/scala;
Sat, 26 Mar 2011 16:10:22 +0100 updated generated file;
wenzelm [Sat, 26 Mar 2011 16:10:22 +0100] rev 42123
updated generated file; tuned whitespace;
Sat, 26 Mar 2011 15:55:22 +0100 merged
wenzelm [Sat, 26 Mar 2011 15:55:22 +0100] rev 42122
merged
Sat, 26 Mar 2011 00:23:20 +0100 SML_makeall: run with -j 3
krauss [Sat, 26 Mar 2011 00:23:20 +0100] rev 42121
SML_makeall: run with -j 3
Fri, 25 Mar 2011 22:17:32 +0100 fixed incomplete rename (1cdf54e845fa)
krauss [Fri, 25 Mar 2011 22:17:32 +0100] rev 42120
fixed incomplete rename (1cdf54e845fa)
Fri, 25 Mar 2011 21:38:41 +0100 eliminated hardwired MUTABELLE_OUTPUT_PATH (cf. 6a147393c62a)
krauss [Fri, 25 Mar 2011 21:38:41 +0100] rev 42119
eliminated hardwired MUTABELLE_OUTPUT_PATH (cf. 6a147393c62a)
Fri, 25 Mar 2011 17:09:21 +0100 merged
bulwahn [Fri, 25 Mar 2011 17:09:21 +0100] rev 42118
merged
Fri, 25 Mar 2011 16:03:49 +0100 changing iteration scheme of functions to use minimal number of function updates for exhaustive testing
bulwahn [Fri, 25 Mar 2011 16:03:49 +0100] rev 42117
changing iteration scheme of functions to use minimal number of function updates for exhaustive testing
Thu, 24 Mar 2011 23:42:06 +0100 added configurations SML_HOL and SML_makeall (even though the latter is practically infeasible)
krauss [Thu, 24 Mar 2011 23:42:06 +0100] rev 42116
added configurations SML_HOL and SML_makeall (even though the latter is practically infeasible)
Thu, 24 Mar 2011 23:35:49 +0100 mira interface to 'isabelle make' in addition to usedir and makeall;
krauss [Thu, 24 Mar 2011 23:35:49 +0100] rev 42115
mira interface to 'isabelle make' in addition to usedir and makeall; do not require dependencies
Thu, 24 Mar 2011 23:28:07 +0100 clarified
krauss [Thu, 24 Mar 2011 23:28:07 +0100] rev 42114
clarified
Thu, 24 Mar 2011 23:14:49 +0100 parameterize configurations by custom settings
krauss [Thu, 24 Mar 2011 23:14:49 +0100] rev 42113
parameterize configurations by custom settings
Fri, 25 Mar 2011 15:22:09 +0100 Change coercion for RealDef to use function application (not composition)
noschinl [Fri, 25 Mar 2011 15:22:09 +0100] rev 42112
Change coercion for RealDef to use function application (not composition)
Fri, 25 Mar 2011 11:19:01 +0100 revisiting Code_Prolog (cf. 6fe4abb9437b)
bulwahn [Fri, 25 Mar 2011 11:19:01 +0100] rev 42111
revisiting Code_Prolog (cf. 6fe4abb9437b)
Fri, 25 Mar 2011 11:19:00 +0100 fixed postprocessing for term presentation in quickcheck; tuned spacing
bulwahn [Fri, 25 Mar 2011 11:19:00 +0100] rev 42110
fixed postprocessing for term presentation in quickcheck; tuned spacing
Thu, 24 Mar 2011 22:12:38 +0100 enable Z3 in the test configuration
krauss [Thu, 24 Mar 2011 22:12:38 +0100] rev 42109
enable Z3 in the test configuration
Thu, 24 Mar 2011 17:56:59 +0100 add "-?" to "nitrox" tool
blanchet [Thu, 24 Mar 2011 17:56:59 +0100] rev 42108
add "-?" to "nitrox" tool
Thu, 24 Mar 2011 17:49:27 +0100 clean up new Skolemizer code -- some old hacks are no longer necessary
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42107
clean up new Skolemizer code -- some old hacks are no longer necessary
Thu, 24 Mar 2011 17:49:27 +0100 specify proper defaults for Nitpick and Refute on TPTP + tuning
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42106
specify proper defaults for Nitpick and Refute on TPTP + tuning
Thu, 24 Mar 2011 17:49:27 +0100 added "nitrox" tool (Nitpick for first-order TPTP problems) to components
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42105
added "nitrox" tool (Nitpick for first-order TPTP problems) to components
Thu, 24 Mar 2011 17:49:27 +0100 made one more Metis example use the new Skolemizer
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42104
made one more Metis example use the new Skolemizer
Thu, 24 Mar 2011 17:49:27 +0100 Metis examples use the new Skolemizer to test it
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42103
Metis examples use the new Skolemizer to test it
Thu, 24 Mar 2011 17:49:27 +0100 new version of Metis 2.3 (29 Dec. 2010)
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42102
new version of Metis 2.3 (29 Dec. 2010)
Thu, 24 Mar 2011 17:49:27 +0100 remove newly added wrong logic
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42101
remove newly added wrong logic
Thu, 24 Mar 2011 17:49:27 +0100 more precise failure reporting in Sledgehammer/SMT
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42100
more precise failure reporting in Sledgehammer/SMT
Thu, 24 Mar 2011 17:49:27 +0100 avoid evil "export_without_context", which breaks if there are local "fixes"
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42099
avoid evil "export_without_context", which breaks if there are local "fixes"
Thu, 24 Mar 2011 17:49:27 +0100 more robust handling of variables in new Skolemizer
blanchet [Thu, 24 Mar 2011 17:49:27 +0100] rev 42098
more robust handling of variables in new Skolemizer
Thu, 24 Mar 2011 17:10:23 +0100 merged
haftmann [Thu, 24 Mar 2011 17:10:23 +0100] rev 42097
merged
Thu, 24 Mar 2011 17:10:13 +0100 added subsection on Scala specialities
haftmann [Thu, 24 Mar 2011 17:10:13 +0100] rev 42096
added subsection on Scala specialities
Thu, 24 Mar 2011 16:39:37 +0100 added more judgement day provers
krauss [Thu, 24 Mar 2011 16:39:37 +0100] rev 42095
added more judgement day provers
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip