haftmann [Fri, 14 Aug 2009 15:36:55 +0200] rev 32373
formally stylized
haftmann [Fri, 14 Aug 2009 15:36:54 +0200] rev 32372
formally stylized
haftmann [Fri, 14 Aug 2009 15:36:53 +0200] rev 32371
corrected Pair to Char
webertj [Fri, 14 Aug 2009 13:45:52 +0100] rev 32370
merged
webertj [Fri, 14 Aug 2009 13:44:14 +0100] rev 32369
Fixed a bug where the simplifier would hang on
lemma "f a = M { nat j |j. 0 <= j & j < f b}"
pre_decomp/pre_tac no longer split terms that contain (non-locally) bound
variables (e.g., "nat j" in the above example).
paulson [Thu, 13 Aug 2009 17:19:54 +0100] rev 32368
merged
paulson [Thu, 13 Aug 2009 17:19:42 +0100] rev 32367
Removal of redundant settings of unification trace and search bounds.
paulson [Thu, 13 Aug 2009 17:19:10 +0100] rev 32366
Demonstrations of sledgehammer in protocol proofs.
wenzelm [Wed, 12 Aug 2009 00:26:01 +0200] rev 32365
added PARALLEL_CHOICE, PARALLEL_GOALS;
wenzelm [Tue, 11 Aug 2009 20:40:02 +0200] rev 32364
merged
Philipp Meyer [Mon, 10 Aug 2009 13:53:42 +0200] rev 32363
SOS: function to set default prover; output channel changed
Philipp Meyer [Mon, 10 Aug 2009 13:02:05 +0200] rev 32362
interrupt handler for neos csdp client
wenzelm [Tue, 11 Aug 2009 15:53:13 +0200] rev 32361
clarified situation about unidentified repository versions -- in a distributed setting there is not "the" repository;
haftmann [Tue, 11 Aug 2009 10:58:36 +0200] rev 32360
updated generated document
haftmann [Tue, 11 Aug 2009 10:46:11 +0200] rev 32359
dropped temporary adjustments to non-working eta expansion in recfun_codegen.ML
haftmann [Tue, 11 Aug 2009 10:43:43 +0200] rev 32358
proper eta expansion in recfun_codegen.ML; no eta expansion at all in code_thingol.ML
haftmann [Tue, 11 Aug 2009 10:05:53 +0200] rev 32357
merged
haftmann [Tue, 11 Aug 2009 10:05:16 +0200] rev 32356
temporary adjustment to dubious state of eta expansion in recfun_codegen
haftmann [Mon, 10 Aug 2009 13:34:50 +0200] rev 32355
properly merged
haftmann [Mon, 10 Aug 2009 12:25:30 +0200] rev 32354
same_typscheme replaces ugly common_typ_eqns
haftmann [Mon, 10 Aug 2009 12:24:49 +0200] rev 32353
moved all technical processing of code equations to code_thingol.ML
haftmann [Mon, 10 Aug 2009 12:24:47 +0200] rev 32352
added map_transpose
haftmann [Mon, 10 Aug 2009 10:25:00 +0200] rev 32351
merged
haftmann [Mon, 10 Aug 2009 08:37:37 +0200] rev 32350
attempt to move desymbolization to translation
haftmann [Fri, 31 Jul 2009 10:49:09 +0200] rev 32349
added a somehow clueless comment
haftmann [Fri, 31 Jul 2009 10:49:08 +0200] rev 32348
repair mess produced by resolution afterwards
haftmann [Fri, 31 Jul 2009 09:46:09 +0200] rev 32347
using certify_instantiate
haftmann [Fri, 31 Jul 2009 09:34:21 +0200] rev 32346
merged
haftmann [Fri, 31 Jul 2009 09:34:05 +0200] rev 32345
cleaned up variable desymbolification and argument expansion
haftmann [Thu, 30 Jul 2009 15:21:31 +0200] rev 32344
more appropriate printing of function terms
haftmann [Thu, 30 Jul 2009 15:21:18 +0200] rev 32343
improved handling of parameters
haftmann [Thu, 30 Jul 2009 15:20:57 +0200] rev 32342
path-sensitive tuple combinators carry a "p"(ath) prefix; combinators for standard right-fold tuples
haftmann [Thu, 30 Jul 2009 13:52:18 +0200] rev 32341
towards proper handling of argument order in comprehensions
haftmann [Thu, 30 Jul 2009 13:52:18 +0200] rev 32340
cleaned up
haftmann [Thu, 30 Jul 2009 13:52:17 +0200] rev 32339
termT and term_of_const
nipkow [Mon, 10 Aug 2009 18:12:55 +0200] rev 32338
added bij lemmas
nipkow [Mon, 10 Aug 2009 17:00:41 +0200] rev 32337
new lemma bij_comp
wenzelm [Sat, 08 Aug 2009 11:40:22 +0200] rev 32336
refined mac-poly64 tests;
wenzelm [Fri, 07 Aug 2009 19:16:04 +0200] rev 32335
tuned spacing of sections;
reduced line length;
wenzelm [Thu, 06 Aug 2009 22:30:27 +0200] rev 32334
more platforms;
wenzelm [Thu, 06 Aug 2009 20:46:33 +0200] rev 32333
tuned header;
visible text instead of source comments;
wenzelm [Thu, 06 Aug 2009 19:51:59 +0200] rev 32332
misc changes to SOS by Philipp Meyer:
CSDP_EXE as central setting;
separate component src/HOL/Library/Sum_Of_Squares;
misc tuning and rearrangement of neos_csdp_client;
more robust treatment of shell paths;
debugging depends on local flag;
removed unused parts;
wenzelm [Wed, 05 Aug 2009 17:10:10 +0200] rev 32331
settings for ATP_Manager component;
wenzelm [Wed, 05 Aug 2009 16:17:30 +0200] rev 32330
merged
wenzelm [Wed, 05 Aug 2009 15:39:34 +0200] rev 32329
SUBPROOF: recovered Goal.check_finished;
tuned;
wenzelm [Tue, 04 Aug 2009 23:25:00 +0200] rev 32328
added Isabelle_System.components;
wenzelm [Tue, 04 Aug 2009 19:20:24 +0200] rev 32327
src/HOL/Tools/ATP_Manager as separate component, with (almost) everything in one place;
wenzelm [Tue, 04 Aug 2009 16:13:16 +0200] rev 32326
etc/components;
isabelle makeall operates on all components with IsaMakefile;
wenzelm [Tue, 04 Aug 2009 16:11:11 +0200] rev 32325
turned object-logics into components;
isabelle makeall: operate on all components with IsaMakefile, not just hardwired "logics";
wenzelm [Tue, 04 Aug 2009 16:09:46 +0200] rev 32324
spelling;
wenzelm [Tue, 04 Aug 2009 15:59:57 +0200] rev 32323
tuned "Bootstrapping the environment";
added "Additional components";
wenzelm [Tue, 04 Aug 2009 15:05:34 +0200] rev 32322
change IFS only locally -- thanks to bash arrays;
wenzelm [Tue, 04 Aug 2009 13:35:33 +0200] rev 32321
more uniform handling of ISABELLE_HOME_USER component;
discontinued ISABELLE_IGNORE_USER_SETTINGS (ever used? cf. c567f9fd61a2);
wenzelm [Tue, 04 Aug 2009 13:29:52 +0200] rev 32320
options for more precise performance figures of at-poly, which happens to run on macbroy21;
bulwahn [Tue, 04 Aug 2009 08:45:03 +0200] rev 32319
removing tracing messages in predicate compiler
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32318
improved use of context with cases rule in predicate compiler; predicate compiler based on Main for faster debugging
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32317
commented rpred compilation; tuned
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32316
added generator compilation of higher-order predicates; refined mode analysis for generators; some tuning
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32315
tuned proof procedure; added size-limiting predicate compilation of higher order predicates; added guessing of number parameters for registrating predicates; removed debug messages
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32314
changed resolving depending predicates and fetching in the predicate compiler
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32313
refactoring predicate compiler; repaired proof procedure to handle all test cases
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32312
refactoring predicate compiler; added type synonyms and functions split_smode and split_mode
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32311
adapted predicate compiler for quickcheck generators; added compilation of depth-limited search functions for predicates
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32310
extended mode inference by adding generators; adopted compilation; added some functions for constructing term closures
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32309
imported patch changed mode inference of predicate compiler to return infered dataflow
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32308
imported patch generic compilation of predicate compiler with different monads
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32307
exported functions for quickcheck generator; renamed type constructing functions to fit with the type name in the Predicate theory
bulwahn [Tue, 04 Aug 2009 08:34:56 +0200] rev 32306
removed debug messages; exported to_pred in InductiveSet; added further display function; adjusted mode analysis
wenzelm [Tue, 04 Aug 2009 01:01:23 +0200] rev 32305
basic support for components (which imitate the usual Isabelle directory layout);
berghofe [Sun, 02 Aug 2009 21:03:38 +0200] rev 32304
Tuned.
Christian Urban <urbanc@in.tum.de> [Sun, 02 Aug 2009 17:58:19 +0200] rev 32303
the derived induction principles can be given an explicit name
wenzelm [Sat, 01 Aug 2009 20:34:34 +0200] rev 32302
updated Variable.import;
wenzelm [Sat, 01 Aug 2009 00:39:51 +0200] rev 32301
merged
wenzelm [Sat, 01 Aug 2009 00:39:45 +0200] rev 32300
merged
wenzelm [Fri, 31 Jul 2009 11:34:14 +0200] rev 32299
modernized generated example session;
boehmes [Fri, 31 Jul 2009 23:31:11 +0200] rev 32298
added Mirabelle
boehmes [Fri, 31 Jul 2009 23:30:21 +0200] rev 32297
Quickcheck callable from ML
wenzelm [Sat, 01 Aug 2009 00:17:03 +0200] rev 32296
future scheduler: uninterruptible cancelation;
wenzelm [Sat, 01 Aug 2009 00:09:45 +0200] rev 32295
renamed Multithreading.regular_interrupts to Multithreading.public_interrupts;
renamed Multithreading.restricted_interrupts to Multithreading.private_interrupts;
added Multithreading.sync_interrupts;
Multithreading.sync_wait: more careful treatment of attributes;
Multithreading.tracing: uninterruptible;
Multithreading.system_out: signal within critical region, more careful sync_wait;
eliminated redundant Thread.testInterrupt;
Future.wait_timeout: uniform Multithreading.sync_wait;
future scheduler: interruptible body (sync!), to improve reactivity;
future_job: reject duplicate assignments -- system error;
misc tuning;
wenzelm [Thu, 30 Jul 2009 23:50:11 +0200] rev 32294
recovered polyml-5.2 -- need to reload ML-Systems/multithreading.ML after overriding Thread structures;
wenzelm [Thu, 30 Jul 2009 23:37:53 +0200] rev 32293
tuned tracing;
wenzelm [Thu, 30 Jul 2009 23:23:52 +0200] rev 32292
ISABELLE_USEDIR_OPTIONS: -q 2 by default;
wenzelm [Thu, 30 Jul 2009 23:09:29 +0200] rev 32291
merged
wenzelm [Thu, 30 Jul 2009 21:27:15 +0200] rev 32290
merged
haftmann [Thu, 30 Jul 2009 08:18:22 +0200] rev 32289
merged
haftmann [Wed, 29 Jul 2009 16:54:20 +0200] rev 32288
cleaned up abstract tuple operations and named them consistently
haftmann [Wed, 29 Jul 2009 16:48:34 +0200] rev 32287
cleaned up abstract tuple operations and named them consistently
wenzelm [Thu, 30 Jul 2009 23:06:06 +0200] rev 32286
added Multithreading.sync_wait, which turns enabled interrupts to sync ones, to ensure that wait will reaquire its lock when interrupted;
wenzelm [Thu, 30 Jul 2009 18:43:52 +0200] rev 32285
trancl_tac etc.: back to static context -- problem was caused by bad solver in AFP/JiveDataStoreModel;
wenzelm [Thu, 30 Jul 2009 17:54:57 +0200] rev 32284
retrofit: more precise handling of locally introduced schematic variables (avoid zero_var_indexes);
wenzelm [Thu, 30 Jul 2009 12:20:43 +0200] rev 32283
qualified Subgoal.FOCUS;
wenzelm [Thu, 30 Jul 2009 11:23:57 +0200] rev 32282
FOCUS_PREMS as full replacement for METAHYPS, where the conclusion may still contain schematic variables;
wenzelm [Thu, 30 Jul 2009 11:23:17 +0200] rev 32281
focus: more precise treatment of schematic variables, only the "visible" part of the text is fixed;
added FOCUS_PREMS, which may serve as full replacement for OldGoals.METAHYPS;
wenzelm [Thu, 30 Jul 2009 01:14:40 +0200] rev 32280
Variable.importT/import: return full instantiations, tuned;
wenzelm [Thu, 30 Jul 2009 01:12:33 +0200] rev 32279
added certify_inst, certify_instantiate;
wenzelm [Wed, 29 Jul 2009 22:38:35 +0200] rev 32278
merged