wenzelm [Tue, 13 Aug 2013 14:20:22 +0200] rev 53009
merged
Christian Sternagel [Fri, 09 Aug 2013 19:34:23 +0900] rev 53008
indicate error-functions more prominently (by name prefix instead of suffix);
Christian Sternagel [Fri, 09 Aug 2013 19:34:23 +0900] rev 53007
avoid low-level Same structure;
Christian Sternagel [Fri, 09 Aug 2013 19:34:23 +0900] rev 53006
avoid misleading "instances" in function name;
Christian Sternagel [Fri, 09 Aug 2013 19:34:23 +0900] rev 53005
move treatment of polymorphism to adhoc overloading command;
Christian Sternagel [Fri, 09 Aug 2013 19:34:23 +0900] rev 53004
clarify function;
wenzelm [Tue, 13 Aug 2013 13:18:26 +0200] rev 53003
attempt to transfer focus back to main window after closing popups, which is potentially relevant for heavy-weight windows (cf. workaround in org/gjt/sp/jedit/gui/CompletionPopup.java);
wenzelm [Tue, 13 Aug 2013 12:48:06 +0200] rev 53002
imitate "noWordSep" of isabelle mode, e.g. relevant for word selection via double-click;
wenzelm [Tue, 13 Aug 2013 12:19:45 +0200] rev 53001
support somewhat standard "select all" by default;
wenzelm [Tue, 13 Aug 2013 11:57:42 +0200] rev 53000
more cleanup;
wenzelm [Tue, 13 Aug 2013 11:49:01 +0200] rev 52999
more explicit error, e.g. for sledgehammer query operation applied in non-HOL session;
wenzelm [Tue, 13 Aug 2013 11:13:26 +0200] rev 52998
tuned proofs;
blanchet [Tue, 13 Aug 2013 11:34:56 +0200] rev 52997
added flag for jEdit/PIDE asynchronous mode
blanchet [Tue, 13 Aug 2013 10:29:49 +0200] rev 52996
updated Vampire version numbers
blanchet [Tue, 13 Aug 2013 10:26:56 +0200] rev 52995
Vampire 3.0 requires types to be declared -- make it happy (and get rid of "implicit" types since only Satallax seems to support them anymore)
blanchet [Tue, 13 Aug 2013 09:58:08 +0200] rev 52994
whitepsace tuning
blanchet [Tue, 13 Aug 2013 09:57:55 +0200] rev 52993
more robust parsing of Vampire proofs with "introduced" names
blanchet [Mon, 12 Aug 2013 23:36:43 +0200] rev 52992
fixed "sorry"d proofs
blanchet [Mon, 12 Aug 2013 23:21:06 +0200] rev 52991
repaired proofs (after change to xxx_case_def)
traytel [Mon, 12 Aug 2013 22:38:39 +0200] rev 52990
temporary sorry's for temporarily nonterminating (due to 2b430bbb5a1a) proofs
blanchet [Mon, 12 Aug 2013 21:30:37 +0200] rev 52989
qualify intermediate typedefs
blanchet [Mon, 12 Aug 2013 21:30:36 +0200] rev 52988
avoid double qualification for case constants
blanchet [Mon, 12 Aug 2013 21:30:35 +0200] rev 52987
qualify more generated names with optional type name component
traytel [Mon, 12 Aug 2013 20:04:03 +0200] rev 52986
eliminated bogus assumption from theorem (that was instantiated with refl and resulted in flexflex pairs)
traytel [Mon, 12 Aug 2013 15:36:55 +0200] rev 52985
generalized library function
wenzelm [Mon, 12 Aug 2013 18:03:47 +0200] rev 52984
updated keywords;
wenzelm [Mon, 12 Aug 2013 18:02:01 +0200] rev 52983
merged
wenzelm [Mon, 12 Aug 2013 17:57:51 +0200] rev 52982
clarified Query_Operation.register: avoid hard-wired parallel policy;
sledgehammer: more conventional parallel exception handling -- print just one interrupt;