Thu, 25 Aug 2011 19:05:40 +0200 added one more known Z3 failure
blanchet [Thu, 25 Aug 2011 19:05:40 +0200] rev 44497
added one more known Z3 failure
Thu, 25 Aug 2011 19:02:47 +0200 added config options to control two aspects of the translation, for evaluation purposes
blanchet [Thu, 25 Aug 2011 19:02:47 +0200] rev 44496
added config options to control two aspects of the translation, for evaluation purposes
Thu, 25 Aug 2011 13:55:52 +0100 added choice operator output for
nik [Thu, 25 Aug 2011 13:55:52 +0100] rev 44495
added choice operator output for Satallax
Thu, 25 Aug 2011 14:25:07 +0200 rationalized option names -- mono becomes raw_mono and mangled becomes mono
blanchet [Thu, 25 Aug 2011 14:25:07 +0200] rev 44494
rationalized option names -- mono becomes raw_mono and mangled becomes mono
Thu, 25 Aug 2011 14:25:07 +0200 handle nonmangled monomorphich the same way as mangled monomorphic when it comes to helper -- otherwise we can end up generating too tight type guards
blanchet [Thu, 25 Aug 2011 14:25:07 +0200] rev 44493
handle nonmangled monomorphich the same way as mangled monomorphic when it comes to helper -- otherwise we can end up generating too tight type guards
Thu, 25 Aug 2011 14:25:07 +0200 avoid using ":" for anything but systematic type tag annotations, because Hurd's Metis gives it that special semantics
blanchet [Thu, 25 Aug 2011 14:25:07 +0200] rev 44492
avoid using ":" for anything but systematic type tag annotations, because Hurd's Metis gives it that special semantics
Thu, 25 Aug 2011 14:25:06 +0200 fixed bang encoding detection of which types to encode
blanchet [Thu, 25 Aug 2011 14:25:06 +0200] rev 44491
fixed bang encoding detection of which types to encode
Thu, 25 Aug 2011 14:06:34 +0200 lemma Compl_insert: "- insert x A = (-A) - {x}"
krauss [Thu, 25 Aug 2011 14:06:34 +0200] rev 44490
lemma Compl_insert: "- insert x A = (-A) - {x}"
Thu, 25 Aug 2011 11:15:31 +0200 avoid variable clashes by properly incrementing indices
boehmes [Thu, 25 Aug 2011 11:15:31 +0200] rev 44489
avoid variable clashes by properly incrementing indices
Thu, 25 Aug 2011 11:15:31 +0200 improved completeness and efficiency of Z3 proof reconstruction, especially by an improved handling of Skolemization
boehmes [Thu, 25 Aug 2011 11:15:31 +0200] rev 44488
improved completeness and efficiency of Z3 proof reconstruction, especially by an improved handling of Skolemization
Thu, 25 Aug 2011 00:00:36 +0200 include chained facts for minimizer, otherwise it won't work
blanchet [Thu, 25 Aug 2011 00:00:36 +0200] rev 44487
include chained facts for minimizer, otherwise it won't work
Wed, 24 Aug 2011 22:12:30 +0200 remove Vampire imconplete proof detection -- the bug it was trying to work around has been fixed in version 1.8, and the check is too sensitive anyway
blanchet [Wed, 24 Aug 2011 22:12:30 +0200] rev 44486
remove Vampire imconplete proof detection -- the bug it was trying to work around has been fixed in version 1.8, and the check is too sensitive anyway
Fri, 26 Aug 2011 22:25:41 +0200 back to tradition Scratch.thy default -- execution wrt. perspective overcomes the main problems of 226563829580;
wenzelm [Fri, 26 Aug 2011 22:25:41 +0200] rev 44485
back to tradition Scratch.thy default -- execution wrt. perspective overcomes the main problems of 226563829580;
Fri, 26 Aug 2011 22:14:12 +0200 tuned Session.edit_node: update_perspective based on last_exec_offset;
wenzelm [Fri, 26 Aug 2011 22:14:12 +0200] rev 44484
tuned Session.edit_node: update_perspective based on last_exec_offset;
Fri, 26 Aug 2011 21:27:58 +0200 tuned signature -- iterate subsumes both fold and get_first;
wenzelm [Fri, 26 Aug 2011 21:27:58 +0200] rev 44483
tuned signature -- iterate subsumes both fold and get_first;
Fri, 26 Aug 2011 21:18:42 +0200 further clarification of Document.updated, based on last_common and after_entry;
wenzelm [Fri, 26 Aug 2011 21:18:42 +0200] rev 44482
further clarification of Document.updated, based on last_common and after_entry; tuned;
Fri, 26 Aug 2011 16:06:58 +0200 tuned signature;
wenzelm [Fri, 26 Aug 2011 16:06:58 +0200] rev 44481
tuned signature;
Fri, 26 Aug 2011 15:56:30 +0200 improved Document.edit: more accurate update_start and no_execs;
wenzelm [Fri, 26 Aug 2011 15:56:30 +0200] rev 44480
improved Document.edit: more accurate update_start and no_execs; tuned;
Fri, 26 Aug 2011 15:09:54 +0200 refined document state assignment: observe perspective, more explicit assignment message;
wenzelm [Fri, 26 Aug 2011 15:09:54 +0200] rev 44479
refined document state assignment: observe perspective, more explicit assignment message; misc tuning and clarification;
Thu, 25 Aug 2011 19:12:58 +0200 tuned signature -- emphasize traditional read/eval/print terminology, which is still relevant here;
wenzelm [Thu, 25 Aug 2011 19:12:58 +0200] rev 44478
tuned signature -- emphasize traditional read/eval/print terminology, which is still relevant here;
Thu, 25 Aug 2011 17:38:12 +0200 maintain last_execs assignment on Scala side;
wenzelm [Thu, 25 Aug 2011 17:38:12 +0200] rev 44477
maintain last_execs assignment on Scala side; prefer tables over IDs instead of objects;
Thu, 25 Aug 2011 16:44:06 +0200 propagate information about last command with exec state assignment through document model;
wenzelm [Thu, 25 Aug 2011 16:44:06 +0200] rev 44476
propagate information about last command with exec state assignment through document model;
Thu, 25 Aug 2011 13:24:41 +0200 tuned signature;
wenzelm [Thu, 25 Aug 2011 13:24:41 +0200] rev 44475
tuned signature;
Thu, 25 Aug 2011 11:41:48 +0200 slightly more abstract Command.Perspective;
wenzelm [Thu, 25 Aug 2011 11:41:48 +0200] rev 44474
slightly more abstract Command.Perspective;
Thu, 25 Aug 2011 11:27:37 +0200 slightly more abstract Text.Perspective;
wenzelm [Thu, 25 Aug 2011 11:27:37 +0200] rev 44473
slightly more abstract Text.Perspective;
Wed, 24 Aug 2011 23:20:05 +0200 tuned proofs;
wenzelm [Wed, 24 Aug 2011 23:20:05 +0200] rev 44472
tuned proofs;
Wed, 24 Aug 2011 23:19:40 +0200 tuned syntax -- avoid ambiguities;
wenzelm [Wed, 24 Aug 2011 23:19:40 +0200] rev 44471
tuned syntax -- avoid ambiguities;
Wed, 24 Aug 2011 23:00:53 +0200 more accurate treatment of index syntax constants, for proper entity references in concrete notation (e.g. infix "\<oplus>\<index>");
wenzelm [Wed, 24 Aug 2011 23:00:53 +0200] rev 44470
more accurate treatment of index syntax constants, for proper entity references in concrete notation (e.g. infix "\<oplus>\<index>");
Wed, 24 Aug 2011 09:23:26 -0700 delete commented-out dead code
huffman [Wed, 24 Aug 2011 09:23:26 -0700] rev 44469
delete commented-out dead code
Wed, 24 Aug 2011 09:08:07 -0700 merged
huffman [Wed, 24 Aug 2011 09:08:07 -0700] rev 44468
merged
(0) -30000 -10000 -3000 -1000 -300 -100 -50 -30 +30 +50 +100 +300 +1000 +3000 +10000 +30000 tip