blanchet [Thu, 25 Aug 2011 14:25:06 +0200] rev 44491
fixed bang encoding detection of which types to encode
krauss [Thu, 25 Aug 2011 14:06:34 +0200] rev 44490
lemma Compl_insert: "- insert x A = (-A) - {x}"
boehmes [Thu, 25 Aug 2011 11:15:31 +0200] rev 44489
avoid variable clashes by properly incrementing indices
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
blanchet [Thu, 25 Aug 2011 00:00:36 +0200] rev 44487
include chained facts for minimizer, otherwise it won't work
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
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;
wenzelm [Fri, 26 Aug 2011 22:14:12 +0200] rev 44484
tuned Session.edit_node: update_perspective based on last_exec_offset;
wenzelm [Fri, 26 Aug 2011 21:27:58 +0200] rev 44483
tuned signature -- iterate subsumes both fold and get_first;
wenzelm [Fri, 26 Aug 2011 21:18:42 +0200] rev 44482
further clarification of Document.updated, based on last_common and after_entry;
tuned;