Thu, 25 Aug 2011 23:54:57 +0200 blanchet honor TFF Implicit
Thu, 25 Aug 2011 23:38:09 +0200 blanchet make polymorphic encodings more complete
Thu, 25 Aug 2011 22:06:25 +0200 blanchet make default unsound mode less unsound
Thu, 25 Aug 2011 22:05:18 +0200 blanchet make TFF output less explicit where possible
Thu, 25 Aug 2011 19:09:39 +0200 blanchet use more appropriate encoding for Z3 TPTP, as confirmed by evaluation
Thu, 25 Aug 2011 19:05:40 +0200 blanchet added one more known Z3 failure
Thu, 25 Aug 2011 19:02:47 +0200 blanchet added config options to control two aspects of the translation, for evaluation purposes
Thu, 25 Aug 2011 13:55:52 +0100 nik added choice operator output for
Thu, 25 Aug 2011 14:25:07 +0200 blanchet rationalized option names -- mono becomes raw_mono and mangled becomes mono
Thu, 25 Aug 2011 14:25:07 +0200 blanchet 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 blanchet 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 blanchet fixed bang encoding detection of which types to encode
Thu, 25 Aug 2011 14:06:34 +0200 krauss lemma Compl_insert: "- insert x A = (-A) - {x}"
Thu, 25 Aug 2011 11:15:31 +0200 boehmes avoid variable clashes by properly incrementing indices
Thu, 25 Aug 2011 11:15:31 +0200 boehmes improved completeness and efficiency of Z3 proof reconstruction, especially by an improved handling of Skolemization
Thu, 25 Aug 2011 00:00:36 +0200 blanchet include chained facts for minimizer, otherwise it won't work
Wed, 24 Aug 2011 22:12:30 +0200 blanchet 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 wenzelm back to tradition Scratch.thy default -- execution wrt. perspective overcomes the main problems of 226563829580;
Fri, 26 Aug 2011 22:14:12 +0200 wenzelm tuned Session.edit_node: update_perspective based on last_exec_offset;
Fri, 26 Aug 2011 21:27:58 +0200 wenzelm tuned signature -- iterate subsumes both fold and get_first;
Fri, 26 Aug 2011 21:18:42 +0200 wenzelm further clarification of Document.updated, based on last_common and after_entry;
Fri, 26 Aug 2011 16:06:58 +0200 wenzelm tuned signature;
Fri, 26 Aug 2011 15:56:30 +0200 wenzelm improved Document.edit: more accurate update_start and no_execs;
Fri, 26 Aug 2011 15:09:54 +0200 wenzelm refined document state assignment: observe perspective, more explicit assignment message;
Thu, 25 Aug 2011 19:12:58 +0200 wenzelm tuned signature -- emphasize traditional read/eval/print terminology, which is still relevant here;
Thu, 25 Aug 2011 17:38:12 +0200 wenzelm maintain last_execs assignment on Scala side;
Thu, 25 Aug 2011 16:44:06 +0200 wenzelm propagate information about last command with exec state assignment through document model;
Thu, 25 Aug 2011 13:24:41 +0200 wenzelm tuned signature;
Thu, 25 Aug 2011 11:41:48 +0200 wenzelm slightly more abstract Command.Perspective;
Thu, 25 Aug 2011 11:27:37 +0200 wenzelm slightly more abstract Text.Perspective;
Wed, 24 Aug 2011 23:20:05 +0200 wenzelm tuned proofs;
Wed, 24 Aug 2011 23:19:40 +0200 wenzelm tuned syntax -- avoid ambiguities;
Wed, 24 Aug 2011 23:00:53 +0200 wenzelm 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 huffman delete commented-out dead code
Wed, 24 Aug 2011 09:08:07 -0700 huffman merged
Wed, 24 Aug 2011 09:08:00 -0700 huffman change some subsection headings to subsubsection
Tue, 23 Aug 2011 16:47:48 -0700 huffman remove unnecessary lemma card_ge1
Tue, 23 Aug 2011 16:17:22 -0700 huffman move connected_real_lemma to the one place it is used
Wed, 24 Aug 2011 17:30:25 +0200 wenzelm merged
Wed, 24 Aug 2011 15:25:39 +0200 blanchet make sure that all facts are passed to ATP from minimizer
Wed, 24 Aug 2011 11:17:33 +0200 blanchet more reliable "sledgehammer\_tac" reconstruction, by avoiding "insert_tac"
Wed, 24 Aug 2011 11:17:33 +0200 blanchet specify timeout for "sledgehammer_tac"
Wed, 24 Aug 2011 11:17:33 +0200 blanchet tuning
Wed, 24 Aug 2011 10:59:22 +0900 Cezary Kaliszyk Quotient Package: add mem_rsp, mem_prs, tune proofs.
Tue, 23 Aug 2011 15:46:53 -0700 huffman merged
Tue, 23 Aug 2011 14:11:02 -0700 huffman declare euclidean_simps [simp] at the point they are proved;
Tue, 23 Aug 2011 07:12:05 -0700 huffman merged
Mon, 22 Aug 2011 18:15:33 -0700 huffman merged
Mon, 22 Aug 2011 17:22:49 -0700 huffman avoid warnings
Mon, 22 Aug 2011 16:49:45 -0700 huffman comment out dead code to avoid compiler warnings
Mon, 22 Aug 2011 10:43:10 -0700 huffman legacy theorem names
Mon, 22 Aug 2011 10:19:39 -0700 huffman remove duplicate lemma
Tue, 23 Aug 2011 23:18:13 +0200 blanchet fixed "hBOOL" of existential variables, and generate more helpers
Tue, 23 Aug 2011 22:44:08 +0200 blanchet don't select facts when using sledgehammer_tac for reconstruction
Tue, 23 Aug 2011 20:35:41 +0200 blanchet don't perform a triviality check if the goal is skipped anyway
Tue, 23 Aug 2011 19:50:25 +0200 blanchet optional reconstructor
Wed, 24 Aug 2011 17:25:45 +0200 wenzelm misc tuning and simplification;
Wed, 24 Aug 2011 17:16:48 +0200 wenzelm tuned pri: prefer purging of canceled execution;
Wed, 24 Aug 2011 17:14:31 +0200 wenzelm tuned Document.node: maintain "touched" flag to indicate changes in entries etc.;
Wed, 24 Aug 2011 16:49:48 +0200 wenzelm clarified Document.Node.clear -- retain header (cf. ML version);
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip