wenzelm [Tue, 05 Apr 2011 14:25:18 +0200] rev 42224
discontinued special treatment of structure Ast: no pervasive content, no inclusion in structure Syntax;
wenzelm [Tue, 05 Apr 2011 13:07:40 +0200] rev 42223
more precise propagation of reports/results through some inner syntax layers;
misc reorganization;
wenzelm [Mon, 04 Apr 2011 23:52:56 +0200] rev 42222
accumulate parsetrees in canonical reverse order;
wenzelm [Mon, 04 Apr 2011 23:26:32 +0200] rev 42221
tuned;
wenzelm [Mon, 04 Apr 2011 22:58:15 +0200] rev 42220
tuned -- removed redundancy;
wenzelm [Mon, 04 Apr 2011 22:49:41 +0200] rev 42219
tuned signatures;
wenzelm [Mon, 04 Apr 2011 22:21:36 +0200] rev 42218
streamlined token list operations, assuming that the order of union does not matter;
wenzelm [Mon, 04 Apr 2011 21:35:59 +0200] rev 42217
misc tuning and clarification;
wenzelm [Mon, 04 Apr 2011 16:35:46 +0200] rev 42216
merged
blanchet [Mon, 04 Apr 2011 16:28:36 +0200] rev 42215
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
bulwahn [Mon, 04 Apr 2011 14:44:11 +0200] rev 42214
refactoring generator definition in quickcheck and removing clone
blanchet [Mon, 04 Apr 2011 14:37:20 +0200] rev 42213
use the proper contexts/simpsets/etc. in the TPTP proof method
blanchet [Mon, 04 Apr 2011 13:41:56 +0200] rev 42212
merged
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
paulson [Mon, 04 Apr 2011 12:40:00 +0100] rev 42210
merged
paulson [Mon, 04 Apr 2011 12:39:14 +0100] rev 42209
Deletion of all semicolons, because they interfere with Proof General
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.
haftmann [Sun, 03 Apr 2011 11:40:32 +0200] rev 42207
tuned proofs
haftmann [Sat, 02 Apr 2011 18:07:29 +0200] rev 42206
tuned proof
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;
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;
wenzelm [Sun, 03 Apr 2011 18:17:21 +0200] rev 42203
show more tooltip/sub-expression markup;
wenzelm [Sun, 03 Apr 2011 17:35:16 +0200] rev 42202
show tooltip/sub-expression for entity markup;
wenzelm [Fri, 01 Apr 2011 18:29:10 +0200] rev 42201
merged
hoelzl [Fri, 01 Apr 2011 17:20:56 +0200] rev 42200
remove unnecessary prob_preserving
hoelzl [Fri, 01 Apr 2011 17:20:33 +0200] rev 42199
add prob_space_vimage
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);
krauss [Fri, 01 Apr 2011 16:29:58 +0200] rev 42197
fixed accidental redefinition
boehmes [Fri, 01 Apr 2011 15:49:19 +0200] rev 42196
save reflexivity steps in discharging Z3 Skolemization hypotheses
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