Mon, 30 May 2011 17:00:38 +0200 blanchet don't slice if there are too few facts
Mon, 30 May 2011 17:00:38 +0200 blanchet nicer failure message when one-line proof reconstruction fails
Mon, 30 May 2011 17:00:38 +0200 blanchet make SML/NJ happy
Mon, 30 May 2011 17:00:38 +0200 blanchet avoid monomorphic encoding with so many facts -- it makes the old monomorphizer explode on some examples
Mon, 30 May 2011 17:00:38 +0200 blanchet make all messages urgent in verbose mode
Mon, 30 May 2011 17:00:38 +0200 blanchet minimize automatically even if Metis failed, if the external prover was really fast
Mon, 30 May 2011 17:00:38 +0200 blanchet fixed syntax of min options
Mon, 30 May 2011 17:00:38 +0200 blanchet no more bonus for E -- with the soft timeout, this punishes everybody -- the bonus was designed for a hard timeout
Mon, 30 May 2011 17:00:38 +0200 blanchet better merging of similar outputs
Mon, 30 May 2011 17:00:38 +0200 blanchet update minimization documentation
Mon, 30 May 2011 17:00:38 +0200 blanchet imported patch sledge_doc_metis_as_prover
Mon, 30 May 2011 17:00:38 +0200 blanchet automatically minimize with Metis when this can be done within a few seconds
Mon, 30 May 2011 17:00:38 +0200 blanchet minimize with Metis if possible
Mon, 30 May 2011 17:00:38 +0200 blanchet support "metis" and "metisFT" as provers in the architecture, so they can be used for minimizing
Mon, 30 May 2011 15:30:05 +0100 paulson Workaround for hyperref bug affecting index entries involving the | symbol
Mon, 30 May 2011 13:58:00 +0200 bulwahn improving heuristics of type annotations in contravariant positions for the special case with instances of the class partial_term_of
Mon, 30 May 2011 13:57:59 +0200 bulwahn automatic derivation of partial_term_of functions; renaming type and term to longer names narrowing_type and narrowing_term; hiding constant C; adding overlord option
Mon, 30 May 2011 12:20:04 +0100 paulson merged multiple heads
Mon, 30 May 2011 12:15:17 +0100 paulson Fix to exception THM 1 raised (line 212 of conv.ML), reported by Andreas Lochbihler
Sun, 29 May 2011 19:40:56 +0200 blanchet always check plain "metis" even if the ATP proof seems to require "metisFT" -- maybe the proof is needlessly complicated
Sun, 29 May 2011 19:40:56 +0200 blanchet normalize indices in chained facts to make sure that backtick facts (which often result in different names) are recognized + changed definition of urgent messages
Fri, 27 May 2011 21:11:44 +0200 krauss function tutorial: do not omit termination proof, even when discussing other things
Fri, 27 May 2011 16:45:24 +0200 boehmes added re-implemented monomorphizer for types with better control for number of generated instances (strict as opposed to the SMT monomorphizer) and with fact annotations controlling in which round certain facts are considered for monomorphization
Fri, 27 May 2011 10:41:09 +0200 blanchet document new "try"
Fri, 27 May 2011 10:33:16 +0200 blanchet tuned comments
Fri, 27 May 2011 10:30:08 +0200 blanchet new timeout section (cf. Nitpick manual)
Fri, 27 May 2011 10:30:08 +0200 blanchet cleanup proof text generation code
Fri, 27 May 2011 10:30:08 +0200 blanchet more Sledgehammer documentation updates
Fri, 27 May 2011 10:30:08 +0200 blanchet minor update
Fri, 27 May 2011 10:30:08 +0200 blanchet try both "metis" and (on failure) "metisFT" in replay
Fri, 27 May 2011 10:30:08 +0200 blanchet show time taken for reconstruction
Fri, 27 May 2011 10:30:08 +0200 blanchet unbreak "max_potential" logic
Fri, 27 May 2011 10:30:08 +0200 blanchet more concise output
Fri, 27 May 2011 10:30:08 +0200 blanchet compile
Fri, 27 May 2011 10:30:08 +0200 blanchet use helpers and tweak Quickcheck's priority to it comes second (to give Solve Direct slightly more time before another prover runs)
Fri, 27 May 2011 10:30:08 +0200 blanchet repaired theory merging and defined/used helpers
Fri, 27 May 2011 10:30:08 +0200 blanchet make Sledgehammer a little bit less verbose in "try"
Fri, 27 May 2011 10:30:08 +0200 blanchet handle non-auto try cases gracefully in Try Methods
Fri, 27 May 2011 10:30:08 +0200 blanchet handle non-auto try case gracefully in Solve Direct
Fri, 27 May 2011 10:30:08 +0200 blanchet prioritize try and auto try's tools, with fast ones first, with a slight preference for provers vs. counterexample generators
Fri, 27 May 2011 10:30:08 +0200 blanchet update SML section of documentation
Fri, 27 May 2011 10:30:08 +0200 blanchet handle non-auto try case gracefully in Nitpick
Fri, 27 May 2011 10:30:08 +0200 blanchet handle non-auto try case of Sledgehammer better
Fri, 27 May 2011 10:30:08 +0200 blanchet added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
Fri, 27 May 2011 10:30:08 +0200 blanchet removed FIXME: "try_methods" doesn't take a clasimpmod, because it needs to generate Isar proof text in case of success and hence needs total control over its arguments
Fri, 27 May 2011 10:30:08 +0200 blanchet renamed "Auto_Tools" "Try"
Fri, 27 May 2011 10:30:08 +0200 blanchet removed THF equality proxy hack now that Geoff Sutcliffe has fixed SystemOnTPTP
Fri, 27 May 2011 10:30:08 +0200 blanchet renamed "try" "try_methods"
Fri, 27 May 2011 10:30:08 +0200 blanchet renamed "metis_timeout" to "preplay_timeout" and continued implementation
Fri, 27 May 2011 10:30:08 +0200 blanchet minor fixes to Sledgehammer docs
Fri, 27 May 2011 10:30:08 +0200 blanchet shorten minimizer command further, exploiting until-now-undocumented syntax
Fri, 27 May 2011 10:30:07 +0200 blanchet minor tweaks to the Nitpick documentation
Fri, 27 May 2011 10:30:07 +0200 blanchet added syntax for specifying Metis timeout (currently used only by SMT solvers)
Fri, 27 May 2011 10:30:07 +0200 blanchet readded Waldmeister as default to the documentation and other minor changes
Fri, 27 May 2011 10:30:07 +0200 blanchet reintroduced Waldmeister but limit the number of remote threads created
Fri, 27 May 2011 10:30:07 +0200 blanchet renamed "minimize" to "min" to make Sledgehammer output a little bit more concise
Fri, 27 May 2011 10:30:07 +0200 blanchet minor doc adjustments
Fri, 27 May 2011 10:30:07 +0200 blanchet make output more concise
Fri, 27 May 2011 10:30:07 +0200 blanchet merge timeout messages from several ATPs into one message to avoid clutter
Fri, 27 May 2011 10:30:07 +0200 blanchet fix soundness bug in Sledgehammer: distinguish params in goals from fixed variables in context
Fri, 27 May 2011 10:30:07 +0200 blanchet tuning
Fri, 27 May 2011 10:30:07 +0200 blanchet mention contributions from LCP and explain metis and metisFT encodings
Fri, 27 May 2011 10:30:07 +0200 blanchet fixed trivial fact detection
Fri, 27 May 2011 10:30:07 +0200 blanchet cleaner handling of equality and proxies (esp. for THF)
Fri, 27 May 2011 10:30:07 +0200 blanchet recognize more ATP failures
Fri, 27 May 2011 10:30:07 +0200 blanchet fully support all type system encodings in typed formats (TFF, THF)
Fri, 27 May 2011 10:30:07 +0200 blanchet take out Waldmeister from default for now -- success rate too low on Judgment Day
Fri, 27 May 2011 10:30:07 +0200 blanchet document relevance filter a bit more
Fri, 27 May 2011 10:30:07 +0200 blanchet always run Sledgehammer synchronously in the jEdit interface (until the multithreading support for Proof General is ported)
Fri, 27 May 2011 10:30:07 +0200 blanchet towards supporting non-simply-typed encodings for TFF and THF (for orthogonality and experiments)
Thu, 26 May 2011 23:21:00 +0200 noschinl instance inat for complete_lattice
Thu, 26 May 2011 22:02:40 +0200 boehmes iteratively deepen abstractions to avoid rare Z3 proof reconstruction failures, e.g. when pulling if-then-else from below uninterpreted constants (suggested by Jasmin Christian Blanchette)
Thu, 26 May 2011 20:51:03 +0200 hoelzl integral strong monotone; finite subadditivity for measure
Thu, 26 May 2011 20:49:56 +0200 hoelzl composition of convex and measurable function is measurable
Thu, 26 May 2011 17:59:39 +0200 hoelzl introduce independence of two random variables
Thu, 26 May 2011 17:40:01 +0200 hoelzl add lemma indep_distribution_eq_measure
Thu, 26 May 2011 14:12:06 +0200 hoelzl add lemma indep_rv_finite
Thu, 26 May 2011 14:12:03 +0200 hoelzl generalize setsum_cases
Thu, 26 May 2011 14:12:02 +0200 hoelzl add lemma borel_0_1_law
Thu, 26 May 2011 14:12:01 +0200 hoelzl add lemma sigma_sets_singleton
Thu, 26 May 2011 14:12:00 +0200 hoelzl use abbrevitation events == sets M
Thu, 26 May 2011 14:11:58 +0200 hoelzl add lemma kolmogorov_0_1_law
Thu, 26 May 2011 14:11:57 +0200 hoelzl add lemma indep_sets_collect_sigma
Thu, 26 May 2011 09:42:04 +0200 bulwahn improving code_int setup in Quickcheck_Narrowing; adding partial_term_of class in Quickcheck_Narrowing
Thu, 26 May 2011 09:42:02 +0200 bulwahn extending terms of Code_Evaluation by Free to allow partial terms
Thu, 26 May 2011 00:20:28 +0200 krauss adhoc event handler to insert 'sendback' text into the buffer, replacing the original command
Thu, 26 May 2011 00:12:30 +0200 krauss css rules for highlighting sendback text
Thu, 26 May 2011 00:12:01 +0200 krauss invert event propagation flag -- in lobobrowser api, true means re-propagate
Wed, 25 May 2011 08:31:36 +0200 blanchet eta-expand to make SML/NJ happy
Tue, 24 May 2011 18:04:23 +0200 blanchet ensure that the argument of logical negation is enclosed in parentheses in THF mode
Tue, 24 May 2011 17:05:29 +0200 blanchet hack to obtain potable step names from Waldmeister
Tue, 24 May 2011 17:04:35 +0200 blanchet respect user's intention better when setting the CNF_UEQ type system (esp. w.r.t. "erased")
Tue, 24 May 2011 13:29:32 +0200 blanchet further reduce the number of facts passed to less used remote ATPs
Tue, 24 May 2011 11:55:59 +0200 blanchet added quietness flag
Tue, 24 May 2011 10:03:15 +0200 blanchet pass fewer relevant facts to less used remote systems
Tue, 24 May 2011 10:01:03 +0200 blanchet more work on parsing LEO-II proofs and extracting uses of extensionality
Tue, 24 May 2011 10:01:00 +0200 blanchet tuning
Tue, 24 May 2011 10:00:38 +0200 blanchet more work on parsing LEO-II proofs without lambdas
Tue, 24 May 2011 00:01:33 +0200 blanchet slightly gracefuller handling of LEO-II and Satallax output
Tue, 24 May 2011 00:01:33 +0200 blanchet document primitive support for LEO-II and Satallax
Tue, 24 May 2011 00:01:33 +0200 blanchet identify HOL functions with THF functions
Tue, 24 May 2011 00:01:33 +0200 blanchet started adding support for THF output (but no lambdas)
Tue, 24 May 2011 00:01:33 +0200 blanchet eliminated more code duplication in Nitrox
Tue, 24 May 2011 00:01:33 +0200 blanchet reduce code duplication in Nitrox
Tue, 24 May 2011 00:01:33 +0200 blanchet use \<emdash> rather than \<midarrow>
Tue, 24 May 2011 00:01:33 +0200 blanchet fixed de Bruijn index bug
Tue, 24 May 2011 00:01:33 +0200 blanchet use "eq_thm_prop" for slacker comparison -- ensures that backtick-quoted chained facts are recognized in the minimizer, among other things
Tue, 24 May 2011 00:01:33 +0200 blanchet filter Waldmeister facts better -- and don't encode type classes as predicates, since it doesn't like conditional equations
Tue, 24 May 2011 00:01:33 +0200 blanchet clearer SystemOnTPTP errors
Tue, 24 May 2011 00:01:33 +0200 blanchet give fewer equations to Waldmeister
Tue, 24 May 2011 00:01:33 +0200 blanchet detect inappropriate problems and crashes better in Waldmeister
Tue, 24 May 2011 00:01:33 +0200 blanchet tuning -- the "appropriate" terminology is inspired from TPTP
Tue, 24 May 2011 00:01:33 +0200 blanchet pass no type args to hAPP in "poly_args" type system, which is unsound anyway and should correspond as closely as possible to the old unsound encoding
Mon, 23 May 2011 19:21:05 +0200 hoelzl move lemmas to Extended_Reals and Extended_Real_Limits
Mon, 23 May 2011 10:58:21 +0200 krauss separate initializations for different modes of partial_function -- generation of induction rules will be non-uniform
Sun, 22 May 2011 22:22:25 +0200 krauss reverted 7fdd8d4908dc -- keeping images from Isabelle_makeall would be too expensive
Sun, 22 May 2011 20:59:13 +0200 krauss fun command produces warning when patterns are incomplete (somewhat analogous to primrec)
Sun, 22 May 2011 14:51:42 +0200 blanchet added message when Waldmeister isn't run
Sun, 22 May 2011 14:51:42 +0200 blanchet slightly improved documentation
Sun, 22 May 2011 14:51:42 +0200 blanchet improved Waldmeister support -- even run it by default on unit equational goals
Sun, 22 May 2011 14:51:41 +0200 blanchet fish out axioms in Waldmeister output
Sun, 22 May 2011 14:51:04 +0200 blanchet removed SNARK hack now that SNARK is fixed
Sun, 22 May 2011 14:51:04 +0200 blanchet recognize one more SystemOnTPTP error
Sun, 22 May 2011 14:51:04 +0200 blanchet document Waldmeister
Sun, 22 May 2011 14:51:01 +0200 blanchet added support for remote Waldmeister
Sun, 22 May 2011 14:50:32 +0200 blanchet added Waldmeister
Sun, 22 May 2011 14:49:35 +0200 blanchet reorganized ATP formats a little bit
Mon, 06 Jun 2011 22:02:34 +0200 wenzelm tuned;
Mon, 06 Jun 2011 19:13:48 +0200 wenzelm removed odd remains of low-level session management;
Mon, 06 Jun 2011 19:08:46 +0200 wenzelm moved incr_boundvars;
Mon, 06 Jun 2011 18:05:38 +0200 wenzelm modernized and re-unified Thm.transfer;
Mon, 06 Jun 2011 17:51:14 +0200 wenzelm removed obsolete material (superseded by implementation manual);
Sun, 05 Jun 2011 22:09:04 +0200 wenzelm removed somewhat low-level stuff (cf. attribute "swapped" in isar-ref);
Sun, 05 Jun 2011 22:02:54 +0200 wenzelm updated and re-unified classical proof methods;
Sun, 05 Jun 2011 20:23:05 +0200 wenzelm tuned;
Sun, 05 Jun 2011 20:15:47 +0200 wenzelm updated and re-unified classical rule declarations;
Sat, 04 Jun 2011 22:09:42 +0200 wenzelm moved/updated introduction to Classical Reasoner;
Sat, 04 Jun 2011 19:39:45 +0200 wenzelm tuned secref (still dangling);
Fri, 03 Jun 2011 22:39:23 +0200 wenzelm updated and re-unified material on simprocs;
Fri, 03 Jun 2011 21:32:48 +0200 wenzelm removed some old stuff;
Thu, 02 Jun 2011 14:11:24 +0200 wenzelm tuned headings;
Thu, 02 Jun 2011 14:08:46 +0200 wenzelm some material on "Generalized elimination and cases";
Thu, 02 Jun 2011 13:59:23 +0200 wenzelm some material on "Structured induction proofs";
Wed, 01 Jun 2011 13:06:45 +0200 wenzelm some material on "Structured Natural Deduction";
Wed, 01 Jun 2011 12:39:04 +0200 wenzelm some material on "Calculational reasoning";
Wed, 01 Jun 2011 12:20:48 +0200 wenzelm tuned;
Tue, 31 May 2011 22:47:18 +0200 wenzelm added Synopsis, with some "Notepad" material;
Tue, 31 May 2011 22:18:37 +0200 wenzelm more accurate deps;
Tue, 31 May 2011 22:15:39 +0200 wenzelm turned "Overview" into "Preface" (similar to doc-src/Intro/intro.tex);
Thu, 26 May 2011 22:42:52 +0200 wenzelm moved/updated basic HOL overview;
Thu, 26 May 2011 21:39:02 +0200 wenzelm updated and re-unified (co)inductive definitions in HOL;
Thu, 26 May 2011 15:56:39 +0200 wenzelm clarified current 'primrec' vs. old 'recdef';
Thu, 26 May 2011 14:24:26 +0200 wenzelm record examples;
Thu, 26 May 2011 14:12:14 +0200 wenzelm updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
Thu, 26 May 2011 13:37:11 +0200 wenzelm updated and re-unified HOL rep_datatype;
Wed, 25 May 2011 22:21:38 +0200 wenzelm rearranged some sections;
Wed, 25 May 2011 22:12:46 +0200 wenzelm updated and re-unified HOL typedef, with some live examples;
Sat, 21 May 2011 11:31:59 +0200 wenzelm optional jedit_build/etc/user-settings enable to override defaults produced by late component initialization;
Sat, 21 May 2011 00:09:18 +0200 wenzelm merged
Fri, 20 May 2011 21:38:32 +0200 hoelzl add divide_.._cancel, inverse_.._iff
Fri, 20 May 2011 21:38:32 +0200 hoelzl add surj_vimage_empty
Fri, 20 May 2011 21:38:32 +0200 hoelzl Add restricted borel measure to {0 .. 1}
Fri, 20 May 2011 21:38:32 +0200 hoelzl equations for subsets of atLeastAtMost
Sat, 21 May 2011 00:01:15 +0200 wenzelm build and run Isabelle/jEdit on the spot -- requires auxiliary "jedit_build" component;
Sat, 21 May 2011 00:00:14 +0200 wenzelm misc tuning and update;
Fri, 20 May 2011 23:59:46 +0200 wenzelm updated versions;
Fri, 20 May 2011 20:44:03 +0200 wenzelm added Isabelle_Process.is_active;
Fri, 20 May 2011 18:12:12 +0200 blanchet update example
Fri, 20 May 2011 18:01:46 +0200 blanchet name tuning
Fri, 20 May 2011 17:16:13 +0200 blanchet further improvements to "poly_{preds,tags}_{bang,query}" -- better solution to the combinator problem + make sure type assumptions can be discharged
Fri, 20 May 2011 17:16:13 +0200 blanchet prevent unsound combinator proofs in partially typed polymorphic type systems
Fri, 20 May 2011 16:23:03 +0200 hoelzl add lemma prob_finite_product
Fri, 20 May 2011 16:22:24 +0200 hoelzl simp rules for empty intervals on dense linear order
Fri, 20 May 2011 14:12:59 +0200 wenzelm merged
Fri, 20 May 2011 12:59:33 +0200 blanchet exercise more type systems (but only sound or quasi-sound ones)
Fri, 20 May 2011 12:47:59 +0200 blanchet added see also
Fri, 20 May 2011 12:47:59 +0200 blanchet document new type system and soundness properties of the different systems
Fri, 20 May 2011 12:47:59 +0200 blanchet improved "poly_preds_{bang,query}" by picking up good witnesses for the possible infinity of common type classes and ensuring that "?'a::type" doesn't ruin everything
Fri, 20 May 2011 12:47:59 +0200 blanchet reintroduced type encodings "poly_preds_{bang,query}", but this time being more liberal about type variables of known safe sorts
Fri, 20 May 2011 12:47:59 +0200 blanchet more doc fiddling
Fri, 20 May 2011 12:47:59 +0200 blanchet more FAQs
Fri, 20 May 2011 12:47:59 +0200 blanchet make sure the Vampire incomplete proof detection code kicks in
Fri, 20 May 2011 12:47:59 +0200 blanchet automatically use "metisFT" when typed helpers are necessary
Fri, 20 May 2011 12:47:58 +0200 blanchet tuning
Fri, 20 May 2011 12:47:58 +0200 blanchet generate useful information for type axioms
Fri, 20 May 2011 12:47:58 +0200 blanchet slightly fewer type predicates introduced in the lightweight encoding, based on the observation that only universal positive equalities are dangerous
Fri, 20 May 2011 12:47:58 +0200 blanchet updated FAQ
Fri, 20 May 2011 12:47:58 +0200 blanchet more informative message when Sledgehammer finds an unsound proof
Fri, 20 May 2011 12:35:44 +0200 haftmann tuned proofs
Fri, 20 May 2011 12:09:54 +0200 haftmann NEWS
Fri, 20 May 2011 12:07:17 +0200 haftmann point-free characterization of operations on finite sets
Fri, 20 May 2011 11:44:34 +0200 haftmann merged
(0) -30000 -10000 -3000 -1000 -192 +192 +1000 +3000 +10000 +30000 tip