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);
Wed, 24 Aug 2011 16:27:27 +0200 wenzelm clarified norm_header/header_edit -- disallow update of loaded theories;
Wed, 24 Aug 2011 15:55:43 +0200 wenzelm misc tuning and simplification;
Wed, 24 Aug 2011 15:30:43 +0200 wenzelm ignore irrelevant timings;
Wed, 24 Aug 2011 13:40:10 +0200 wenzelm print state only for visible command, to avoid wasting resources for the larger part of the text;
Wed, 24 Aug 2011 13:38:07 +0200 wenzelm early filtering of unchanged perspective;
Wed, 24 Aug 2011 13:37:43 +0200 wenzelm more reliable update_perspective handler based on actual text visibility (e.g. on startup or when resizing without scrolling);
Wed, 24 Aug 2011 13:03:39 +0200 wenzelm update_perspective without actual edits, bypassing the full state assignment protocol;
Tue, 23 Aug 2011 21:19:24 +0200 wenzelm tuned;
Tue, 23 Aug 2011 21:14:59 +0200 wenzelm handle potentially more approriate BufferUpdate.LOADED event;
Mon, 22 Aug 2011 23:39:05 +0200 wenzelm special treatment of structure index 1 in Pure, including legacy warning;
Tue, 23 Aug 2011 19:49:21 +0200 blanchet compile
Tue, 23 Aug 2011 19:00:48 +0200 blanchet added "max_calls" option to get a fixed number of Sledgehammer calls per theory
Tue, 23 Aug 2011 18:42:05 +0200 blanchet beef up "sledgehammer_tac" reconstructor
Tue, 23 Aug 2011 18:42:05 +0200 blanchet clean up Sledgehammer tactic
Tue, 23 Aug 2011 17:44:31 +0200 wenzelm fixed document;
Tue, 23 Aug 2011 17:43:06 +0200 wenzelm tuned signature;
Tue, 23 Aug 2011 17:12:54 +0200 wenzelm merged
Tue, 23 Aug 2011 16:37:23 +0200 blanchet always use TFF if possible
Tue, 23 Aug 2011 16:14:19 +0200 blanchet clearer separator in generated file names
Tue, 23 Aug 2011 16:07:01 +0200 blanchet exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
Tue, 23 Aug 2011 15:50:27 +0200 blanchet updated known failures for Z3 3.0 TPTP
Tue, 23 Aug 2011 15:18:46 +0200 blanchet updated Z3 docs
Tue, 23 Aug 2011 15:15:43 +0200 blanchet avoid TFF format with older Vampire versions
Tue, 23 Aug 2011 14:57:16 +0200 blanchet update the Vampire related parts of the documentation
Tue, 23 Aug 2011 14:44:19 +0200 blanchet fixed TFF slicing
Tue, 23 Aug 2011 14:44:19 +0200 blanchet kindly ask Vampire to output axiom names
Tue, 23 Aug 2011 14:44:19 +0200 blanchet added formats to the slice and use TFF for remote Vampire
Tue, 23 Aug 2011 07:14:09 +0200 haftmann tuned specifications, syntax and proofs
Mon, 22 Aug 2011 22:00:36 +0200 haftmann tuned specifications and syntax
Tue, 23 Aug 2011 03:34:17 +0900 Cezary Kaliszyk Quotient Package: some infrastructure for lifting inside sets
Mon, 22 Aug 2011 15:02:45 +0200 blanchet include all encodings in tests, now that the incompleteness of some encodings has been addressed
Mon, 22 Aug 2011 15:02:45 +0200 blanchet change Metis's default settings if type information axioms are generated
Mon, 22 Aug 2011 15:02:45 +0200 blanchet we must tag any type whose ground types intersect a nonmonotonic type
Mon, 22 Aug 2011 15:02:45 +0200 blanchet prefer the lighter, slightly unsound monotonicity-based encodings for Metis
Mon, 22 Aug 2011 15:02:45 +0200 blanchet made reconstruction of type tag equalities "\?x = \?x" reliable
Mon, 22 Aug 2011 15:02:45 +0200 blanchet tuning ATP problem output
Mon, 22 Aug 2011 15:02:45 +0200 blanchet revert guard logic -- make sure that typing information is generated for existentials
Mon, 22 Aug 2011 15:02:45 +0200 blanchet generate tag equations for existential variables
Mon, 22 Aug 2011 15:02:45 +0200 blanchet tuning, plus started implementing tag equation generation for existential variables
Mon, 22 Aug 2011 15:02:45 +0200 blanchet precisely distinguish between universal and existential quantifiers, instead of assuming the worst (universal), for monotonicity analysis
Mon, 22 Aug 2011 15:02:45 +0200 blanchet clearer terminology
Mon, 22 Aug 2011 15:02:45 +0200 blanchet renamed "heavy" to "uniform", based on discussion with Nick Smallbone
Mon, 22 Aug 2011 15:02:45 +0200 blanchet removed unused configuration option
Mon, 22 Aug 2011 15:02:45 +0200 blanchet added caching for (in)finiteness checks
Mon, 22 Aug 2011 15:02:45 +0200 blanchet remove needless typing information
Mon, 22 Aug 2011 15:02:45 +0200 blanchet cleaner handling of polymorphic monotonicity inference
Mon, 22 Aug 2011 15:02:45 +0200 blanchet started cleaning up polymorphic monotonicity-based encodings, based on discussions with Nick Smallbone
Mon, 22 Aug 2011 15:02:45 +0200 blanchet more precise warning
Mon, 22 Aug 2011 15:02:45 +0200 blanchet added option to control soundness of encodings more precisely, for evaluation purposes
Mon, 22 Aug 2011 15:02:45 +0200 blanchet make sound mode more sound (and clean up code)
Mon, 22 Aug 2011 15:02:45 +0200 blanchet reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
Mon, 22 Aug 2011 15:02:45 +0200 blanchet gracefully handle empty SPASS problems
Mon, 22 Aug 2011 15:02:45 +0200 blanchet pass sound option to Sledgehammer tactic
Tue, 23 Aug 2011 16:53:05 +0200 wenzelm tuned signature -- contrast physical output primitives versus Output.raw_message;
Tue, 23 Aug 2011 16:41:16 +0200 wenzelm tuned signature;
Tue, 23 Aug 2011 16:39:21 +0200 wenzelm discontinued slightly odd Future/Lazy.get_finished, which do not really fit into the execution model of Future.cancel/join_tasks (canceled tasks need to be dequeued and terminated explicitly);
Tue, 23 Aug 2011 15:48:41 +0200 wenzelm some support for toplevel printing wrt. editor perspective (still inactive);
Tue, 23 Aug 2011 12:20:12 +0200 wenzelm propagate editor perspective through document model;
Mon, 22 Aug 2011 21:42:02 +0200 wenzelm some support for editor perspective;
Mon, 22 Aug 2011 21:09:26 +0200 wenzelm discontinued redundant Edit_Command_ID;
Mon, 22 Aug 2011 20:11:44 +0200 wenzelm reduced warnings;
Mon, 22 Aug 2011 20:00:04 +0200 wenzelm tuned message;
Mon, 22 Aug 2011 17:10:22 +0200 wenzelm old-style numbered structure index is legacy feature (hardly ever used now);
Mon, 22 Aug 2011 16:12:23 +0200 wenzelm added official Text.Range.Ordering;
Mon, 22 Aug 2011 14:15:52 +0200 wenzelm tuned signature;
Mon, 22 Aug 2011 12:17:22 +0200 wenzelm reverted some odd changes to HOL/Import (cf. 74c08021ab2e);
Mon, 22 Aug 2011 10:57:33 +0200 krauss merged
Sun, 21 Aug 2011 22:13:04 +0200 krauss modernized specifications
Sun, 21 Aug 2011 22:13:04 +0200 krauss removed session HOL/Subst -- now subsumed my more modern HOL/ex/Unification.thy
Sun, 21 Aug 2011 22:13:04 +0200 krauss removed technical or trivial unused facts
Sun, 21 Aug 2011 22:13:04 +0200 krauss more precise authors and comments;
Sun, 21 Aug 2011 22:13:04 +0200 krauss added proof of idempotence, roughly after HOL/Subst/Unify.thy
Sun, 21 Aug 2011 22:13:04 +0200 krauss tuned proofs, sledgehammering overly verbose parts
Sun, 21 Aug 2011 22:13:04 +0200 krauss tuned notation
Sun, 21 Aug 2011 22:13:04 +0200 krauss ported some lemmas from HOL/Subst/*;
Sun, 21 Aug 2011 22:13:04 +0200 krauss changed constant names and notation to match HOL/Subst/*.thy, from which this theory is a clone.
Sun, 21 Aug 2011 21:18:59 -0700 huffman merged
Sun, 21 Aug 2011 12:22:31 -0700 huffman add lemmas interior_Times and closure_Times
Sun, 21 Aug 2011 22:56:55 +0200 haftmann avoid pred/set mixture
Sun, 21 Aug 2011 19:47:52 +0200 haftmann avoid pred/set mixture
Sun, 21 Aug 2011 22:04:01 +0200 wenzelm merged
Sun, 21 Aug 2011 11:03:15 -0700 huffman remove unnecessary euclidean_space class constraints
Sun, 21 Aug 2011 09:46:20 -0700 huffman section -> subsection
Sun, 21 Aug 2011 09:38:31 -0700 huffman scale dependency graph to fit on page
Sun, 21 Aug 2011 21:24:42 +0200 wenzelm more robust initialization of token marker and line context wrt. session startup;
Sun, 21 Aug 2011 20:42:26 +0200 wenzelm tuned Parse.group: delayed failure message;
Sun, 21 Aug 2011 20:25:49 +0200 wenzelm avoid actual Color.white, which would be turned into Color.black by org.gjt.sp.jedit.print.BufferPrintable;
Sun, 21 Aug 2011 20:04:02 +0200 wenzelm default style for user fonts -- to prevent org.gjt.sp.jedit.print.BufferPrintable from choking on null;
Sun, 21 Aug 2011 19:32:20 +0200 wenzelm tuned;
Sun, 21 Aug 2011 14:16:44 +0200 wenzelm discontinued somewhat pointless Par_List.map_name -- most of the time is spent in tokenization;
Sun, 21 Aug 2011 13:42:55 +0200 wenzelm discontinued obsolete Thy_Syntax.report_span -- information can be reproduced in Isabelle/Scala;
Sun, 21 Aug 2011 13:36:23 +0200 wenzelm merged
Sat, 20 Aug 2011 15:19:35 -0700 huffman replace lemma realpow_two_diff with new lemma square_diff_square_factored
Sat, 20 Aug 2011 15:54:26 -0700 huffman remove redundant lemma real_0_le_divide_iff in favor or zero_le_divide_iff
Sat, 20 Aug 2011 13:07:00 -0700 huffman move lemma add_eq_0_iff to Groups.thy
Sat, 20 Aug 2011 12:51:15 -0700 huffman remove redundant lemma realpow_two_disj, use square_eq_iff or power2_eq_iff instead
Sat, 20 Aug 2011 10:08:47 -0700 huffman rename real_squared_diff_one_factored to square_diff_one_factored and move to Rings.thy
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip