Thu, 09 Sep 2010 17:58:11 +0200 merged
bulwahn [Thu, 09 Sep 2010 17:58:11 +0200] rev 39256
merged
Thu, 09 Sep 2010 17:23:08 +0200 adding an example with integers and String.literals
bulwahn [Thu, 09 Sep 2010 17:23:08 +0200] rev 39255
adding an example with integers and String.literals
Thu, 09 Sep 2010 17:23:07 +0200 adding an example to show how code_pred must be invoked with locales
bulwahn [Thu, 09 Sep 2010 17:23:07 +0200] rev 39254
adding an example to show how code_pred must be invoked with locales
Thu, 09 Sep 2010 17:23:03 +0200 removing report from the arguments of the quickcheck functions and refering to it by picking it from the context
bulwahn [Thu, 09 Sep 2010 17:23:03 +0200] rev 39253
removing report from the arguments of the quickcheck functions and refering to it by picking it from the context
Thu, 09 Sep 2010 16:43:57 +0200 changing the container for the quickcheck options to a generic data
bulwahn [Thu, 09 Sep 2010 16:43:57 +0200] rev 39252
changing the container for the quickcheck options to a generic data
Thu, 09 Sep 2010 16:47:03 +0100 Tidied up proofs using sledgehammer, also deleting unnecessary semicolons
paulson [Thu, 09 Sep 2010 16:47:03 +0100] rev 39251
Tidied up proofs using sledgehammer, also deleting unnecessary semicolons
Thu, 09 Sep 2010 14:38:14 +0200 changing String.literal to a type instead of a datatype
bulwahn [Thu, 09 Sep 2010 14:38:14 +0200] rev 39250
changing String.literal to a type instead of a datatype
Thu, 09 Sep 2010 11:10:44 +0200 increasing the number of iterations to ensure to find a counterexample by random generation
bulwahn [Thu, 09 Sep 2010 11:10:44 +0200] rev 39249
increasing the number of iterations to ensure to find a counterexample by random generation
Thu, 09 Sep 2010 09:11:13 +0200 only conceal primitive definition theorems, not predicate names
haftmann [Thu, 09 Sep 2010 09:11:13 +0200] rev 39248
only conceal primitive definition theorems, not predicate names
Wed, 08 Sep 2010 19:23:23 +0200 merged
haftmann [Wed, 08 Sep 2010 19:23:23 +0200] rev 39247
merged
Wed, 08 Sep 2010 19:21:46 +0200 modernized primrec
haftmann [Wed, 08 Sep 2010 19:21:46 +0200] rev 39246
modernized primrec
Fri, 10 Sep 2010 15:16:51 +0200 Markup_Tree is already scalable;
wenzelm [Fri, 10 Sep 2010 15:16:51 +0200] rev 39245
Markup_Tree is already scalable;
Fri, 10 Sep 2010 15:05:30 +0200 Isabelle_Markup.tooltip: explicit indication of ML;
wenzelm [Fri, 10 Sep 2010 15:05:30 +0200] rev 39244
Isabelle_Markup.tooltip: explicit indication of ML;
Fri, 10 Sep 2010 14:54:08 +0200 Future.promise: more robust treatment of concurrent abort vs. fulfill (amending 047c96f41455);
wenzelm [Fri, 10 Sep 2010 14:54:08 +0200] rev 39243
Future.promise: more robust treatment of concurrent abort vs. fulfill (amending 047c96f41455);
Fri, 10 Sep 2010 12:39:20 +0200 primitive use_text: let interrupts pass unhindered;
wenzelm [Fri, 10 Sep 2010 12:39:20 +0200] rev 39242
primitive use_text: let interrupts pass unhindered;
Thu, 09 Sep 2010 21:30:33 +0200 Isabelle.load_icon with some sanity checks;
wenzelm [Thu, 09 Sep 2010 21:30:33 +0200] rev 39241
Isabelle.load_icon with some sanity checks;
Thu, 09 Sep 2010 20:09:13 +0200 ML_Compiler.eval: reported positions need to contain offset, to avoid displaced reports due to synthesized line numbers;
wenzelm [Thu, 09 Sep 2010 20:09:13 +0200] rev 39240
ML_Compiler.eval: reported positions need to contain offset, to avoid displaced reports due to synthesized line numbers;
Thu, 09 Sep 2010 18:32:21 +0200 NEWS: some notes on interrupts;
wenzelm [Thu, 09 Sep 2010 18:32:21 +0200] rev 39239
NEWS: some notes on interrupts;
Thu, 09 Sep 2010 18:21:06 +0200 refined Runtime.toplevel_error/Document.run_command: let interrupts pass unhindered;
wenzelm [Thu, 09 Sep 2010 18:21:06 +0200] rev 39238
refined Runtime.toplevel_error/Document.run_command: let interrupts pass unhindered;
Thu, 09 Sep 2010 18:18:34 +0200 removed dead code;
wenzelm [Thu, 09 Sep 2010 18:18:34 +0200] rev 39237
removed dead code;
Thu, 09 Sep 2010 18:17:34 +0200 avoid handling interrupts in user code;
wenzelm [Thu, 09 Sep 2010 18:17:34 +0200] rev 39236
avoid handling interrupts in user code;
Thu, 09 Sep 2010 18:04:35 +0200 Meson.make_clauses_unsorted: removed spurious debug code stemming from 5146d640aa4a -- must not handle arbitrary exceptions in user space;
wenzelm [Thu, 09 Sep 2010 18:04:35 +0200] rev 39235
Meson.make_clauses_unsorted: removed spurious debug code stemming from 5146d640aa4a -- must not handle arbitrary exceptions in user space;
Thu, 09 Sep 2010 18:00:16 +0200 main command loops are supposed to be uninterruptible -- no special treatment here;
wenzelm [Thu, 09 Sep 2010 18:00:16 +0200] rev 39234
main command loops are supposed to be uninterruptible -- no special treatment here;
Thu, 09 Sep 2010 17:38:45 +0200 Exn.is_interrupt: include interrupts that have passed through the IO layer;
wenzelm [Thu, 09 Sep 2010 17:38:45 +0200] rev 39233
Exn.is_interrupt: include interrupts that have passed through the IO layer;
Thu, 09 Sep 2010 17:20:27 +0200 more abstract treatment of interrupts in structure Exn -- hardly ever need to mention Interrupt literally;
wenzelm [Thu, 09 Sep 2010 17:20:27 +0200] rev 39232
more abstract treatment of interrupts in structure Exn -- hardly ever need to mention Interrupt literally;
Thu, 09 Sep 2010 11:05:52 +0200 avoid mixing of static and runtime errors in compiler output, to accomodate Proof General;
wenzelm [Thu, 09 Sep 2010 11:05:52 +0200] rev 39231
avoid mixing of static and runtime errors in compiler output, to accomodate Proof General; refrain from absorbing Exn.Interrupt, to accomodate asynchronous interaction; actually observe Isabelle/ML naming conventions in exception STATIC_ERRORS;
Wed, 08 Sep 2010 23:52:24 +0200 ML_Compiler.eval: discontinued extra "Static Errors" of raw Poly/ML;
wenzelm [Wed, 08 Sep 2010 23:52:24 +0200] rev 39230
ML_Compiler.eval: discontinued extra "Static Errors" of raw Poly/ML;
Wed, 08 Sep 2010 23:40:48 +0200 isabelle-jedit.css: suppress "location" markup, which indicates extra positional information intended for plain-old TTY mode;
wenzelm [Wed, 08 Sep 2010 23:40:48 +0200] rev 39229
isabelle-jedit.css: suppress "location" markup, which indicates extra positional information intended for plain-old TTY mode;
(0) -30000 -10000 -3000 -1000 -300 -100 -50 -28 +28 +50 +100 +300 +1000 +3000 +10000 +30000 tip