Wed, 03 Nov 2010 10:51:40 +0100 try_param_tac: plain user error appears more appropriate;
wenzelm [Wed, 03 Nov 2010 10:51:40 +0100] rev 40315
try_param_tac: plain user error appears more appropriate;
Wed, 03 Nov 2010 10:48:55 +0100 replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
wenzelm [Wed, 03 Nov 2010 10:48:55 +0100] rev 40314
replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
Wed, 03 Nov 2010 10:20:37 +0100 eliminated dead code;
wenzelm [Wed, 03 Nov 2010 10:20:37 +0100] rev 40313
eliminated dead code;
Wed, 03 Nov 2010 10:18:05 +0100 more conventional exceptions for abstract syntax operations -- eliminated ancient SYS_ERROR;
wenzelm [Wed, 03 Nov 2010 10:18:05 +0100] rev 40312
more conventional exceptions for abstract syntax operations -- eliminated ancient SYS_ERROR; proper signature constraint;
Wed, 03 Nov 2010 08:29:32 +0100 removed assumption
nipkow [Wed, 03 Nov 2010 08:29:32 +0100] rev 40311
removed assumption
Tue, 02 Nov 2010 21:59:21 +0100 more on naming tactics;
wenzelm [Tue, 02 Nov 2010 21:59:21 +0100] rev 40310
more on naming tactics;
Tue, 02 Nov 2010 21:24:07 +0100 merged
wenzelm [Tue, 02 Nov 2010 21:24:07 +0100] rev 40309
merged
Tue, 02 Nov 2010 20:32:33 +0100 merged
haftmann [Tue, 02 Nov 2010 20:32:33 +0100] rev 40308
merged
Tue, 02 Nov 2010 16:59:40 +0100 tuned proof
haftmann [Tue, 02 Nov 2010 16:59:40 +0100] rev 40307
tuned proof
Tue, 02 Nov 2010 16:48:19 +0100 tuned proof
haftmann [Tue, 02 Nov 2010 16:48:19 +0100] rev 40306
tuned proof
Tue, 02 Nov 2010 16:36:33 +0100 tuned lemma proposition of properties_for_sort_key
haftmann [Tue, 02 Nov 2010 16:36:33 +0100] rev 40305
tuned lemma proposition of properties_for_sort_key
Tue, 02 Nov 2010 16:31:57 +0100 lemmas sorted_map_same, sorted_same
haftmann [Tue, 02 Nov 2010 16:31:57 +0100] rev 40304
lemmas sorted_map_same, sorted_same
Tue, 02 Nov 2010 16:31:56 +0100 lemmas multiset_of_filter, sort_key_by_quicksort
haftmann [Tue, 02 Nov 2010 16:31:56 +0100] rev 40303
lemmas multiset_of_filter, sort_key_by_quicksort
Tue, 02 Nov 2010 21:21:07 +0100 more on "Time" in Isabelle/ML;
wenzelm [Tue, 02 Nov 2010 21:21:07 +0100] rev 40302
more on "Time" in Isabelle/ML;
Tue, 02 Nov 2010 20:55:12 +0100 simplified some time constants;
wenzelm [Tue, 02 Nov 2010 20:55:12 +0100] rev 40301
simplified some time constants;
Tue, 02 Nov 2010 20:31:46 +0100 added convenience operation seconds: real -> time;
wenzelm [Tue, 02 Nov 2010 20:31:46 +0100] rev 40300
added convenience operation seconds: real -> time;
Tue, 02 Nov 2010 20:16:56 +0100 avoid catch-all exception handling;
wenzelm [Tue, 02 Nov 2010 20:16:56 +0100] rev 40299
avoid catch-all exception handling;
Tue, 02 Nov 2010 20:15:57 +0100 eliminated fragile catch-all pattern, based on educated guess about the intended exception;
wenzelm [Tue, 02 Nov 2010 20:15:57 +0100] rev 40298
eliminated fragile catch-all pattern, based on educated guess about the intended exception;
Tue, 02 Nov 2010 12:37:12 +0100 Attribute map_function -> coercion_map;
traytel [Tue, 02 Nov 2010 12:37:12 +0100] rev 40297
Attribute map_function -> coercion_map; tuned;
Sun, 31 Oct 2010 13:26:37 +0100 syntax category "real" subsumes plain "int";
wenzelm [Sun, 31 Oct 2010 13:26:37 +0100] rev 40296
syntax category "real" subsumes plain "int";
Sun, 31 Oct 2010 11:45:45 +0100 merged
nipkow [Sun, 31 Oct 2010 11:45:45 +0100] rev 40295
merged
Fri, 29 Oct 2010 17:57:36 +0200 Plus -> Sum_Type.Plus
nipkow [Fri, 29 Oct 2010 17:57:36 +0200] rev 40294
Plus -> Sum_Type.Plus
Sun, 31 Oct 2010 11:38:09 +0100 Minor reformat.
ballarin [Sun, 31 Oct 2010 11:38:09 +0100] rev 40293
Minor reformat.
Sat, 30 Oct 2010 21:08:20 +0200 support for real valued preferences;
wenzelm [Sat, 30 Oct 2010 21:08:20 +0200] rev 40292
support for real valued preferences;
Sat, 30 Oct 2010 16:33:58 +0200 support for real valued configuration options;
wenzelm [Sat, 30 Oct 2010 16:33:58 +0200] rev 40291
support for real valued configuration options;
Sat, 30 Oct 2010 15:26:40 +0200 support for floating-point tokens in outer syntax (coinciding with inner syntax version);
wenzelm [Sat, 30 Oct 2010 15:26:40 +0200] rev 40290
support for floating-point tokens in outer syntax (coinciding with inner syntax version);
Fri, 29 Oct 2010 23:15:01 +0200 merged
wenzelm [Fri, 29 Oct 2010 23:15:01 +0200] rev 40289
merged
Fri, 29 Oct 2010 21:41:14 +0200 added rule let_mono
krauss [Fri, 29 Oct 2010 21:41:14 +0200] rev 40288
added rule let_mono
Fri, 29 Oct 2010 22:59:40 +0200 CONTRIBUTORS;
wenzelm [Fri, 29 Oct 2010 22:59:40 +0200] rev 40287
CONTRIBUTORS;
Fri, 29 Oct 2010 22:54:54 +0200 more sharing of operations, without aliases;
wenzelm [Fri, 29 Oct 2010 22:54:54 +0200] rev 40286
more sharing of operations, without aliases;
Fri, 29 Oct 2010 22:22:36 +0200 simplified data lookup;
wenzelm [Fri, 29 Oct 2010 22:22:36 +0200] rev 40285
simplified data lookup;
Fri, 29 Oct 2010 22:19:27 +0200 export declarations by default, to allow other ML packages by-pass concrete syntax;
wenzelm [Fri, 29 Oct 2010 22:19:27 +0200] rev 40284
export declarations by default, to allow other ML packages by-pass concrete syntax; proper Args parsing for attribute syntax (required for proper treatment of morphisms when declarations are moved between contexts); tuned;
Fri, 29 Oct 2010 22:07:48 +0200 proper signature constraint for ML structure;
wenzelm [Fri, 29 Oct 2010 22:07:48 +0200] rev 40283
proper signature constraint for ML structure; explicit theory setup, which is customary outside Pure; formal @{binding} instead of Binding.name;
Fri, 29 Oct 2010 21:49:33 +0200 proper header;
wenzelm [Fri, 29 Oct 2010 21:49:33 +0200] rev 40282
proper header; tuned whitespace;
Fri, 29 Oct 2010 21:34:07 +0200 Coercive subtyping via subtype constraints, by Dmitriy Traytel (21-Oct-2010).
wenzelm [Fri, 29 Oct 2010 21:34:07 +0200] rev 40281
Coercive subtyping via subtype constraints, by Dmitriy Traytel (21-Oct-2010).
Fri, 29 Oct 2010 18:17:11 +0200 updated SMT certificates
boehmes [Fri, 29 Oct 2010 18:17:11 +0200] rev 40280
updated SMT certificates
Fri, 29 Oct 2010 18:17:10 +0200 eta-expand built-in constants; also rewrite partially applied natural number terms
boehmes [Fri, 29 Oct 2010 18:17:10 +0200] rev 40279
eta-expand built-in constants; also rewrite partially applied natural number terms
Fri, 29 Oct 2010 18:17:09 +0200 optionally drop assumptions which cannot be preprocessed
boehmes [Fri, 29 Oct 2010 18:17:09 +0200] rev 40278
optionally drop assumptions which cannot be preprocessed
Fri, 29 Oct 2010 18:17:08 +0200 added crafted list of SMT built-in constants
boehmes [Fri, 29 Oct 2010 18:17:08 +0200] rev 40277
added crafted list of SMT built-in constants
Fri, 29 Oct 2010 18:17:06 +0200 clarified error message
boehmes [Fri, 29 Oct 2010 18:17:06 +0200] rev 40276
clarified error message
Fri, 29 Oct 2010 18:17:05 +0200 tuned
boehmes [Fri, 29 Oct 2010 18:17:05 +0200] rev 40275
tuned
Fri, 29 Oct 2010 18:17:04 +0200 introduced SMT.distinct as a representation of the solvers' built-in predicate; check that SMT.distinct is always applied to an explicit list
boehmes [Fri, 29 Oct 2010 18:17:04 +0200] rev 40274
introduced SMT.distinct as a representation of the solvers' built-in predicate; check that SMT.distinct is always applied to an explicit list
Fri, 29 Oct 2010 17:38:57 +0200 merged
wenzelm [Fri, 29 Oct 2010 17:38:57 +0200] rev 40273
merged
Fri, 29 Oct 2010 17:28:27 +0200 added listrel1
nipkow [Fri, 29 Oct 2010 17:28:27 +0200] rev 40272
added listrel1
Fri, 29 Oct 2010 17:25:22 +0200 hide Sum_Type.Plus
nipkow [Fri, 29 Oct 2010 17:25:22 +0200] rev 40271
hide Sum_Type.Plus
Fri, 29 Oct 2010 16:51:20 +0200 merged
wenzelm [Fri, 29 Oct 2010 16:51:20 +0200] rev 40270
merged
Fri, 29 Oct 2010 16:04:35 +0200 added user aliasses (still unclear how to specify names with whitespace contained)
haftmann [Fri, 29 Oct 2010 16:04:35 +0200] rev 40269
added user aliasses (still unclear how to specify names with whitespace contained)
Fri, 29 Oct 2010 14:06:10 +0200 merged
haftmann [Fri, 29 Oct 2010 14:06:10 +0200] rev 40268
merged
Fri, 29 Oct 2010 14:03:02 +0200 tuned structure of theory
haftmann [Fri, 29 Oct 2010 14:03:02 +0200] rev 40267
tuned structure of theory
Fri, 29 Oct 2010 13:49:49 +0200 remove term_of equations for Heap type explicitly
haftmann [Fri, 29 Oct 2010 13:49:49 +0200] rev 40266
remove term_of equations for Heap type explicitly
Fri, 29 Oct 2010 12:49:05 +0200 no need for setting up the kodkodi environment since Kodkodi 1.2.9
blanchet [Fri, 29 Oct 2010 12:49:05 +0200] rev 40265
no need for setting up the kodkodi environment since Kodkodi 1.2.9
Fri, 29 Oct 2010 12:49:05 +0200 fixed order of quantifier instantiation in new Skolemizer
blanchet [Fri, 29 Oct 2010 12:49:05 +0200] rev 40264
fixed order of quantifier instantiation in new Skolemizer
Fri, 29 Oct 2010 12:49:05 +0200 restructure Skolemization code slightly
blanchet [Fri, 29 Oct 2010 12:49:05 +0200] rev 40263
restructure Skolemization code slightly
Fri, 29 Oct 2010 12:49:05 +0200 ensure that MESON correctly preserves the name of variables (needed by the new Skolemizer)
blanchet [Fri, 29 Oct 2010 12:49:05 +0200] rev 40262
ensure that MESON correctly preserves the name of variables (needed by the new Skolemizer)
Fri, 29 Oct 2010 12:49:05 +0200 more work on new Skolemizer without Hilbert_Choice
blanchet [Fri, 29 Oct 2010 12:49:05 +0200] rev 40261
more work on new Skolemizer without Hilbert_Choice
Fri, 29 Oct 2010 12:49:05 +0200 fix cluster numbering in the absense of Hilbert_Choice (reverts acde1b606b0e, effectively reintroducing most of 0bfaaa81fc62)
blanchet [Fri, 29 Oct 2010 12:49:05 +0200] rev 40260
fix cluster numbering in the absense of Hilbert_Choice (reverts acde1b606b0e, effectively reintroducing most of 0bfaaa81fc62)
Fri, 29 Oct 2010 12:49:05 +0200 prevent type errors because of inconsistent skolem Var types by giving fresh indices to Skolems
blanchet [Fri, 29 Oct 2010 12:49:05 +0200] rev 40259
prevent type errors because of inconsistent skolem Var types by giving fresh indices to Skolems
Fri, 29 Oct 2010 12:49:05 +0200 make handling of parameters more robust, by querying the goal
blanchet [Fri, 29 Oct 2010 12:49:05 +0200] rev 40258
make handling of parameters more robust, by querying the goal
Fri, 29 Oct 2010 11:35:28 +0200 actually pass "verbose" argument
haftmann [Fri, 29 Oct 2010 11:35:28 +0200] rev 40257
actually pass "verbose" argument
Fri, 29 Oct 2010 16:16:10 +0200 eliminated obsolete \_ escape;
wenzelm [Fri, 29 Oct 2010 16:16:10 +0200] rev 40256
eliminated obsolete \_ escape;
Fri, 29 Oct 2010 11:49:56 +0200 eliminated obsolete \_ escapes in rail environments;
wenzelm [Fri, 29 Oct 2010 11:49:56 +0200] rev 40255
eliminated obsolete \_ escapes in rail environments;
Fri, 29 Oct 2010 11:35:47 +0200 proper markup of formal text;
wenzelm [Fri, 29 Oct 2010 11:35:47 +0200] rev 40254
proper markup of formal text;
Fri, 29 Oct 2010 11:07:21 +0200 merged
wenzelm [Fri, 29 Oct 2010 11:07:21 +0200] rev 40253
merged
Fri, 29 Oct 2010 11:04:41 +0200 hide_const various constants, in particular to avoid ugly qualifiers in HOLCF
krauss [Fri, 29 Oct 2010 11:04:41 +0200] rev 40252
hide_const various constants, in particular to avoid ugly qualifiers in HOLCF
Fri, 29 Oct 2010 10:40:36 +0200 reverted e31e3f0071d4 because "foo.bar(5)" (with quotes) is wrong
blanchet [Fri, 29 Oct 2010 10:40:36 +0200] rev 40251
reverted e31e3f0071d4 because "foo.bar(5)" (with quotes) is wrong
Fri, 29 Oct 2010 10:14:49 +0200 merged
Lars Noschinski <noschinl@in.tum.de> [Fri, 29 Oct 2010 10:14:49 +0200] rev 40250
merged
Wed, 22 Sep 2010 09:56:39 +0200 Remove unnecessary premise of mult1_union
Lars Noschinski <noschinl@in.tum.de> [Wed, 22 Sep 2010 09:56:39 +0200] rev 40249
Remove unnecessary premise of mult1_union
Fri, 29 Oct 2010 08:44:49 +0200 adapting HOL-Mutabelle to changes in quickcheck
bulwahn [Fri, 29 Oct 2010 08:44:49 +0200] rev 40248
adapting HOL-Mutabelle to changes in quickcheck
Fri, 29 Oct 2010 08:44:46 +0200 NEWS
bulwahn [Fri, 29 Oct 2010 08:44:46 +0200] rev 40247
NEWS
Fri, 29 Oct 2010 08:44:44 +0200 changed global fixed timeout to a configurable timeout for quickcheck; test parameters in quickcheck are now fully passed around with the context
bulwahn [Fri, 29 Oct 2010 08:44:44 +0200] rev 40246
changed global fixed timeout to a configurable timeout for quickcheck; test parameters in quickcheck are now fully passed around with the context
Fri, 29 Oct 2010 08:44:43 +0200 updating documentation on quickcheck in the Isar reference
bulwahn [Fri, 29 Oct 2010 08:44:43 +0200] rev 40245
updating documentation on quickcheck in the Isar reference
Thu, 28 Oct 2010 18:36:34 +0200 merged
bulwahn [Thu, 28 Oct 2010 18:36:34 +0200] rev 40244
merged
Thu, 28 Oct 2010 17:28:45 +0200 adding a simple check to only run with a SWI-Prolog version known to work
bulwahn [Thu, 28 Oct 2010 17:28:45 +0200] rev 40243
adding a simple check to only run with a SWI-Prolog version known to work * * * taking the isabelle platform into account when finding the prolog system
Thu, 28 Oct 2010 23:54:39 +0200 tuned messages;
wenzelm [Thu, 28 Oct 2010 23:54:39 +0200] rev 40242
tuned messages;
Thu, 28 Oct 2010 23:19:52 +0200 discontinued obsolete ML antiquotation @{theory_ref};
wenzelm [Thu, 28 Oct 2010 23:19:52 +0200] rev 40241
discontinued obsolete ML antiquotation @{theory_ref};
Thu, 28 Oct 2010 22:59:33 +0200 tuned;
wenzelm [Thu, 28 Oct 2010 22:59:33 +0200] rev 40240
tuned;
Thu, 28 Oct 2010 22:39:59 +0200 moved FOL/ex/Iff_Oracle.thy to HOL/ex where it is more accessible to most readers of isar-ref;
wenzelm [Thu, 28 Oct 2010 22:39:59 +0200] rev 40239
moved FOL/ex/Iff_Oracle.thy to HOL/ex where it is more accessible to most readers of isar-ref; tuned;
Thu, 28 Oct 2010 22:23:11 +0200 type attribute is derived concept outside the kernel;
wenzelm [Thu, 28 Oct 2010 22:23:11 +0200] rev 40238
type attribute is derived concept outside the kernel;
Thu, 28 Oct 2010 22:12:08 +0200 preserve original source position of exn;
wenzelm [Thu, 28 Oct 2010 22:12:08 +0200] rev 40237
preserve original source position of exn;
Thu, 28 Oct 2010 22:11:06 +0200 handle Type.TYPE_MATCH, not arbitrary exceptions via MATCH_TYPE variable;
wenzelm [Thu, 28 Oct 2010 22:11:06 +0200] rev 40236
handle Type.TYPE_MATCH, not arbitrary exceptions via MATCH_TYPE variable; clarified handle/raise wrt. Quotient_Info.NotFound -- avoid fragile unqualified NotFound depending on "open" scope; added helpful comments;
Thu, 28 Oct 2010 22:04:00 +0200 use Exn.interruptible_capture to keep user-code interruptible (Exn.capture not immediately followed by Exn.release here);
wenzelm [Thu, 28 Oct 2010 22:04:00 +0200] rev 40235
use Exn.interruptible_capture to keep user-code interruptible (Exn.capture not immediately followed by Exn.release here);
Thu, 28 Oct 2010 21:59:01 +0200 added Exn.interruptible_capture, which reraises interrupts as required by user-code (when Exn.capture is not immediately followed by Exn.release);
wenzelm [Thu, 28 Oct 2010 21:59:01 +0200] rev 40234
added Exn.interruptible_capture, which reraises interrupts as required by user-code (when Exn.capture is not immediately followed by Exn.release); refined Exn.is_interrupt: detect nested IO Interrupts; generalized Exn.map_result; more precise dependencies;
Thu, 28 Oct 2010 21:52:33 +0200 eliminated dead code;
wenzelm [Thu, 28 Oct 2010 21:52:33 +0200] rev 40233
eliminated dead code;
Thu, 28 Oct 2010 21:51:34 +0200 tuned white-space;
wenzelm [Thu, 28 Oct 2010 21:51:34 +0200] rev 40232
tuned white-space;
Thu, 28 Oct 2010 17:54:25 +0200 merged
nipkow [Thu, 28 Oct 2010 17:54:25 +0200] rev 40231
merged
Thu, 28 Oct 2010 17:54:09 +0200 added lemmas about listrel(1)
nipkow [Thu, 28 Oct 2010 17:54:09 +0200] rev 40230
added lemmas about listrel(1)
Thu, 28 Oct 2010 17:25:46 +0200 tuned;
wenzelm [Thu, 28 Oct 2010 17:25:46 +0200] rev 40229
tuned;
Thu, 28 Oct 2010 15:10:34 +0200 merged
wenzelm [Thu, 28 Oct 2010 15:10:34 +0200] rev 40228
merged
Thu, 28 Oct 2010 12:33:24 +0200 support non-identifier-like fact names in Sledgehammer (e.g., "my lemma") by quoting them
blanchet [Thu, 28 Oct 2010 12:33:24 +0200] rev 40227
support non-identifier-like fact names in Sledgehammer (e.g., "my lemma") by quoting them
Thu, 28 Oct 2010 10:38:29 +0200 merged
blanchet [Thu, 28 Oct 2010 10:38:29 +0200] rev 40226
merged
Thu, 28 Oct 2010 09:40:57 +0200 clear identification
blanchet [Thu, 28 Oct 2010 09:40:57 +0200] rev 40225
clear identification
Thu, 28 Oct 2010 09:36:51 +0200 clear identification;
blanchet [Thu, 28 Oct 2010 09:36:51 +0200] rev 40224
clear identification; thread "Auto S/H" (vs. manual S/H) setting through SMT
Thu, 28 Oct 2010 09:29:57 +0200 clear identification
blanchet [Thu, 28 Oct 2010 09:29:57 +0200] rev 40223
clear identification
Wed, 27 Oct 2010 19:14:33 +0200 reintroduced Auto Try, but this time really off by default -- and leave some classical+simp reasoners out for Auto Try (but keep them for Try)
blanchet [Wed, 27 Oct 2010 19:14:33 +0200] rev 40222
reintroduced Auto Try, but this time really off by default -- and leave some classical+simp reasoners out for Auto Try (but keep them for Try)
Wed, 27 Oct 2010 16:32:13 +0200 do not let Metis be confused by higher-order reasoning leading to literals of the form "~ ~ p", which are really the same as "p"
blanchet [Wed, 27 Oct 2010 16:32:13 +0200] rev 40221
do not let Metis be confused by higher-order reasoning leading to literals of the form "~ ~ p", which are really the same as "p"
Wed, 27 Oct 2010 09:22:40 +0200 generalize to handle any prover (not just E)
blanchet [Wed, 27 Oct 2010 09:22:40 +0200] rev 40220
generalize to handle any prover (not just E)
Wed, 27 Oct 2010 11:11:35 -0700 merged
huffman [Wed, 27 Oct 2010 11:11:35 -0700] rev 40219
merged
Wed, 27 Oct 2010 11:10:36 -0700 make domain package work with non-cpo argument types
huffman [Wed, 27 Oct 2010 11:10:36 -0700] rev 40218
make domain package work with non-cpo argument types
Wed, 27 Oct 2010 11:06:53 -0700 make op -->> infixr, to match op --->
huffman [Wed, 27 Oct 2010 11:06:53 -0700] rev 40217
make op -->> infixr, to match op --->
Tue, 26 Oct 2010 14:19:59 -0700 use Named_Thms instead of Theory_Data for some domain package theorems
huffman [Tue, 26 Oct 2010 14:19:59 -0700] rev 40216
use Named_Thms instead of Theory_Data for some domain package theorems
Tue, 26 Oct 2010 09:00:07 -0700 change types of ML commands add_domain, add_new_domain to take 'sort' instead of 'string option'
huffman [Tue, 26 Oct 2010 09:00:07 -0700] rev 40215
change types of ML commands add_domain, add_new_domain to take 'sort' instead of 'string option'
Tue, 26 Oct 2010 08:36:52 -0700 use Term.add_tfreesT
huffman [Tue, 26 Oct 2010 08:36:52 -0700] rev 40214
use Term.add_tfreesT
Sun, 24 Oct 2010 15:42:57 -0700 rename case combinators generated by domain package to 'foo_case' instead of 'foo_when'
huffman [Sun, 24 Oct 2010 15:42:57 -0700] rev 40213
rename case combinators generated by domain package to 'foo_case' instead of 'foo_when'
Sun, 24 Oct 2010 15:19:17 -0700 rename constant 'one_when' to 'one_case'
huffman [Sun, 24 Oct 2010 15:19:17 -0700] rev 40212
rename constant 'one_when' to 'one_case'
Wed, 27 Oct 2010 16:40:34 +0200 merged
haftmann [Wed, 27 Oct 2010 16:40:34 +0200] rev 40211
merged
Wed, 27 Oct 2010 16:40:31 +0200 sorting: avoid _key suffix if lemma applies both to simple and generalized variant; generalized insort_insert to insort_insert_key; additional lemmas
haftmann [Wed, 27 Oct 2010 16:40:31 +0200] rev 40210
sorting: avoid _key suffix if lemma applies both to simple and generalized variant; generalized insort_insert to insort_insert_key; additional lemmas
Wed, 27 Oct 2010 13:46:30 +0200 regenerated keyword file
krauss [Wed, 27 Oct 2010 13:46:30 +0200] rev 40209
regenerated keyword file
Wed, 27 Oct 2010 08:58:03 +0200 made SML/NJ happy
boehmes [Wed, 27 Oct 2010 08:58:03 +0200] rev 40208
made SML/NJ happy
Tue, 26 Oct 2010 21:51:04 +0200 adapted SMT solver error handling to reflect latest changes in "SMT_Solver"
blanchet [Tue, 26 Oct 2010 21:51:04 +0200] rev 40207
adapted SMT solver error handling to reflect latest changes in "SMT_Solver"
Tue, 26 Oct 2010 21:43:50 +0200 better list of irrelevant SMT constants
blanchet [Tue, 26 Oct 2010 21:43:50 +0200] rev 40206
better list of irrelevant SMT constants
Tue, 26 Oct 2010 21:34:01 +0200 if "debug" is on, print list of relevant facts (poweruser request);
blanchet [Tue, 26 Oct 2010 21:34:01 +0200] rev 40205
if "debug" is on, print list of relevant facts (poweruser request); internal renaming
Tue, 26 Oct 2010 21:01:28 +0200 standardize on "fact" terminology (vs. "axiom" or "theorem") in Sledgehammer -- but keep "Axiom" in the lower-level "ATP_Problem" module
blanchet [Tue, 26 Oct 2010 21:01:28 +0200] rev 40204
standardize on "fact" terminology (vs. "axiom" or "theorem") in Sledgehammer -- but keep "Axiom" in the lower-level "ATP_Problem" module
Tue, 26 Oct 2010 20:12:33 +0200 "Nitpick" -> "Sledgehammer";
blanchet [Tue, 26 Oct 2010 20:12:33 +0200] rev 40203
"Nitpick" -> "Sledgehammer"; reparagraphing
Tue, 26 Oct 2010 20:09:38 +0200 merge
blanchet [Tue, 26 Oct 2010 20:09:38 +0200] rev 40202
merge
Tue, 26 Oct 2010 16:59:19 +0200 merged
blanchet [Tue, 26 Oct 2010 16:59:19 +0200] rev 40201
merged
Tue, 26 Oct 2010 16:56:54 +0200 remove needless context argument;
blanchet [Tue, 26 Oct 2010 16:56:54 +0200] rev 40200
remove needless context argument; prefer "Proof.context_of" to "#context o Proof.goal", since it considers any "using [[...]]"
Tue, 26 Oct 2010 17:35:54 +0200 use proper context
boehmes [Tue, 26 Oct 2010 17:35:54 +0200] rev 40199
use proper context
Tue, 26 Oct 2010 17:35:52 +0200 trace assumptions before giving them to the SMT solver
boehmes [Tue, 26 Oct 2010 17:35:52 +0200] rev 40198
trace assumptions before giving them to the SMT solver
Tue, 26 Oct 2010 17:35:51 +0200 capture out-of-memory warnings of Z3 and turn them into proper exceptions; be more precise about SMT solver run-time: return NONE instead of ~1
boehmes [Tue, 26 Oct 2010 17:35:51 +0200] rev 40197
capture out-of-memory warnings of Z3 and turn them into proper exceptions; be more precise about SMT solver run-time: return NONE instead of ~1
Tue, 26 Oct 2010 17:35:49 +0200 honor choice of either local or remote SMT solver only for smt_filter and keep default behaviour for the SMT tactic; omit messages when running smt_filter
boehmes [Tue, 26 Oct 2010 17:35:49 +0200] rev 40196
honor choice of either local or remote SMT solver only for smt_filter and keep default behaviour for the SMT tactic; omit messages when running smt_filter
Tue, 26 Oct 2010 16:39:21 +0200 include ATP in theory List -- avoid theory edge by-passing the prominent list theory
haftmann [Tue, 26 Oct 2010 16:39:21 +0200] rev 40195
include ATP in theory List -- avoid theory edge by-passing the prominent list theory
Tue, 26 Oct 2010 15:06:36 +0200 fixed typo
krauss [Tue, 26 Oct 2010 15:06:36 +0200] rev 40194
fixed typo
Tue, 26 Oct 2010 15:01:39 +0200 merged
blanchet [Tue, 26 Oct 2010 15:01:39 +0200] rev 40193
merged
Tue, 26 Oct 2010 15:01:02 +0200 merged
blanchet [Tue, 26 Oct 2010 15:01:02 +0200] rev 40192
merged
Tue, 26 Oct 2010 14:49:48 +0200 put theorems added using "add:" at the beginning of the list returned by the relevance filter, so that they don't get truncated away
blanchet [Tue, 26 Oct 2010 14:49:48 +0200] rev 40191
put theorems added using "add:" at the beginning of the list returned by the relevance filter, so that they don't get truncated away
Tue, 26 Oct 2010 14:48:55 +0200 tuning
blanchet [Tue, 26 Oct 2010 14:48:55 +0200] rev 40190
tuning
Tue, 26 Oct 2010 15:00:57 +0200 merged
haftmann [Tue, 26 Oct 2010 15:00:57 +0200] rev 40189
merged
Tue, 26 Oct 2010 14:06:22 +0200 consider base sorts of superclasses simultaneously during processing of class specification -- avoids clash of different base sorts
haftmann [Tue, 26 Oct 2010 14:06:22 +0200] rev 40188
consider base sorts of superclasses simultaneously during processing of class specification -- avoids clash of different base sorts
(0) -30000 -10000 -3000 -1000 -128 +128 +1000 +3000 +10000 +30000 tip