Fri, 04 Nov 2011 17:19:33 +0100 wenzelm prefer global Quotient_Info lookup to accomodate Quotient_Term, which is not quite localized yet (cf. 9fd6fce8a230);
Fri, 04 Nov 2011 15:05:59 +0000 blanchet document new experimental provers
Fri, 04 Nov 2011 15:05:58 +0000 blanchet added remote iProver(-Eq) for experimentation
Fri, 04 Nov 2011 13:52:19 +0100 wenzelm merged
Fri, 04 Nov 2011 08:19:24 +0100 huffman ex/Tree23.thy: automate proof of gfull_add
Fri, 04 Nov 2011 08:00:48 +0100 huffman ex/Tree23.thy: simplify proof of bal_del0
Fri, 04 Nov 2011 07:37:37 +0100 huffman ex/Tree23.thy: simplify proof of bal_add0
Fri, 04 Nov 2011 07:04:34 +0100 huffman ex/Tree23.thy: simpler definition of ordered-ness predicate
Thu, 03 Nov 2011 17:40:50 +0100 huffman ex/Tree23.thy: prove that deletion preserves balance
Fri, 04 Nov 2011 00:07:45 +0100 wenzelm more liberal Parse.fixes, to avoid overlap of mixfix with is-pattern (notably in 'obtain' syntax);
Thu, 03 Nov 2011 23:55:53 +0100 wenzelm more general Proof_Context.bind_propp, which allows outer parameters;
Thu, 03 Nov 2011 23:32:31 +0100 wenzelm tuned whitespace;
Thu, 03 Nov 2011 22:51:37 +0100 wenzelm tuned signature;
Thu, 03 Nov 2011 22:23:41 +0100 wenzelm tuned signature -- canonical argument order;
Thu, 03 Nov 2011 22:15:47 +0100 wenzelm tuned -- Variable.declare_term is already part of Variable.auto_fixes;
Thu, 03 Nov 2011 11:18:06 +0100 huffman ex/Tree23.thy: prove that insertion preserves tree balance and order
Thu, 03 Nov 2011 18:10:47 +1100 kleing more IMP fragments
Thu, 03 Nov 2011 18:10:13 +1100 kleing string -> vname
Thu, 03 Nov 2011 16:22:29 +1100 kleing JMPF(LESS|GE) -> JMP(LESS|GE) because jumps are int now.
Thu, 03 Nov 2011 15:54:19 +1100 kleing more IMP text fragments
Thu, 03 Nov 2011 10:29:05 +1100 kleing moved latex generation for HOL-IMP out of distribution
Tue, 01 Nov 2011 10:05:28 +0100 bulwahn renaming Quotient_Set and List_Quotient_Set to Quotient_Cset and List_Quotient_Cset to avoid name clash with existing Quotient_Set (again, cf. 66823a0066db)
Mon, 31 Oct 2011 19:12:41 +0100 bulwahn merged
Mon, 31 Oct 2011 18:29:25 +0100 bulwahn more robust, declarative and unsurprising computation of types in the quotient type definition
Mon, 31 Oct 2011 17:51:01 +0100 blanchet improve handling of bound type variables (esp. for TFF1)
Mon, 31 Oct 2011 17:51:01 +0100 blanchet improved TFF1 output
Mon, 31 Oct 2011 08:50:35 +0100 bulwahn clarified signature
Mon, 31 Oct 2011 08:43:21 +0100 bulwahn tuned
Mon, 31 Oct 2011 08:22:56 +0100 bulwahn tuned
Sun, 30 Oct 2011 22:35:18 +0100 wenzelm even more uniform Local_Theory.declaration for locales (cf. 57def0b39696, aa35859c8741);
Sun, 30 Oct 2011 22:20:45 +0100 wenzelm removed obsolete argument (cf. aa35859c8741);
Sun, 30 Oct 2011 09:42:13 +0100 huffman removed ad-hoc simp rules sin_cos_eq[symmetric], minus_sin_cos_eq[symmetric], cos_sin_eq[symmetric]
Sun, 30 Oct 2011 09:07:02 +0100 huffman extend cancellation simproc patterns to cover terms like '- (2 * pi) < pi'
Sun, 30 Oct 2011 07:08:33 +0100 huffman merged
Sat, 29 Oct 2011 10:00:35 +0200 huffman remove unused function
Sat, 29 Oct 2011 13:51:35 +0200 blanchet also export DFG formats
Sat, 29 Oct 2011 13:15:58 +0200 blanchet always use DFG format to talk to SPASS -- since that's what we'll need to use anyway to benefit from sorts and other extensions
Sat, 29 Oct 2011 13:15:58 +0200 blanchet added DFG unsorted support (like in the old days)
Sat, 29 Oct 2011 13:15:58 +0200 blanchet gracefully do nothing if the SPASS input file is already in DFG format
Sat, 29 Oct 2011 13:15:58 +0200 blanchet added sorted DFG output for coming version of SPASS
Sat, 29 Oct 2011 13:15:58 +0200 blanchet specify proof output level 1 (i.e. no detailed, potentially huge E proofs) to LEO-II; requires version 1.2.9
Sat, 29 Oct 2011 13:15:58 +0200 blanchet check "sound" flag before doing something unsound...
Sat, 29 Oct 2011 12:57:43 +0200 wenzelm uniform treatment of syntax declaration wrt. aux. context (NB: notation avoids duplicate mixfix internally);
Sat, 29 Oct 2011 12:55:34 +0200 wenzelm tuned;
Fri, 28 Oct 2011 16:49:15 +0200 huffman more accurate class constraints on cancellation simproc patterns
Sat, 29 Oct 2011 00:23:58 +0200 wenzelm tuned;
Fri, 28 Oct 2011 23:41:16 +0200 wenzelm tuned Named_Thms: proper binding;
Fri, 28 Oct 2011 23:16:50 +0200 wenzelm refined Local_Theory.declaration {syntax = false, pervasive} semantics: update is applied to auxiliary context as well;
Fri, 28 Oct 2011 23:10:44 +0200 wenzelm more robust data storage (NB: the morphism can change the shape of qconst, and in the auxiliary context it is not even a constant yet);
Fri, 28 Oct 2011 22:17:30 +0200 wenzelm uniform Local_Theory.declaration with explicit params;
Fri, 28 Oct 2011 17:15:52 +0200 wenzelm tuned signature -- refined terminology;
Fri, 28 Oct 2011 15:38:41 +0200 wenzelm slightly more explicit/syntactic modelling of morphisms;
Fri, 28 Oct 2011 14:10:19 +0200 hoelzl correct import path
Fri, 28 Oct 2011 14:06:06 +0200 hoelzl allow to build Probability and MV-Analysis with one ROOT.ML
Fri, 28 Oct 2011 12:37:18 +0200 bulwahn removing dead code
Fri, 28 Oct 2011 10:33:23 +0200 huffman ex/Simproc_Tests.thy: remove duplicate simprocs
Fri, 28 Oct 2011 11:02:27 +0200 huffman use simproc_setup for cancellation simprocs, to get proper name bindings
Thu, 27 Oct 2011 22:37:19 +0200 wenzelm tuned;
Thu, 27 Oct 2011 22:20:55 +0200 wenzelm eliminated aliases of standard functions;
Thu, 27 Oct 2011 21:52:57 +0200 wenzelm more standard attribute setup;
Thu, 27 Oct 2011 21:02:10 +0200 wenzelm localized quotient data;
Thu, 27 Oct 2011 20:26:38 +0200 wenzelm simplified/standardized signatures;
Thu, 27 Oct 2011 19:41:08 +0200 wenzelm tuned signature;
Thu, 27 Oct 2011 16:28:34 +0200 nipkow uses IMP and hence requires its tex setup
Thu, 27 Oct 2011 15:59:33 +0200 nipkow merged
Thu, 27 Oct 2011 15:59:25 +0200 nipkow tuned text
Thu, 27 Oct 2011 13:52:31 +0200 bulwahn respecting isabelle's programming style in the quotient package by simplifying qconsts_lookup function for data access; removing odd NotFound exception
Thu, 27 Oct 2011 13:50:55 +0200 bulwahn respecting isabelle's programming style in the quotient package by simplifying map_lookup function for data access
Thu, 27 Oct 2011 13:50:54 +0200 bulwahn respecting isabelle's programming style in the quotient package by simplifying quotdata_lookup function for data access
Thu, 27 Oct 2011 07:48:07 +0200 huffman merged
Thu, 27 Oct 2011 07:46:57 +0200 huffman fix bug in cancel_factor simprocs so they will work on goals like 'x * y < x * z' where the common term is already on the left
Wed, 26 Oct 2011 22:51:06 +0200 wenzelm more robust ML pretty printing (cf. b6c527c64789);
Wed, 26 Oct 2011 22:50:40 +0200 wenzelm tuned;
Tue, 25 Oct 2011 16:37:11 +0200 bulwahn renaming Cset and List_Cset in Quotient_Examples to Quotient_Set and List_Quotient_Set to avoid a name clash of theory names with the ones in HOL-Library
Tue, 25 Oct 2011 16:09:02 +0200 nipkow tuned text
Tue, 25 Oct 2011 15:59:15 +0200 nipkow tuned names to avoid shadowing
Tue, 25 Oct 2011 12:00:52 +0200 huffman merge Gcd/GCD and Lcm/LCM
Tue, 25 Oct 2011 08:48:36 +0200 boehmes clarify types of terms: use proper set type
Mon, 24 Oct 2011 16:47:24 +0200 huffman instance bool :: linorder
Mon, 24 Oct 2011 12:26:05 +0200 bulwahn removing poor man's dictionary construction which were only for the ancient code generator with no support of type classes
Mon, 24 Oct 2011 11:40:31 +0200 bulwahn fixed typo
Mon, 24 Oct 2011 10:45:54 +0200 nipkow latex output not needed because errors manifest themselves earlier
Sun, 23 Oct 2011 23:11:53 +0200 wenzelm some text on inner-syntax;
Sun, 23 Oct 2011 16:03:59 +0200 nipkow renamed in ASM
Sun, 23 Oct 2011 14:15:24 +0200 nipkow tuned order of eqns
Sun, 23 Oct 2011 14:03:37 +0200 nipkow tuned
Sun, 23 Oct 2011 17:37:21 +1100 kleing script for exporting filtered IMP files as tar.gz
Sun, 23 Oct 2011 17:12:14 +1100 kleing removed Norbert's email from isatest (bounces)
Sat, 22 Oct 2011 23:43:01 +0200 wenzelm class Lexicon as abstract datatype;
Sat, 22 Oct 2011 23:30:02 +0200 wenzelm more private stuff;
Sat, 22 Oct 2011 23:29:44 +0200 wenzelm class Text.Edit as abstract datatype;
Sat, 22 Oct 2011 23:29:11 +0200 wenzelm class Time as abstract datatype;
Sat, 22 Oct 2011 23:28:24 +0200 wenzelm class Volatile as abstract datatype;
Sat, 22 Oct 2011 20:18:01 +0200 nipkow merged
Sat, 22 Oct 2011 20:17:50 +0200 nipkow added isaverbatimwrite that allows to cut out snippets of thy files in their latex form and dump them in a file
Sat, 22 Oct 2011 19:22:13 +0200 wenzelm experimental support for Scala 2.9.1.final;
Sat, 22 Oct 2011 19:15:32 +0200 wenzelm class Path as abstract datatype;
Sat, 22 Oct 2011 19:00:03 +0200 wenzelm class Counter as abstract datatype;
Sat, 22 Oct 2011 16:57:24 +0200 wenzelm discontinued redundant ASCII syntax;
Sat, 22 Oct 2011 16:44:34 +0200 wenzelm modernized specifications;
Fri, 21 Oct 2011 22:44:55 +0200 wenzelm proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
Fri, 21 Oct 2011 17:39:07 +0200 nipkow merged
Fri, 21 Oct 2011 17:39:00 +0200 nipkow tuned
Fri, 21 Oct 2011 16:21:12 +0200 wenzelm merged
Fri, 21 Oct 2011 14:25:38 +0200 bulwahn replacing metis proofs with facts xt1 by new proof with more readable names
Fri, 21 Oct 2011 14:06:15 +0200 blanchet more robust parsing of TSTP sources -- Vampire has nonstandard "introduced()" tags and Waldmeister(OnTPTP) has weird "theory(...)" dependencies
Fri, 21 Oct 2011 12:44:20 +0200 blanchet disable Vampire's BDD optimization, which sometimes yields so huge proofs that this causes problems for reconstruction
Fri, 21 Oct 2011 11:17:16 +0200 bulwahn NEWS
Fri, 21 Oct 2011 11:17:15 +0200 bulwahn updating documentation: code_inline -> code_unfold; added documentation about attribute code_unfold_post
Fri, 21 Oct 2011 11:17:14 +0200 bulwahn replacing code_inline by code_unfold, removing obsolete code_unfold, code_inline del now that the ancient code generator is removed
Fri, 21 Oct 2011 11:17:12 +0200 bulwahn removing redundant attribute code_inline in the code generator
Fri, 21 Oct 2011 11:27:21 +0200 wenzelm tuned;
Fri, 21 Oct 2011 11:26:14 +0200 wenzelm tuned;
Fri, 21 Oct 2011 10:37:03 +0200 bulwahn improving mutabelle script again after missing some changes in f4896c792316
Fri, 21 Oct 2011 10:32:42 +0200 bulwahn correcting code_prolog
Fri, 21 Oct 2011 09:51:45 +0200 huffman merged
Fri, 21 Oct 2011 08:42:11 +0200 huffman add HOL/ex/Simproc_Tests.thy: testing for Tools/numeral_simprocs.ML
Fri, 21 Oct 2011 08:25:04 +0200 nipkow merged
Fri, 21 Oct 2011 08:24:57 +0200 nipkow tuned
Thu, 20 Oct 2011 22:26:02 +0200 blanchet mark "xt..." rules as "no_atp", since they are easy consequences of other better named properties
Thu, 20 Oct 2011 22:02:49 +0200 huffman merged
Thu, 20 Oct 2011 17:27:14 +0200 huffman removed mult_Bit1 from int_arith_rules (cf. 882403378a41 and 3078fd2eec7b, where mult_num1 erroneously replaced mult_1)
Thu, 20 Oct 2011 12:30:43 -0400 kleing removed [trans] concept from basic material
Thu, 20 Oct 2011 10:44:00 +0200 nipkow merged
Thu, 20 Oct 2011 10:43:47 +0200 nipkow tuned
Thu, 20 Oct 2011 09:59:12 +0200 bulwahn merged
Thu, 20 Oct 2011 09:11:13 +0200 bulwahn modernizing predicate_compile_quickcheck
Thu, 20 Oct 2011 08:20:35 +0200 bulwahn adding depth as an quickcheck configuration
Thu, 20 Oct 2011 09:48:00 +0200 nipkow renamed name -> vname
Wed, 19 Oct 2011 23:07:48 +0200 haftmann removed some remaining artefacts of ancient SML code generator
Wed, 19 Oct 2011 22:54:26 +0200 haftmann NEWS
Wed, 19 Oct 2011 21:40:32 +0200 blanchet cleaner LEO-II extensionality step detection
Wed, 19 Oct 2011 21:40:32 +0200 blanchet marginally cleaner proof parsing, that doesn't stumble upon LEO-II's E-step proofs
Wed, 19 Oct 2011 21:40:32 +0200 blanchet one more LEO-II failure
Wed, 19 Oct 2011 19:45:19 +0200 wenzelm merged
Wed, 19 Oct 2011 17:45:25 +0200 huffman merged
Tue, 18 Oct 2011 15:19:06 +0200 huffman hide typedef-generated constants Product_Type.prod and Sum_Type.sum
Wed, 19 Oct 2011 16:36:13 +0200 blanchet more uniform SZS status handling
Wed, 19 Oct 2011 16:36:13 +0200 blanchet avoid generating too meta theorems -- this sometimes leads to type errors, e.g. when "pp" is applied to a "prop" instead of a "bool"
Wed, 19 Oct 2011 16:32:30 +0200 nipkow merged
Wed, 19 Oct 2011 16:32:12 +0200 nipkow renamed B to Bc
Wed, 19 Oct 2011 17:04:43 +0200 wenzelm tuned comment;
Wed, 19 Oct 2011 17:03:07 +0200 wenzelm proper source positions for @{lemma};
Wed, 19 Oct 2011 16:45:46 +0200 wenzelm more robust toplevel_error reporting (NB: Context.proof_of on a stale theory crashes ungracefully);
Wed, 19 Oct 2011 15:42:43 +0200 wenzelm inlined @{thms} (ML compile-time) allows to get rid of legacy zadd_ac as well (cf. 49e305100097);
Wed, 19 Oct 2011 15:41:12 +0200 wenzelm tuned legacy signature;
Wed, 19 Oct 2011 14:40:49 +0200 wenzelm further cleanup of stats (cf. 97e81a8aa277);
Wed, 19 Oct 2011 14:22:06 +0200 wenzelm updated keywords;
Wed, 19 Oct 2011 14:21:29 +0200 wenzelm really document just one code generator;
Wed, 19 Oct 2011 09:11:21 +0200 bulwahn NEWS
Wed, 19 Oct 2011 09:11:20 +0200 bulwahn removing old code generator
Wed, 19 Oct 2011 09:11:19 +0200 bulwahn removing declaration of code_unfold to address the old code generator
Wed, 19 Oct 2011 09:11:18 +0200 bulwahn removing dependency of the generic code generator to old code generator functions thyname_of_type and thyname_of_const
Wed, 19 Oct 2011 09:11:18 +0200 bulwahn removing documentation about the old code generator
Wed, 19 Oct 2011 09:11:16 +0200 bulwahn removing old code generator setup for executable sets
Wed, 19 Oct 2011 09:11:15 +0200 bulwahn removing old code generator setup for efficient natural numbers; cleaned typo
Wed, 19 Oct 2011 09:11:14 +0200 bulwahn removing old code generator setup for real numbers; tuned
Wed, 19 Oct 2011 09:11:14 +0200 bulwahn removing old code generator setup for rational numbers; tuned
Wed, 19 Oct 2011 08:37:29 +0200 bulwahn removing old code generator setup for strings
Wed, 19 Oct 2011 08:37:27 +0200 bulwahn removing old code generator setup for lists
Wed, 19 Oct 2011 08:37:26 +0200 bulwahn removing old code generator setup for integers
Wed, 19 Oct 2011 08:37:25 +0200 bulwahn removing old code generator for inductive predicates
Wed, 19 Oct 2011 08:37:24 +0200 bulwahn removing quickcheck tester SML-inductive based on the old code generator
Wed, 19 Oct 2011 08:37:23 +0200 bulwahn removing old code generator setup for inductive sets in the inductive set package
Wed, 19 Oct 2011 08:37:22 +0200 bulwahn removing old code generator setup of inductive predicates
Wed, 19 Oct 2011 08:37:21 +0200 bulwahn removing old code generator setup for product types
Wed, 19 Oct 2011 08:37:20 +0200 bulwahn removing old code generator setup for function types
Wed, 19 Oct 2011 08:37:19 +0200 bulwahn removing old code generator setup for datatypes
Wed, 19 Oct 2011 08:37:17 +0200 bulwahn removing old code generator for recursive functions
Wed, 19 Oct 2011 08:37:16 +0200 bulwahn removing old code generator setup in the HOL theory
Wed, 19 Oct 2011 08:37:15 +0200 bulwahn removing invocations of the evaluation method based on the old code generator
Wed, 19 Oct 2011 08:37:14 +0200 bulwahn removing invocations of the old code generator
Tue, 18 Oct 2011 15:40:59 +0200 blanchet freeze conjecture schematics before applying lambda-translation, which sometimes calls "close_form" and ruins it for freezing
Tue, 18 Oct 2011 15:40:58 +0200 blanchet gracefully handle quantifiers of the form "All $ t" where "t" is not a lambda-abstraction in higher-order translations
Tue, 18 Oct 2011 15:27:18 +0200 bulwahn tuned
Tue, 18 Oct 2011 15:27:17 +0200 bulwahn adding testing of quickcheck narrowing with finite types to mutabelle script; modified is_executable in mutabelle_extra
Tue, 18 Oct 2011 11:59:03 +0200 krauss mira: collect size of heap images
Mon, 17 Oct 2011 21:37:38 +0200 blanchet updated doc related to Satallax
Mon, 17 Oct 2011 21:37:37 +0200 blanchet parse Satallax unsat cores
Mon, 17 Oct 2011 18:05:14 +0200 wenzelm merged
Mon, 17 Oct 2011 14:22:14 +0200 noschinl (old) NEWS
Mon, 17 Oct 2011 10:19:01 +0200 bulwahn moving some common functions from quickcheck to the more HOL-specific quickcheck_common; renamed inductive_SML's configurations to more canonical names; adds automatically left and right hand sides of equations as evaluation terms
Mon, 17 Oct 2011 11:24:22 +0200 wenzelm always use sockets on Windows/Cygwin;
Sun, 16 Oct 2011 21:49:47 +0200 krauss mira configuration: use official polyml 5.4.1 on lxbroy10
Sun, 16 Oct 2011 18:48:30 +0200 wenzelm added Term.dummy_pattern conveniences;
Sun, 16 Oct 2011 16:56:01 +0200 wenzelm slightly more standard-conformant XML parsing (see also 94033767ef9b);
Sun, 16 Oct 2011 14:48:01 +0200 haftmann tuned proof
Sun, 16 Oct 2011 14:48:00 +0200 haftmann tuned type annnotation
Sun, 16 Oct 2011 14:48:00 +0200 haftmann hide not_member as also member
Sat, 15 Oct 2011 20:40:13 +0200 wenzelm misc tuning and modernization;
Sat, 15 Oct 2011 18:14:36 +0200 wenzelm updated to Scala 2.8.2.final;
Sat, 15 Oct 2011 17:00:17 +0200 wenzelm prefer recent polyml-5.4.1, but retain potentially fragile polyml-5.2.1 as experimental test;
Sat, 15 Oct 2011 16:58:37 +0200 wenzelm updated to polyml-5.4.1;
Sat, 15 Oct 2011 15:55:10 +0200 wenzelm updated to polyml-5.4.1;
Sat, 15 Oct 2011 00:18:00 +0200 haftmann merged
Fri, 14 Oct 2011 22:42:56 +0200 haftmann monadic bind
Fri, 14 Oct 2011 18:55:59 +0200 haftmann moved sublists to More_List.thy
Fri, 14 Oct 2011 18:55:29 +0200 haftmann NEWS
Fri, 14 Oct 2011 11:34:30 +0200 wenzelm more complete stats, including small sessions which provide some clues on main HOL baseline performance;
Thu, 13 Oct 2011 23:35:15 +0200 haftmann avoid very specific code equation for card; corrected spelling
Thu, 13 Oct 2011 23:27:46 +0200 haftmann bouned transitive closure
Thu, 13 Oct 2011 23:02:59 +0200 haftmann moved acyclic predicate up in hierarchy
Thu, 13 Oct 2011 22:56:19 +0200 haftmann tuned
Thu, 13 Oct 2011 22:56:19 +0200 haftmann modernized definitions
Thu, 13 Oct 2011 22:50:35 +0200 wenzelm static dummy_task (again) to avoid a few extra allocations;
Thu, 13 Oct 2011 13:49:55 +0200 noschinl tuned markup
Thu, 13 Oct 2011 11:45:33 +0200 wenzelm discontinued obsolete 'types' command;
Wed, 12 Oct 2011 22:48:23 +0200 wenzelm modernized structure Induct_Tacs;
Wed, 12 Oct 2011 22:21:38 +0200 wenzelm tuned signature;
Wed, 12 Oct 2011 21:39:33 +0200 wenzelm misc tuning and clarification;
Wed, 12 Oct 2011 20:57:40 +0200 wenzelm tuned ML style;
Wed, 12 Oct 2011 20:16:48 +0200 wenzelm tuned proofs -- eliminated vacuous "induct arbitrary: ..." situations;
Wed, 12 Oct 2011 16:21:07 +0200 wenzelm discontinued obsolete alias structure ProofContext;
Wed, 12 Oct 2011 09:16:30 +0200 nipkow separated monotonicity reasoning and defined narrowing with while_option
Mon, 10 Oct 2011 20:14:25 +0200 wenzelm include no-smlnj targets into library (cf. e54a985daa61);
Mon, 10 Oct 2011 16:47:45 +0200 bulwahn increasing values_timeout to avoid SML_makeall failures on our current tests
Mon, 10 Oct 2011 11:12:09 +0200 wenzelm merged
Mon, 10 Oct 2011 11:10:45 +0200 wenzelm removed obsolete RC tags;
Sun, 09 Oct 2011 11:13:53 +0200 huffman Int.thy: discontinued some legacy theorems
Sun, 09 Oct 2011 08:30:48 +0200 huffman Set.thy: remove redundant [simp] declarations
Mon, 03 Oct 2011 22:21:19 +0200 bulwahn removing code equation for card on finite types when loading the Executable_Set theory; should resolve a code generation issue with CoreC++
Mon, 03 Oct 2011 15:39:30 +0200 bulwahn tune text for document generation
Mon, 03 Oct 2011 14:43:15 +0200 bulwahn adding examples with relations to Quickcheck_Examples to show that quickcheck can actually handle operators on relations as well
Mon, 03 Oct 2011 14:43:14 +0200 bulwahn adding code equations for cardinality and (reflexive) transitive closure on finite types
Mon, 03 Oct 2011 14:43:13 +0200 bulwahn adding lemma about rel_pow in Transitive_Closure for executable equation of the (refl) transitive closure
Mon, 03 Oct 2011 14:43:12 +0200 bulwahn adding lemma to List library for executable equation of the (refl) transitive closure
Thu, 29 Sep 2011 21:42:03 +0200 Jean Pichon fixed typos in IMP
Wed, 28 Sep 2011 10:35:56 +0200 nipkow added nice interval syntax
Wed, 28 Sep 2011 09:59:55 +0200 nipkow Added dependecies
Wed, 28 Sep 2011 09:55:11 +0200 nipkow Added Hoare-like Abstract Interpretation
Wed, 28 Sep 2011 08:51:55 +0200 nipkow moved IMP/AbsInt stuff into subdirectory Abs_Int_Den
Mon, 26 Sep 2011 21:13:26 +0200 wenzelm back to post-release mode;
Sun, 09 Oct 2011 17:06:19 +0200 wenzelm Added tag Isabelle2011-1 for changeset 76fef3e57004
Sun, 09 Oct 2011 16:47:58 +0200 wenzelm tuned; Isabelle2011-1
Sun, 09 Oct 2011 15:46:06 +0200 wenzelm updated ISABELLE_HOME_USER;
Tue, 04 Oct 2011 14:51:51 +0200 wenzelm more explicit check of Java executable -- relevant for Linux x86/x86_64 mismatch and absence on Mac OS Lion;
Mon, 03 Oct 2011 11:16:51 +0200 wenzelm Added tag Isabelle2011-1-RC2 for changeset a45121ffcfcb
Mon, 03 Oct 2011 11:14:19 +0200 wenzelm some amendments due to Jean Pichon;
Thu, 29 Sep 2011 09:37:59 +0200 traytel correct coercion generation in case of unknown map functions
Wed, 28 Sep 2011 13:52:14 +0200 wenzelm proper platform_file_url for Windows UNC paths (server shares);
Tue, 27 Sep 2011 22:35:57 +0200 wenzelm proper platform_file_url;
Tue, 27 Sep 2011 22:14:15 +0200 wenzelm observe base URL of rendered document;
Tue, 27 Sep 2011 21:39:55 +0200 wenzelm more README;
Tue, 27 Sep 2011 20:45:15 +0200 wenzelm tuned README.html;
Tue, 27 Sep 2011 20:25:15 +0200 wenzelm tuned;
Tue, 27 Sep 2011 14:17:40 +0200 wenzelm retain output, which is required for non-existent JRE, for example (cf. b455e4f42c04);
Tue, 27 Sep 2011 00:03:11 +0200 wenzelm tuned message, which is displayed after termination of Isabelle.app on Mac OS;
Mon, 26 Sep 2011 23:51:59 +0200 wenzelm keep top-level "Isabelle" executable -- now an alias for "isabelle jedit";
Mon, 26 Sep 2011 23:43:52 +0200 wenzelm tuned;
Mon, 26 Sep 2011 21:41:39 +0200 wenzelm ensure Isabelle env;
Mon, 26 Sep 2011 21:17:25 +0200 wenzelm Added tag Isabelle2011-1-RC1 for changeset 24ad77c3a147
Mon, 26 Sep 2011 21:09:28 +0200 wenzelm tuned;
Mon, 26 Sep 2011 20:53:53 +0200 wenzelm misc tuning for release;
Mon, 26 Sep 2011 20:39:18 +0200 wenzelm reverted 09cdc4209d25 for formal reasons: it did not say what was "broken" nor "fixed", but broke IsaMakefile dependencies;
Mon, 26 Sep 2011 20:31:41 +0200 wenzelm makedist for release;
Mon, 26 Sep 2011 14:03:43 +0200 blanchet put MiniSat back first -- Torlak's eval seemed to suggest that Crypto and Lingeling were better, but Crypto is slower on "Nitpick_Examples" and Crypto crashes
Mon, 26 Sep 2011 11:41:52 +0200 blanchet require Java 1.6 in the Nitpick documentation -- technically 1.5 will also work with Kodkodi 1.2.16, but it won't work with Kodkodi 1.5.0
Mon, 26 Sep 2011 11:41:52 +0200 blanchet put CryptoMiniSat first and remove warning about unsoundness now that it has been fixed in Kodkod
Mon, 26 Sep 2011 10:57:20 +0200 bulwahn adding an example with inductive predicates to quickcheck narrowing examples
Mon, 26 Sep 2011 10:30:37 +0200 bulwahn importing the Generated_Code module qualified to reduce the probability of name clashes between the static code and the generated code in the narrowing-based Quickcheck
Sun, 25 Sep 2011 19:34:20 +0200 blanchet clarify platforms
Sun, 25 Sep 2011 18:43:25 +0200 blanchet killed JNI version of zChaff, since Kodkod 1.5 does not support it anymore
Sun, 25 Sep 2011 18:43:25 +0200 blanchet updated Nitpick SAT Solver doc
Sun, 25 Sep 2011 18:43:25 +0200 blanchet update list of SAT solvers reflecting Kodkod 1.5
Sun, 25 Sep 2011 17:25:34 +0200 wenzelm tuned signature;
Sun, 25 Sep 2011 13:48:59 +0200 wenzelm more uniform defaults;
Sun, 25 Sep 2011 09:37:33 +0200 haftmann Quotient_Set.thy is part of library
Sun, 25 Sep 2011 00:32:49 +0200 nipkow fixed typo
Sat, 24 Sep 2011 17:18:39 +0200 wenzelm standardize drive letters -- important for proper document node identification;
Sat, 24 Sep 2011 10:45:57 +0200 wenzelm more user aliases;
Sat, 24 Sep 2011 00:17:32 +0100 sultana fixed IsaMakefile action for HOL-TPTP.
Fri, 23 Sep 2011 23:46:13 +0200 wenzelm prefer socket comminication on Cygwin, which is more stable here than fifos;
Fri, 23 Sep 2011 21:51:49 +0200 wenzelm tuned proof;
Fri, 23 Sep 2011 17:35:06 +0200 wenzelm made SML/NJ happy;
Fri, 23 Sep 2011 17:23:54 +0200 wenzelm discontinued stream-based Socket_IO, which causes too many problems with Poly/ML and SML/NJ (reverting major parts of 5c0b0d67f9b1);
Fri, 23 Sep 2011 17:11:08 +0200 wenzelm updated header;
Fri, 23 Sep 2011 16:50:39 +0200 wenzelm merged;
Fri, 23 Sep 2011 16:44:51 +0200 blanchet reintroduced E-SInE now that it's unexpectedly working again (thanks to Geoff)
Fri, 23 Sep 2011 14:25:53 +0200 blanchet first step towards extending Minipick with more translations
Fri, 23 Sep 2011 14:08:50 +0200 berghofe Include keywords print_coercions and print_coercion_maps
Wed, 17 Aug 2011 19:49:07 +0200 traytel local coercion insertion algorithm to support complex coercions
Wed, 17 Aug 2011 19:49:07 +0200 traytel printing and deleting of coercions
Fri, 23 Sep 2011 14:59:29 +0200 wenzelm raw unbuffered socket IO, which bypasses the fragile BinIO layer in Poly/ML 5.4.x;
Fri, 23 Sep 2011 14:13:15 +0200 wenzelm default print mode for Isabelle/Scala, not just Isabelle/jEdit;
Fri, 23 Sep 2011 14:12:09 +0200 wenzelm augment existing print mode;
Fri, 23 Sep 2011 13:44:31 +0200 wenzelm explicit option for socket vs. fifo communication;
Fri, 23 Sep 2011 13:43:44 +0200 wenzelm tuned proof;
Fri, 23 Sep 2011 10:31:12 +0200 blanchet synchronized section names with manual
Fri, 23 Sep 2011 00:11:29 +0200 wenzelm merged;
Thu, 22 Sep 2011 14:12:16 -0700 huffman discontinued legacy theorem names from RealDef.thy
Thu, 22 Sep 2011 13:17:14 -0700 huffman merged
Thu, 22 Sep 2011 12:55:19 -0700 huffman discontinued HOLCF legacy theorem names
Thu, 22 Sep 2011 19:42:06 +0200 blanchet take out remote E-SInE -- it's broken and Geoff says it might take quite a while before he gets to it, plus it's fairly obsolete in the meantime
Thu, 22 Sep 2011 18:23:38 +0200 berghofe Moved extraction part of Higman's lemma to separate theory to allow reuse in
Thu, 22 Sep 2011 17:15:46 +0200 berghofe Removed hcentering and vcentering options, since they are not supported
Thu, 22 Sep 2011 16:56:19 +0200 berghofe merged
Thu, 22 Sep 2011 16:50:23 +0200 berghofe Added documentation for HOL-SPARK
Thu, 22 Sep 2011 16:30:47 +0200 blanchet drop partial monomorphic instances in Metis, like in Sledgehammer
Thu, 22 Sep 2011 16:30:47 +0200 blanchet better type reconstruction -- prevents ill-instantiations in proof replay
Thu, 22 Sep 2011 10:02:16 -0400 hoelzl NEWS: mention replacement lemmas for the removed ones in Complete_Lattices
Thu, 22 Sep 2011 10:48:53 +0200 bulwahn changing quickcheck_timeout to 30 seconds in mutabelle's testing
Thu, 22 Sep 2011 07:26:53 +0200 bulwahn adding post-processing of terms to narrowing-based Quickcheck
Wed, 21 Sep 2011 17:43:13 -0700 huffman HOL/ex/ROOT.ML: only list BinEx once
Wed, 21 Sep 2011 10:59:55 -0700 huffman merged
Wed, 21 Sep 2011 08:28:53 -0700 huffman remove redundant instantiation ereal :: power
Wed, 21 Sep 2011 15:55:16 +0200 blanchet reintroduced Minipick as Nitpick example
Wed, 21 Sep 2011 15:55:15 +0200 blanchet tuned comment
Wed, 21 Sep 2011 06:41:34 -0700 huffman merged
Tue, 20 Sep 2011 11:02:41 -0700 huffman Extended_Real_Limits: generalize some lemmas
Tue, 20 Sep 2011 10:52:08 -0700 huffman add lemmas within_empty and tendsto_bot;
Thu, 22 Sep 2011 21:58:05 +0200 wenzelm made SML/NJ happy;
Thu, 22 Sep 2011 20:33:08 +0200 wenzelm abstract System_Channel in ML (cf. Scala version);
Wed, 21 Sep 2011 22:18:17 +0200 wenzelm alternative Socket_Channel;
Wed, 21 Sep 2011 20:35:50 +0200 wenzelm more abstract wrapping of fifos as System_Channel;
Wed, 21 Sep 2011 17:50:25 +0200 wenzelm slightly more general Socket_IO as part of Pure;
Wed, 21 Sep 2011 16:04:29 +0200 wenzelm more hints on Z3 configuration;
Wed, 21 Sep 2011 15:08:15 +0200 wenzelm reduced default thread stack, to increase the success rate especially on Windows (NB: the actor worker farm tends to produce 100-200 threads for big sessions);
Wed, 21 Sep 2011 07:31:08 +0200 nipkow renamed inv -> filter
Wed, 21 Sep 2011 07:04:04 +0200 nipkow Added proofs about narowing
Wed, 21 Sep 2011 07:03:16 +0200 nipkow added missing makefile dependence
Wed, 21 Sep 2011 06:26:15 +0200 nipkow added example
Wed, 21 Sep 2011 03:24:54 +0200 nipkow tuned
Wed, 21 Sep 2011 02:38:53 +0200 nipkow refined comment
Wed, 21 Sep 2011 09:17:01 +1000 kleing fixed two typos in IMP (by Jean Pichon)
Wed, 21 Sep 2011 00:12:36 +0200 nipkow merged
Tue, 20 Sep 2011 05:48:23 +0200 nipkow Updated IMP to use new induction method
Tue, 20 Sep 2011 05:47:11 +0200 nipkow New proof method "induction" that gives induction hypotheses the name IH.
Tue, 20 Sep 2011 22:11:22 +0200 haftmann official status for UN_singleton
Tue, 20 Sep 2011 21:47:52 +0200 haftmann tuned specification and lemma distribution among theories; tuned proofs
Tue, 20 Sep 2011 15:23:17 +0200 wenzelm more careful treatment of initial update, similar to output panel;
Tue, 20 Sep 2011 15:07:30 +0200 wenzelm proper fact binding;
Tue, 20 Sep 2011 09:30:19 +0200 bulwahn syntactic improvements and tuning names in the code generator due to Florian's code review
Tue, 20 Sep 2011 01:32:04 +0200 krauss match types when applying mono_thm -- previous export generalizes type variables;
Mon, 19 Sep 2011 23:34:22 +0200 wenzelm fixed headers;
Mon, 19 Sep 2011 23:24:32 +0200 wenzelm less ambiguous syntax;
Mon, 19 Sep 2011 23:18:18 +0200 wenzelm tuned proofs;
Mon, 19 Sep 2011 22:48:05 +0200 wenzelm merged
Mon, 19 Sep 2011 16:18:34 +0200 bulwahn catch PatternMatchFail exceptions in narrowing-based quickcheck
Mon, 19 Sep 2011 16:18:33 +0200 bulwahn removing superfluous definition in the quickcheck narrowing invocation as the code generator now generates valid Haskell code with necessary type annotations without a separate definition
Mon, 19 Sep 2011 16:18:30 +0200 bulwahn ensuring that some constants are generated in the source code by adding calls in ensure_testable
Mon, 19 Sep 2011 16:18:23 +0200 bulwahn adding abstraction layer; more precise function names
Mon, 19 Sep 2011 16:18:21 +0200 bulwahn adding type annotations more aggressively and redundantly to make code generation more reliable even when special printers for some constants are used
Mon, 19 Sep 2011 16:18:19 +0200 bulwahn determining the fastype of a case-pattern but ignoring dummy type constructors that were added as markers for type annotations
Mon, 19 Sep 2011 16:18:19 +0200 bulwahn only annotating constants with sort constraints
Mon, 19 Sep 2011 16:18:18 +0200 bulwahn also adding type annotations for the dynamic invocation
Mon, 19 Sep 2011 14:35:51 +0200 noschinl removed legacy lemmas in Complete_Lattices
Mon, 19 Sep 2011 14:24:53 +0200 bulwahn increasing quickcheck timeout to reduce spurious test failures due to massive parallel invocations and bad scheduling
Mon, 19 Sep 2011 22:45:57 +0200 wenzelm more isatest stats;
Mon, 19 Sep 2011 22:42:57 +0200 wenzelm refined Symbol.is_symbolic -- cover recoded versions as well;
Mon, 19 Sep 2011 22:13:51 +0200 wenzelm double clicks switch to document node buffer;
Mon, 19 Sep 2011 21:53:07 +0200 wenzelm tuned;
Mon, 19 Sep 2011 21:41:48 +0200 wenzelm explicit border independent of UI (cf. ad5883642a83, 2bec3b7514cf);
Mon, 19 Sep 2011 16:40:17 +0200 wenzelm at least 2 worker threads to ensure some degree of lifeness, notably for asynchronous Document.print_state;
Mon, 19 Sep 2011 14:40:38 +0200 wenzelm instantaneous cleanup (NB: VIEWER should be synchronous, cf. dd25b3055c4e);
Mon, 19 Sep 2011 14:31:20 +0200 wenzelm unique file names via serial numbers, to allow files like "root" or multiple files with same base name;
Mon, 19 Sep 2011 12:58:52 +0200 wenzelm imitate Apple in setting initial shell PATH -- especially relevant for MacTeX, MacPorts etc.;
Sun, 18 Sep 2011 16:12:43 -0700 huffman merged
Thu, 15 Sep 2011 10:12:36 -0700 huffman numeral_simprocs.ML: use HOL_basic_ss instead of HOL_ss for internal normalization proofs of cancel_factor simprocs, to avoid splitting if-then-else
Sun, 18 Sep 2011 21:41:36 +0200 wenzelm removed obsolete patches for PG 4.1;
Sun, 18 Sep 2011 21:15:31 +0200 wenzelm additional space for borderless UI;
Sun, 18 Sep 2011 20:26:08 +0200 wenzelm more robust treatment of empty insets (NB: border may be null on some UIs, e.g. Windows);
Sun, 18 Sep 2011 19:49:35 +0200 wenzelm explicit master_dir as part of header -- still required (for Cygwin) since Scala layer does not pass file content yet;
Sun, 18 Sep 2011 16:33:30 +0200 wenzelm isatest settings for macbroy6 (Mac OS X Lion);
Sun, 18 Sep 2011 16:24:26 +0200 wenzelm more Mac OS reference hardware;
Sun, 18 Sep 2011 16:11:26 +0200 wenzelm updated to SML/NJ 110.73;
Sun, 18 Sep 2011 15:59:38 +0200 wenzelm tentative announcement based on current NEWS;
Sun, 18 Sep 2011 15:57:36 +0200 wenzelm tuned;
Sun, 18 Sep 2011 15:39:55 +0200 wenzelm separated NEWS for Isabelle2011 from Isabelle2011-1 (cf. e1139e612b55);
Sun, 18 Sep 2011 15:30:31 +0200 wenzelm updated for release;
Sun, 18 Sep 2011 15:30:21 +0200 wenzelm tuned;
Sun, 18 Sep 2011 14:55:45 +0200 wenzelm updated generated file;
Sun, 18 Sep 2011 14:55:27 +0200 wenzelm updated Complete_Lattices;
Sun, 18 Sep 2011 14:48:25 +0200 wenzelm some tuning and re-ordering for release;
Sun, 18 Sep 2011 14:34:24 +0200 wenzelm misc tuning for release;
Sun, 18 Sep 2011 14:25:53 +0200 wenzelm more contributors;
Sun, 18 Sep 2011 14:09:57 +0200 wenzelm tuned proofs;
Sun, 18 Sep 2011 13:56:06 +0200 wenzelm tweak keyboard shortcuts for Mac OS X;
Sun, 18 Sep 2011 13:47:12 +0200 wenzelm explicit check_file wrt. jEdit VFS, to avoid slightly confusing empty buffer after IO error;
Sun, 18 Sep 2011 13:39:33 +0200 wenzelm finite sequences as useful as introductory example;
Sun, 18 Sep 2011 12:48:45 +0200 wenzelm discontinued hard-wired JAVA_HOME treatment for Mac OS X (cf. f471a2fb9a95), which can cause confusions of "isabelle java" vs. "isabelle scala" -- moved settings to external component;
Sun, 18 Sep 2011 00:05:22 +0200 wenzelm graph traversal in topological order;
Sat, 17 Sep 2011 23:04:03 +0200 wenzelm Document.Node.Name convenience;
Sat, 17 Sep 2011 22:13:15 +0200 wenzelm more precise painting;
Sat, 17 Sep 2011 21:28:52 +0200 wenzelm more elaborate Node_Renderer, which paints node_name.theory only;
Sat, 17 Sep 2011 19:55:32 +0200 wenzelm raised default log level -- to avoid confusing warning about scala.tools.nsc.plugins.Plugin, which is mistaken as jEdit plugin;
Sat, 17 Sep 2011 19:44:58 +0200 wenzelm tuned signature;
Sat, 17 Sep 2011 19:25:14 +0200 wenzelm more careful traversal of theory dependencies to retain standard import order;
Sat, 17 Sep 2011 17:55:39 +0200 wenzelm sane default for class Thy_Load;
Sat, 17 Sep 2011 17:05:31 +0200 wenzelm removed obsolete patches for PG 4.1;
Sat, 17 Sep 2011 16:53:01 +0200 wenzelm specific bundle for x86_64-linux, which is especially important for JRE due to its extra library dependencies;
Sat, 17 Sep 2011 16:29:18 +0200 wenzelm added "isabelle scalac" convenience;
Sat, 17 Sep 2011 16:19:40 +0200 wenzelm Symbol.explode as in ML;
Sat, 17 Sep 2011 16:00:54 +0200 wenzelm ignore OUTPUT to avoid spam -- jEdit menu "Troubleshooting / Activity Log" should be sufficient;
Sat, 17 Sep 2011 15:08:55 +0200 haftmann dropped unused argument – avoids problem with SML/NJ
Sat, 17 Sep 2011 00:40:27 +0200 haftmann tuned spacing
Sat, 17 Sep 2011 00:37:21 +0200 haftmann tuned
Sat, 17 Sep 2011 04:41:44 +0200 nipkow tuned post fixpoint setup
Sat, 17 Sep 2011 03:37:14 +0200 nipkow merged
Fri, 16 Sep 2011 09:18:15 +0200 nipkow when applying induction rules, remove names of assumptions that come
Fri, 16 Sep 2011 20:08:29 +0200 noschinl remove stray "using [[simp_trace]]"
Fri, 16 Sep 2011 20:02:35 +0200 noschinl tune indenting
Fri, 16 Sep 2011 12:10:43 +1000 kleing removed unused legacy lemma names, some comment cleanup.
Fri, 16 Sep 2011 12:10:15 +1000 kleing removed word_neq_0_conv from simpset, it's almost never wanted.
Thu, 15 Sep 2011 12:40:08 -0400 hoelzl removed further legacy rules from Complete_Lattices
Thu, 15 Sep 2011 17:06:00 +0200 noschinl NEWS on Complete_Lattices, Lattices
Thu, 15 Sep 2011 10:57:40 +0200 blanchet tail recursive proof preprocessing (needed for huge proofs)
Thu, 15 Sep 2011 10:57:40 +0200 blanchet tuning
Thu, 15 Sep 2011 09:44:27 +0200 nipkow merged
Thu, 15 Sep 2011 09:44:08 +0200 nipkow revised AbsInt and added widening and narrowing
Wed, 14 Sep 2011 23:47:04 +0200 haftmann updated comment
Wed, 14 Sep 2011 23:46:02 +0200 haftmann updated generated code
Tue, 13 Sep 2011 07:56:46 +0200 haftmann tuned
Wed, 14 Sep 2011 10:08:52 -0400 hoelzl renamed Complete_Lattices lemmas, removed legacy names
Wed, 14 Sep 2011 10:55:07 +0200 noschinl merged
Wed, 14 Sep 2011 10:24:22 +0200 noschinl create central list for language extensions used by the haskell code generator
Wed, 14 Sep 2011 09:46:59 +0200 boehmes observe distinction between sets and predicates
Wed, 14 Sep 2011 06:49:24 +0200 nipkow merged
Wed, 14 Sep 2011 06:49:01 +0200 nipkow cleand up AbsInt fixpoint iteration; tuned syntax
Tue, 13 Sep 2011 17:25:19 -0700 huffman tuned proofs
Tue, 13 Sep 2011 17:07:33 -0700 huffman tuned proofs
Tue, 13 Sep 2011 08:21:51 -0700 huffman remove some redundant [simp] declarations;
Tue, 13 Sep 2011 16:22:01 +0200 noschinl tune proofs
Tue, 13 Sep 2011 16:21:48 +0200 noschinl tune simpset for Complete_Lattices
Tue, 13 Sep 2011 13:17:52 +0200 bulwahn merged
Tue, 13 Sep 2011 12:14:29 +0200 bulwahn added lemma motivated by a more specific lemma in the AFP-KBPs theories
Tue, 13 Sep 2011 11:24:58 +0200 blanchet simplified unsound proof detection by removing impossible case
Tue, 13 Sep 2011 09:56:38 +0200 bulwahn correcting NEWS
Tue, 13 Sep 2011 09:28:03 +0200 bulwahn correcting theory name and dependencies
Tue, 13 Sep 2011 09:25:19 +0200 bulwahn renamed AList_Impl to AList
Tue, 13 Sep 2011 07:13:49 +0200 nipkow fastsimp -> fastforce in doc
Mon, 12 Sep 2011 14:49:34 -0700 huffman fix typo
Mon, 12 Sep 2011 14:39:10 -0700 huffman shorten proof of frontier_straddle
Mon, 12 Sep 2011 13:19:10 -0700 huffman NEWS and CONTRIBUTORS
Mon, 12 Sep 2011 11:54:20 -0700 huffman remove redundant lemma Lim_sequentially in favor of lemma LIMSEQ_def
Mon, 12 Sep 2011 11:39:29 -0700 huffman simplify proofs using LIMSEQ lemmas
Mon, 12 Sep 2011 10:43:36 -0700 huffman remove trivial lemma Lim_at_iff_LIM
Mon, 12 Sep 2011 10:28:45 -0700 huffman fix typos
Mon, 12 Sep 2011 09:37:49 -0700 huffman NEWS for euclidean_space class
Mon, 12 Sep 2011 09:21:01 -0700 huffman move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
Mon, 12 Sep 2011 09:57:33 -0400 hoelzl adding NEWS and CONTRIBUTORS
Mon, 12 Sep 2011 13:35:35 +0200 bulwahn merged
Mon, 12 Sep 2011 12:33:37 +0200 bulwahn correcting imports after splitting and renaming AssocList
Mon, 12 Sep 2011 10:59:38 +0200 bulwahn tuned
Mon, 12 Sep 2011 10:57:58 +0200 bulwahn moving connection of association lists to Mappings into a separate theory
Mon, 12 Sep 2011 10:27:36 +0200 bulwahn adding NEWS and CONTRIBUTORS
Mon, 12 Sep 2011 09:45:53 +0200 bulwahn tuned some symbol that probably went there by some strange encoding issue
Mon, 12 Sep 2011 11:05:32 +0200 blanchet added my contributions to NEWS and CONTRIBUTORS
Mon, 12 Sep 2011 10:49:37 +0200 blanchet fixed type intersection (again)
Mon, 12 Sep 2011 10:49:37 +0200 blanchet consistent option naming
Mon, 12 Sep 2011 09:07:23 +0200 nipkow NEWS fastsimp -> fastforce
Mon, 12 Sep 2011 07:55:43 +0200 nipkow new fastforce replacing fastsimp - less confusing name
Sun, 11 Sep 2011 22:56:05 +0200 wenzelm merged
Sun, 11 Sep 2011 13:49:42 -0700 huffman NEWS for Library/Product_Lattice.thy
Sun, 11 Sep 2011 22:55:26 +0200 wenzelm misc tuning and clarification;
Sun, 11 Sep 2011 21:35:35 +0200 wenzelm merged
Sun, 11 Sep 2011 10:30:50 -0700 huffman merged
Sun, 11 Sep 2011 09:40:18 -0700 huffman tuned proofs
Sun, 11 Sep 2011 07:21:45 -0700 huffman Library/Saturated.thy: 'Sat' abbreviates 'of_nat'
Sun, 11 Sep 2011 21:34:23 +0200 wenzelm more CONTRIBUTORS;
Sun, 11 Sep 2011 20:19:20 +0200 wenzelm persistent ISABELLE_INTERFACE_CHOICE;
Sun, 11 Sep 2011 19:52:09 +0200 wenzelm explicit choice of interface;
Sun, 11 Sep 2011 17:30:01 +0200 wenzelm more orthogonal signature;
Sun, 11 Sep 2011 15:20:09 +0200 wenzelm updates for release;
Sun, 11 Sep 2011 14:58:52 +0200 wenzelm misc tuning and clarification (NB: settings are already local for named snapshots/releases);
Sun, 11 Sep 2011 14:42:15 +0200 wenzelm some updates of PLATFORMS;
Sun, 11 Sep 2011 13:27:22 +0200 wenzelm more README;
Sat, 10 Sep 2011 23:28:58 +0200 wenzelm merged
Sat, 10 Sep 2011 22:43:17 +0200 krauss mem_prs and mem_rsp in accordance with sets-as-predicates representation (backported from AFP/Coinductive)
Sat, 10 Sep 2011 23:27:32 +0200 wenzelm misc tuning;
Sat, 10 Sep 2011 22:11:55 +0200 wenzelm misc tuning and clarification;
Sat, 10 Sep 2011 21:47:55 +0200 wenzelm speed up slow proof;
Sat, 10 Sep 2011 20:41:27 +0200 wenzelm merged
Sat, 10 Sep 2011 19:44:41 +0200 haftmann more modularization
Sat, 10 Sep 2011 20:39:13 +0200 wenzelm stronger colors (as background);
Sat, 10 Sep 2011 20:22:22 +0200 wenzelm some color scheme for theory status;
Sat, 10 Sep 2011 16:30:08 +0200 wenzelm some keyboard shortcuts for important actions;
Sat, 10 Sep 2011 14:48:06 +0200 wenzelm explicit jEdit actions -- to enable key mappings, for example;
Sat, 10 Sep 2011 14:28:07 +0200 wenzelm more symbolic file positions via smart replacement of ISABELLE_HOME -- allows Isabelle distribution to be moved later on;
Sat, 10 Sep 2011 13:43:09 +0200 wenzelm tuned usage;
Sat, 10 Sep 2011 13:41:03 +0200 wenzelm simplified default Isabelle application wrapper (NB: build process is already part of isabelle jedit tool);
Sat, 10 Sep 2011 10:29:24 +0200 haftmann renamed theory Complete_Lattice to Complete_Lattices, in accordance with Lattices, Orderings etc.
Sat, 10 Sep 2011 00:44:25 +0200 blanchet fixed definition of type intersection (soundness bug)
Sat, 10 Sep 2011 00:44:25 +0200 blanchet continue with minimization in debug mode in spite of unsoundness
Fri, 09 Sep 2011 09:31:04 -0700 huffman generalize lemma of_nat_number_of_eq to class number_semiring
Fri, 09 Sep 2011 15:14:59 +0200 bulwahn merged
Fri, 09 Sep 2011 14:43:50 +0200 bulwahn stating more explicitly our expectation that these two terms have the same term structure
Fri, 09 Sep 2011 12:33:09 +0200 bulwahn revisiting type annotations for Haskell: necessary type annotations are not inferred on the provided theorems but using the arguments and right hand sides, as these might differ in the case of constants with abstract code types
Fri, 09 Sep 2011 14:30:57 +0200 blanchet made SML/NJ happy
Thu, 08 Sep 2011 12:23:11 +0200 noschinl call ghc with -XEmptyDataDecls
Fri, 09 Sep 2011 06:47:14 +0200 nipkow merged
Fri, 09 Sep 2011 06:45:39 +0200 nipkow tuned headers
Thu, 08 Sep 2011 19:35:23 -0700 huffman Library/Saturated.thy: number_semiring class instance
Thu, 08 Sep 2011 18:47:23 -0700 huffman remove lemmas nat_add_min_{left,right} in favor of generic lemmas min_add_distrib_{left,right}
Thu, 08 Sep 2011 18:13:48 -0700 huffman merged
Thu, 08 Sep 2011 10:07:53 -0700 huffman remove unnecessary intermediate lemmas
Fri, 09 Sep 2011 00:22:18 +0200 krauss added syntactic classes for "inf" and "sup"
Thu, 08 Sep 2011 08:41:28 -0700 huffman prove existence, uniqueness, and other properties of complex arg function
Thu, 08 Sep 2011 07:27:57 -0700 huffman tuned
Thu, 08 Sep 2011 07:16:47 -0700 huffman remove obsolete intermediate lemma complex_inverse_complex_split
Thu, 08 Sep 2011 07:06:59 -0700 huffman tuned
Thu, 08 Sep 2011 11:31:53 +0200 haftmann merged
Thu, 08 Sep 2011 11:31:23 +0200 haftmann tuned
Thu, 08 Sep 2011 00:35:22 +0200 haftmann merged
Wed, 07 Sep 2011 08:13:38 +0200 haftmann merged
Tue, 06 Sep 2011 22:37:32 +0200 haftmann merged
Tue, 06 Sep 2011 22:04:14 +0200 haftmann merged
Tue, 06 Sep 2011 07:23:45 +0200 haftmann merged
Mon, 05 Sep 2011 22:02:32 +0200 haftmann tuned
Mon, 05 Sep 2011 19:18:38 +0200 haftmann merged
Mon, 05 Sep 2011 07:49:31 +0200 haftmann tuned
Sun, 04 Sep 2011 09:28:15 +0200 haftmann tuned
Thu, 08 Sep 2011 09:25:55 +0200 blanchet fixed computation of "in_conj" for polymorphic encodings
Wed, 07 Sep 2011 22:44:26 -0700 huffman add some new lemmas about cis and rcis;
Wed, 07 Sep 2011 20:44:39 -0700 huffman Complex.thy: move theorems into appropriate subsections
Wed, 07 Sep 2011 19:24:28 -0700 huffman merged
Wed, 07 Sep 2011 17:41:29 -0700 huffman remove redundant lemma complex_of_real_minus_one
Wed, 07 Sep 2011 18:47:55 -0700 huffman simplify proof of lemma DeMoivre, removing unnecessary intermediate lemma
Wed, 07 Sep 2011 10:04:07 -0700 huffman removed unused lemma sin_cos_squared_add2_mult
Wed, 07 Sep 2011 09:45:39 -0700 huffman remove duplicate lemma real_of_int_real_of_nat in favor of real_of_int_of_nat_eq
Wed, 07 Sep 2011 09:02:58 -0700 huffman avoid using legacy theorem names
Thu, 08 Sep 2011 00:23:23 +0200 wenzelm merged
Wed, 07 Sep 2011 23:55:40 +0200 haftmann theory of saturated naturals contributed by Peter Gammie
Wed, 07 Sep 2011 23:38:52 +0200 haftmann theory of saturated naturals contributed by Peter Gammie
Wed, 07 Sep 2011 23:07:16 +0200 haftmann lemmas about +, *, min, max on nat
Wed, 07 Sep 2011 21:31:21 +0200 blanchet update Sledgehammer docs
Wed, 07 Sep 2011 21:31:21 +0200 blanchet added new tagged encodings to Metis tests
Wed, 07 Sep 2011 21:31:21 +0200 blanchet also implemented ghost version of the tagged encodings
Wed, 07 Sep 2011 21:31:21 +0200 blanchet added new guards encoding to test
Wed, 07 Sep 2011 21:31:21 +0200 blanchet smarter explicit apply business
Wed, 07 Sep 2011 21:31:21 +0200 blanchet started work on ghost type arg encoding
Wed, 07 Sep 2011 21:31:21 +0200 blanchet stricted type encoding parsing
Thu, 08 Sep 2011 00:20:09 +0200 wenzelm more substructural sharing to gain significant compression;
Wed, 07 Sep 2011 23:08:04 +0200 wenzelm XML.cache for partial sharing (strings only);
Wed, 07 Sep 2011 22:00:41 +0200 wenzelm platform-specific look and feel;
Wed, 07 Sep 2011 21:41:36 +0200 wenzelm more README;
Wed, 07 Sep 2011 21:38:48 +0200 wenzelm clarified terminology;
Wed, 07 Sep 2011 21:31:50 +0200 wenzelm no print_state for final proof commands, which return to theory state;
Wed, 07 Sep 2011 21:10:47 +0200 wenzelm NEWS on IsabelleText font;
Wed, 07 Sep 2011 21:05:53 +0200 wenzelm explicit join_syntax ensures command transaction integrity of 'theory';
Wed, 07 Sep 2011 20:49:45 +0200 wenzelm some updates for release;
Wed, 07 Sep 2011 20:29:54 +0200 wenzelm some tuning for release;
Wed, 07 Sep 2011 18:01:01 +0200 wenzelm updated file locations;
Wed, 07 Sep 2011 17:42:57 +0200 wenzelm merged
Wed, 07 Sep 2011 14:58:40 +0200 bulwahn merged
Wed, 07 Sep 2011 13:51:39 +0200 bulwahn removing previously used function locally_monomorphic in the code generator
Wed, 07 Sep 2011 13:51:38 +0200 bulwahn setting const_sorts to false in the type inference of the code generator
Wed, 07 Sep 2011 13:51:37 +0200 bulwahn adapting Imperative HOL serializer to changes of the iterm datatype in the code generator
Wed, 07 Sep 2011 13:51:36 +0200 bulwahn removing previous crude approximation to add type annotations to disambiguate types
Wed, 07 Sep 2011 13:51:35 +0200 bulwahn adding minimalistic implementation for printing the type annotations
Wed, 07 Sep 2011 13:51:34 +0200 bulwahn adding call to disambiguation annotations
Wed, 07 Sep 2011 13:51:34 +0200 bulwahn adding type inference for disambiguation annotations in code equation
Wed, 07 Sep 2011 13:51:32 +0200 bulwahn adding the body type as well to the code generation for constants as it is required for type annotations of constants
Wed, 07 Sep 2011 13:51:30 +0200 bulwahn changing const type to pass along if typing annotations are necessary for disambigous terms
Wed, 07 Sep 2011 13:50:17 +0200 blanchet fixed THF type constructor syntax
Wed, 07 Sep 2011 13:50:17 +0200 blanchet tweaking polymorphic TFF and THF output
Wed, 07 Sep 2011 13:50:17 +0200 blanchet parse new experimental '@' encodings
Wed, 07 Sep 2011 13:50:17 +0200 blanchet tuning
Wed, 07 Sep 2011 13:50:17 +0200 blanchet tuning
Wed, 07 Sep 2011 13:50:16 +0200 blanchet tuning
Wed, 07 Sep 2011 17:03:34 +0200 wenzelm clarified import;
Wed, 07 Sep 2011 16:53:49 +0200 wenzelm tuned/simplified proofs;
Wed, 07 Sep 2011 16:37:50 +0200 wenzelm tuned proofs;
Wed, 07 Sep 2011 11:36:39 +0200 wenzelm deactivate unfinished charset provider for now, to avoid user confusion;
Wed, 07 Sep 2011 11:26:27 +0200 wenzelm more NEWS;
Wed, 07 Sep 2011 11:17:19 +0200 wenzelm added "check" button: adhoc change to full buffer perspective;
Wed, 07 Sep 2011 11:00:39 +0200 wenzelm added "cancel" button based on cancel_execution, not interrupt (cf. 156be0e43336);
Wed, 07 Sep 2011 09:10:41 +0200 blanchet separate mangling, which can (and should) be done before the formulas are first-orderized, and type arg filtering, which must be done after once the min arities have been computed
Wed, 07 Sep 2011 09:10:41 +0200 blanchet perform mangling before computing symbol arity, to avoid needless "hAPP"s and "hBOOL"s
Wed, 07 Sep 2011 09:10:41 +0200 blanchet tuning
Wed, 07 Sep 2011 09:10:41 +0200 blanchet make mangling sound w.r.t. type arguments
Wed, 07 Sep 2011 09:10:41 +0200 blanchet make "filter_type_args" more robust if the actual arity is higher than the declared one
Wed, 07 Sep 2011 09:10:41 +0200 blanchet updated Sledgehammer documentation
Wed, 07 Sep 2011 09:10:41 +0200 blanchet rationalize uniform encodings
Tue, 06 Sep 2011 22:41:35 -0700 huffman merged
Tue, 06 Sep 2011 19:03:41 -0700 huffman avoid using legacy theorem names
Tue, 06 Sep 2011 16:30:39 -0700 huffman merged
Tue, 06 Sep 2011 14:53:51 -0700 huffman remove redundant lemmas i_mult_eq and i_mult_eq2 in favor of i_squared
Wed, 07 Sep 2011 07:59:45 +0900 Cezary Kaliszyk HOL/Import: Update HOL4 generated files to current Isabelle.
Wed, 07 Sep 2011 00:08:09 +0200 wenzelm tuned proofs;
Tue, 06 Sep 2011 13:16:46 -0700 huffman remove some unnecessary simp rules from simpset
Tue, 06 Sep 2011 21:56:11 +0200 wenzelm some Isabelle/jEdit NEWS;
Tue, 06 Sep 2011 21:40:58 +0200 wenzelm more README;
Tue, 06 Sep 2011 21:11:12 +0200 wenzelm merged
Tue, 06 Sep 2011 10:30:33 -0700 huffman merged
Tue, 06 Sep 2011 10:30:00 -0700 huffman simplify proof of tan_half, removing unused assumptions
Tue, 06 Sep 2011 09:56:09 -0700 huffman convert some proofs to Isar-style
Tue, 06 Sep 2011 18:13:36 +0200 blanchet added dummy polymorphic THF system
Tue, 06 Sep 2011 18:07:44 +0200 boehmes added some examples for pattern and weight annotations
Tue, 06 Sep 2011 17:52:00 +0200 bulwahn merged
Tue, 06 Sep 2011 16:40:22 +0200 bulwahn avoid "Code" as structure name (cf. 3bc39cfe27fe)
Tue, 06 Sep 2011 08:00:28 -0700 huffman remove duplicate copy of lemma sqrt_add_le_add_sqrt
Tue, 06 Sep 2011 07:48:59 -0700 huffman remove redundant lemma real_sum_squared_expand in favor of power2_sum
Tue, 06 Sep 2011 07:45:18 -0700 huffman remove redundant lemma LIMSEQ_Complex in favor of tendsto_Complex
Tue, 06 Sep 2011 07:41:15 -0700 huffman merged
Mon, 05 Sep 2011 22:30:25 -0700 huffman add lemmas about arctan;
Mon, 05 Sep 2011 18:06:02 -0700 huffman convert lemma cos_total to Isar-style proof
Tue, 06 Sep 2011 14:25:16 +0200 nipkow added new lemmas
Tue, 06 Sep 2011 11:31:01 +0200 blanchet updated Sledgehammer's docs
Tue, 06 Sep 2011 11:31:01 +0200 blanchet cleanup "simple" type encodings
Tue, 06 Sep 2011 17:50:04 +0900 Cezary Kaliszyk merge
Tue, 06 Sep 2011 16:45:31 +0900 Cezary Kaliszyk HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
Tue, 06 Sep 2011 09:11:08 +0200 blanchet tuning
Tue, 06 Sep 2011 09:11:08 +0200 blanchet drop more type arguments soundly, when they can be deduced from the arg types
Tue, 06 Sep 2011 20:55:18 +0200 wenzelm bulk reports for improved message throughput;
Tue, 06 Sep 2011 20:37:07 +0200 wenzelm bulk reports for improved message throughput;
Tue, 06 Sep 2011 19:48:57 +0200 wenzelm tuned signature;
Tue, 06 Sep 2011 11:25:27 +0200 wenzelm more specific message channels to avoid potential bottle-neck of raw_messages;
Tue, 06 Sep 2011 11:18:19 +0200 wenzelm buffer prover messages to prevent overloading of session_actor input channel -- which is critical due to synchronous messages wrt. GUI thread;
Tue, 06 Sep 2011 10:27:04 +0200 wenzelm more abstract receiver interface;
Tue, 06 Sep 2011 10:16:12 +0200 wenzelm flush after Output.raw_message (and init message) for reduced latency of important protocol events;
Mon, 05 Sep 2011 17:45:37 -0700 huffman convert lemma cos_is_zero to Isar-style
Mon, 05 Sep 2011 17:05:00 -0700 huffman merged
Mon, 05 Sep 2011 17:00:56 -0700 huffman convert lemma sin_gt_zero to Isar style;
Mon, 05 Sep 2011 16:26:57 -0700 huffman modify lemma sums_group, and shorten proofs that use it
Mon, 05 Sep 2011 16:07:40 -0700 huffman generalize some lemmas
Mon, 05 Sep 2011 12:19:04 -0700 huffman add lemmas cos_arctan and sin_arctan
Mon, 05 Sep 2011 08:38:50 -0700 huffman tuned indentation
Mon, 05 Sep 2011 23:51:16 +0200 wenzelm more visible outdated_color;
Mon, 05 Sep 2011 23:26:41 +0200 wenzelm commands_change_delay within main actor -- prevents overloading of commands_change_buffer input channel;
Mon, 05 Sep 2011 20:30:37 +0200 wenzelm tuned imports;
Mon, 05 Sep 2011 14:42:31 +0200 blanchet fixed handling of "sledgehammer_params", so that "sledgehammer_params [e]" is really the same as "sledgehammer_params [provers = e]"
Mon, 05 Sep 2011 14:17:44 +0200 boehmes tuned
Mon, 05 Sep 2011 11:34:54 +0200 boehmes tuned
Mon, 05 Sep 2011 11:28:10 +0200 boehmes filter out all schematic theorems if the problem contains no ground constants
Sun, 04 Sep 2011 21:04:02 -0700 huffman merged
Sun, 04 Sep 2011 21:03:54 -0700 huffman tuned comments
Sun, 04 Sep 2011 11:16:47 -0700 huffman simplify proof of Bseq_mono_convergent
Sun, 04 Sep 2011 20:37:20 +0200 wenzelm merged
Sun, 04 Sep 2011 10:29:38 -0700 huffman replace lemma expi_imaginary with reoriented lemma cis_conv_exp
Sun, 04 Sep 2011 10:05:52 -0700 huffman remove redundant lemmas expi_add and expi_zero
Sun, 04 Sep 2011 09:49:45 -0700 huffman remove redundant lemmas about LIMSEQ
Sun, 04 Sep 2011 07:15:13 -0700 huffman introduce abbreviation 'int' earlier in Int.thy
Sun, 04 Sep 2011 06:56:10 -0700 huffman remove unused assumptions from natceiling lemmas
Sun, 04 Sep 2011 06:27:59 -0700 huffman move lemmas nat_le_iff and nat_mono into Int.thy
Sun, 04 Sep 2011 19:36:19 +0200 wenzelm eliminated markup for plain identifiers (frequent but insignificant);
Sun, 04 Sep 2011 19:12:06 +0200 wenzelm simplified signatures;
Sun, 04 Sep 2011 19:06:45 +0200 wenzelm synchronous XML.Cache without actor -- potentially more efficient on machines with few cores;
Sun, 04 Sep 2011 17:50:19 +0200 wenzelm tuned document;
Sun, 04 Sep 2011 17:35:34 +0200 wenzelm improved handling of extended styles and hard tabs when prover is inactive;
Sun, 04 Sep 2011 17:21:11 +0200 wenzelm mark hard tabs as single chunks, as required by jEdit;
Sun, 04 Sep 2011 16:37:22 +0200 wenzelm updated READMEs;
Sun, 04 Sep 2011 15:49:59 +0200 wenzelm property "tooltip-dismiss-delay" is edited in ms, not seconds;
Sun, 04 Sep 2011 15:21:50 +0200 wenzelm moved XML/YXML to src/Pure/PIDE;
Sun, 04 Sep 2011 14:29:15 +0200 wenzelm pass raw messages through xml_cache actor, which is important to retain ordering of results (e.g. read_command reports before assign, cf. 383c9d758a56);
Sun, 04 Sep 2011 08:43:06 +0200 haftmann pseudo-definition for perms on sets; tuned
Sat, 03 Sep 2011 16:00:09 -0700 huffman remove duplicate lemma nat_zero in favor of nat_0
Sat, 03 Sep 2011 15:37:41 -0700 huffman merged
Sat, 03 Sep 2011 15:09:51 -0700 huffman merged
Sat, 03 Sep 2011 14:52:40 -0700 huffman modify nominal packages to better respect set/pred distinction
Sat, 03 Sep 2011 14:33:45 -0700 huffman merged
Sat, 03 Sep 2011 11:10:38 -0700 huffman remove unused assumption from lemma posreal_complete
Sat, 03 Sep 2011 23:59:36 +0200 haftmann tuned specifications
Sat, 03 Sep 2011 23:38:06 +0200 haftmann merged
Sat, 03 Sep 2011 17:56:33 +0200 haftmann tuned proof
Sat, 03 Sep 2011 17:32:45 +0200 haftmann merged
Sat, 03 Sep 2011 17:32:35 +0200 haftmann assert Pure equations for theorem references; avoid dynamic reference to fact
Sat, 03 Sep 2011 17:32:34 +0200 haftmann assert Pure equations for theorem references; tuned
Sat, 03 Sep 2011 17:32:34 +0200 haftmann tuned specifications and proofs
Sat, 03 Sep 2011 22:11:49 +0200 wenzelm merged
Sat, 03 Sep 2011 09:26:11 -0700 huffman remove duplicate lemma finite_choice in favor of finite_set_choice
Sat, 03 Sep 2011 09:12:19 -0700 huffman simplify proof
Sat, 03 Sep 2011 08:01:49 -0700 huffman shorten some proofs
Fri, 02 Sep 2011 20:58:31 -0700 huffman remove redundant simp rules ceiling_floor and floor_ceiling
Sat, 03 Sep 2011 22:05:25 +0200 wenzelm misc tuning and simplification of proofs;
Sat, 03 Sep 2011 21:15:35 +0200 wenzelm Document.removed_versions on Scala side;
Sat, 03 Sep 2011 19:47:31 +0200 wenzelm discontinued predefined empty command (obsolete!?);
Sat, 03 Sep 2011 19:39:16 +0200 wenzelm discontinued global execs: store exec value directly within entries;
Sat, 03 Sep 2011 18:08:09 +0200 wenzelm Document.remove_versions on ML side;
Sat, 03 Sep 2011 12:31:27 +0200 wenzelm some support to prune_history;
Fri, 02 Sep 2011 16:58:00 -0700 huffman merged
Fri, 02 Sep 2011 16:57:51 -0700 huffman speed up extremely slow metis proof of Sup_real_iff
Fri, 02 Sep 2011 16:48:30 -0700 huffman remove redundant lemma reals_complete2 in favor of complete_real
Fri, 02 Sep 2011 15:19:59 -0700 huffman simplify proof of Rats_dense_in_real;
Fri, 02 Sep 2011 14:27:55 -0700 huffman remove unused, unnecessary lemmas
Fri, 02 Sep 2011 13:57:12 -0700 huffman remove more duplicate lemmas
Fri, 02 Sep 2011 23:04:12 +0200 wenzelm merged
Fri, 02 Sep 2011 19:29:48 +0200 haftmann merged
Fri, 02 Sep 2011 19:29:36 +0200 haftmann avoid "Code" as structure name
Fri, 02 Sep 2011 22:48:56 +0200 wenzelm more robust chunk painting wrt. hard tabs, when chunk.str == null;
Fri, 02 Sep 2011 21:48:27 +0200 wenzelm raw message function "assign_execs" avoids full overhead of decoding and caching message body;
Fri, 02 Sep 2011 21:06:05 +0200 wenzelm less agressive parsing of commands (priority ~1);
Fri, 02 Sep 2011 20:35:32 +0200 wenzelm tuned;
Fri, 02 Sep 2011 20:29:39 +0200 wenzelm more direct Token.range_pos and Outer_Syntax.read_command, bypassing Thy_Syntax.span;
Fri, 02 Sep 2011 19:25:44 +0200 nipkow merged
Fri, 02 Sep 2011 19:25:18 +0200 nipkow Added Abstract Interpretation theories
Fri, 02 Sep 2011 18:17:45 +0200 wenzelm tuned proofs;
Fri, 02 Sep 2011 17:58:32 +0200 wenzelm proper config option linarith_trace;
Fri, 02 Sep 2011 17:57:37 +0200 wenzelm discontinued slightly odd "Defining record ..." message and corresponding quiet_mode;
Fri, 02 Sep 2011 16:20:09 +0200 wenzelm merged
Fri, 02 Sep 2011 14:43:20 +0200 blanchet renamed "Metis_Tactics" to "Metis_Tactic", now that there is only one Metis tactic ("metisFT" is legacy)
Fri, 02 Sep 2011 14:43:20 +0200 blanchet use new syntax for Pi binder in TFF1 output
Fri, 02 Sep 2011 14:43:20 +0200 blanchet fewer TPTP important messages
Thu, 01 Sep 2011 10:41:19 -0700 huffman simplify some proofs about uniform continuity, and add some new ones;
Thu, 01 Sep 2011 09:02:14 -0700 huffman modernize lemmas about 'continuous' and 'continuous_on';
Thu, 01 Sep 2011 07:31:33 -0700 huffman add lemma tendsto_infnorm
Fri, 02 Sep 2011 15:21:40 +0200 wenzelm more precise iterate_entries_after if start refers to last entry;
Fri, 02 Sep 2011 11:52:13 +0200 wenzelm clarified define_command: store name as structural information;
Thu, 01 Sep 2011 23:08:42 +0200 wenzelm amended last_common, if that happens to the very last entry (important to load HOL/Auth, for example);
Thu, 01 Sep 2011 22:29:57 +0200 wenzelm more redable Document.Node.toString;
Thu, 01 Sep 2011 16:58:41 +0200 wenzelm sort wrt. theory name;
Thu, 01 Sep 2011 16:58:03 +0200 wenzelm modernized theory name;
Thu, 01 Sep 2011 16:46:07 +0200 wenzelm repaired benchmarks;
Thu, 01 Sep 2011 14:35:51 +0200 wenzelm merged
Thu, 01 Sep 2011 14:21:09 +0200 blanchet tuning
Thu, 01 Sep 2011 13:18:27 +0200 blanchet always measure time for ATPs -- auto minimization relies on it
Thu, 01 Sep 2011 13:18:27 +0200 blanchet added two lemmas about "distinct" to help Sledgehammer
Thu, 01 Sep 2011 13:18:27 +0200 blanchet make "sound" sound and "unsound" more sound, based on evaluation
Thu, 01 Sep 2011 16:16:25 +0900 Cezary Kaliszyk HOL/Import: observe distinction between sets and predicates (where possible)
Wed, 31 Aug 2011 13:28:29 -0700 huffman simplify/generalize some proofs
Wed, 31 Aug 2011 10:42:31 -0700 huffman generalize lemma isCont_vec_nth
Wed, 31 Aug 2011 10:24:29 -0700 huffman convert proof to Isar-style
Wed, 31 Aug 2011 13:51:22 -0700 huffman remove redundant lemma card_enum
Wed, 31 Aug 2011 08:11:47 -0700 huffman move lemmas from Topology_Euclidean_Space to Euclidean_Space
Wed, 31 Aug 2011 07:51:55 -0700 huffman convert to Isar-style proof
Wed, 31 Aug 2011 13:22:50 +0200 blanchet make SML/NJ happy
Wed, 31 Aug 2011 11:52:03 +0200 blanchet more tuning
Wed, 31 Aug 2011 11:23:16 +0200 blanchet more tuning
Wed, 31 Aug 2011 11:14:53 +0200 blanchet tuning
Wed, 31 Aug 2011 11:12:27 +0200 blanchet avoid relying on dubious TFF1 feature
Wed, 31 Aug 2011 08:49:10 +0200 blanchet killed FIXME (the ATP exporter outputs TPTP FOF, which is first-order)
Wed, 31 Aug 2011 08:49:10 +0200 blanchet fixed explicit declaration of TFF1 types
Tue, 30 Aug 2011 20:10:48 +0200 bulwahn adding list_size_append (thanks to Rene Thiemann)
Tue, 30 Aug 2011 20:10:47 +0200 bulwahn strengthening list_size_pointwise (thanks to Rene Thiemann)
Thu, 01 Sep 2011 14:10:52 +0200 wenzelm more flexible sorting;
Thu, 01 Sep 2011 13:39:40 +0200 wenzelm tuned signature;
Thu, 01 Sep 2011 13:34:45 +0200 wenzelm more abstract Document.Node.Name;
Thu, 01 Sep 2011 11:33:44 +0200 wenzelm more careful treatment of interrupts, to retain them within forked/joined boundary of command transactions;
Wed, 31 Aug 2011 22:10:07 +0200 wenzelm crude display of node status;
Wed, 31 Aug 2011 20:47:33 +0200 wenzelm explicit cancel_execution before queueing new edits -- potential performance improvement for machines with few cores;
Wed, 31 Aug 2011 20:32:24 +0200 wenzelm explicit running_color;
Wed, 31 Aug 2011 19:52:13 +0200 wenzelm tuned join_commands: avoid traversing cumulative table;
Wed, 31 Aug 2011 17:36:10 +0200 wenzelm some support for theory status overview;
Wed, 31 Aug 2011 17:22:49 +0200 wenzelm tuned Commands_Changed: cover nodes as well;
Wed, 31 Aug 2011 15:41:22 +0200 wenzelm maintain name of *the* enclosing node as part of command -- avoid full document traversal;
Wed, 31 Aug 2011 14:39:41 +0200 wenzelm improved auto loading: selectable file list;
Tue, 30 Aug 2011 18:12:48 +0200 wenzelm tuned document;
Tue, 30 Aug 2011 17:53:03 +0200 wenzelm tuned import;
Tue, 30 Aug 2011 17:51:30 +0200 wenzelm tuned document;
Tue, 30 Aug 2011 17:50:41 +0200 wenzelm tuned color for Mac OS X (very light color profile?);
Tue, 30 Aug 2011 17:36:12 +0200 wenzelm tuned document;
Tue, 30 Aug 2011 17:02:06 +0200 wenzelm merged;
Tue, 30 Aug 2011 16:25:10 +0200 blanchet fixed just introduced silly bug
Tue, 30 Aug 2011 16:23:25 +0200 blanchet "simple" was renamed "mono_simple" and there's now "poly_simple" as well -- but they are not needed here since for Metis they amount to the same as guards
Tue, 30 Aug 2011 16:11:42 +0200 blanchet tuning
Tue, 30 Aug 2011 16:07:46 +0200 blanchet cleaner "pff" dummy TFF0 prover
Tue, 30 Aug 2011 16:07:46 +0200 blanchet generate properly typed TFF1 (PFF) problems in the presence of type class predicates
Tue, 30 Aug 2011 16:07:45 +0200 blanchet added type abstractions (for declaring polymorphic constants) to TFF syntax
Tue, 30 Aug 2011 16:07:45 +0200 blanchet implement more of the polymorphic simply typed format TFF(1)
Tue, 30 Aug 2011 16:07:45 +0200 blanchet flip logic of boolean option so it's off by default
Tue, 30 Aug 2011 16:07:45 +0200 blanchet extended simple types with polymorphism -- the implementation still needs some work though
Tue, 30 Aug 2011 16:07:45 +0200 blanchet added dummy PFF prover, for debugging purposes
Tue, 30 Aug 2011 16:07:34 +0200 blanchet first step towards polymorphic TFF + changed defaults for Vampire
Tue, 30 Aug 2011 16:04:23 +0200 blanchet tuning
Tue, 30 Aug 2011 14:29:39 +0200 nik removed explicit reliance on Hilbert_Choice.Eps
Tue, 30 Aug 2011 14:12:55 +0200 nik improved handling of induction rules in Sledgehammer
Tue, 30 Aug 2011 14:12:55 +0200 nik added generation of induction rules
Mon, 29 Aug 2011 13:50:47 -0700 huffman simplify some proofs
Tue, 30 Aug 2011 16:33:24 +0200 wenzelm restrict perspective to actual buffer_range, to avoid spurious edits due to faulty last_exec_offset (NB: jEdit screenlines may be silently extended by trailing newline);
Tue, 30 Aug 2011 16:04:26 +0200 wenzelm tuned signature;
Tue, 30 Aug 2011 15:49:27 +0200 wenzelm dynamic exec state lookup for implicit position information (e.g. 'definition' without binding);
Tue, 30 Aug 2011 15:43:27 +0200 wenzelm some support for hyperlinks between different buffers;
Tue, 30 Aug 2011 12:24:55 +0200 wenzelm tuned colors -- more distance between outdated_color and quoted_color;
Tue, 30 Aug 2011 12:01:07 +0200 wenzelm do not normalized extra file dependencies for now -- still loaded by prover process;
Tue, 30 Aug 2011 11:43:47 +0200 wenzelm separate module for jEdit primitives for loading theory files;
Mon, 29 Aug 2011 22:10:08 +0200 wenzelm merged
Mon, 29 Aug 2011 08:31:09 -0700 huffman Product_Vector.thy: clean up some proofs
Mon, 29 Aug 2011 21:55:49 +0200 wenzelm actual auto loading of required files;
Mon, 29 Aug 2011 16:38:56 +0200 wenzelm some dialog for auto loading of required files (still inactive);
Mon, 29 Aug 2011 16:28:51 +0200 wenzelm invoke in Swing thread to make double sure;
Sun, 28 Aug 2011 20:56:49 -0700 huffman move class perfect_space into RealVector.thy;
Sun, 28 Aug 2011 16:28:07 -0700 huffman generalize LIM_zero lemmas to arbitrary filters
Sun, 28 Aug 2011 09:22:42 -0700 huffman merged
Sun, 28 Aug 2011 09:20:12 -0700 huffman discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
Sun, 28 Aug 2011 14:16:14 +0200 haftmann tuned
Sun, 28 Aug 2011 13:13:27 +0200 blanchet split timeout among ATPs in and add Metis to the mix as backup
Sun, 28 Aug 2011 13:05:34 +0200 wenzelm more portable cp options, e.g. for non-GNU version on Mac OS X Leopard;
Sun, 28 Aug 2011 12:53:31 +0200 wenzelm tuned positions of ambiguity messages -- less intrusive in IDE view;
Sun, 28 Aug 2011 08:43:25 +0200 haftmann tuned
Sun, 28 Aug 2011 08:13:58 +0200 haftmann merged
Sun, 28 Aug 2011 08:13:30 +0200 haftmann avoid loading List_Cset and Dlist_Cet at the same time
Sun, 28 Aug 2011 08:12:54 +0200 haftmann corrected slip
Sat, 27 Aug 2011 19:52:58 +0200 haftmann Cset, Dlist_Cset, List_Cset: restructured
Sat, 27 Aug 2011 09:44:45 +0200 haftmann Cset, Dlist_Cset, List_Cset: restructured
Sat, 27 Aug 2011 09:02:25 +0200 haftmann adapted to changes in Cset.thy
Fri, 26 Aug 2011 23:02:00 +0200 haftmann adapted to changes in Cset.thy
Fri, 26 Aug 2011 21:11:23 +0200 haftmann separating predicates and sets syntactically
Fri, 26 Aug 2011 18:24:22 +0200 haftmann merged
Fri, 26 Aug 2011 18:23:33 +0200 haftmann avoid intermixing set and predicates; dropped lemmas mem_rsp and mem_prs (now in Quotient_Set.thy)
Thu, 25 Aug 2011 23:32:12 +0200 haftmann updated generated files
Thu, 25 Aug 2011 23:20:44 +0200 haftmann merged
Thu, 25 Aug 2011 23:20:34 +0200 haftmann updated generated files
Sat, 27 Aug 2011 17:26:14 +0200 wenzelm explicit markup for legacy warnings;
Sat, 27 Aug 2011 16:22:59 +0200 wenzelm updated generated files;
Sat, 27 Aug 2011 16:11:24 +0200 wenzelm less aggressive warning icon;
Sat, 27 Aug 2011 16:01:24 +0200 wenzelm tuned colors;
Sat, 27 Aug 2011 15:53:18 +0200 wenzelm transparent foreground color for quoted entities;
Sat, 27 Aug 2011 13:26:06 +0200 wenzelm more precise treatment of nodes that are fully required for partially visible ones;
Sat, 27 Aug 2011 12:22:24 +0200 wenzelm de-assigned commands also count as changed;
Sat, 27 Aug 2011 11:22:21 +0200 blanchet beef up sledgehammer_tac in Mirabelle some more
Sat, 27 Aug 2011 11:22:11 +0200 blanchet merged
Fri, 26 Aug 2011 21:52:11 +0200 blanchet change default for generation of tag idempotence and tag argument equations
Fri, 26 Aug 2011 15:11:33 -0700 huffman merged
Fri, 26 Aug 2011 15:11:26 -0700 huffman NEWS entry for setsum_norm ~> norm_setsum
Fri, 26 Aug 2011 15:00:00 -0700 huffman make HOL-Probability respect set/pred distinction
Fri, 26 Aug 2011 23:14:36 +0200 wenzelm merged
Wed, 08 Sep 2010 16:10:49 -0700 huffman use rename_tac to make proof script more robust (with separate set type, 'clarify' yields different variable names)
Fri, 26 Aug 2011 10:38:29 -0700 huffman merged
Fri, 26 Aug 2011 08:56:29 -0700 huffman generalize and simplify proof of continuous_within_sequentially
Fri, 26 Aug 2011 08:12:38 -0700 huffman add lemma sequentially_imp_eventually_within;
Thu, 25 Aug 2011 19:41:38 -0700 huffman replace some continuous_on lemmas with more general versions
Thu, 25 Aug 2011 16:50:55 -0700 huffman remove legacy theorem Lim_inner
Thu, 25 Aug 2011 16:42:13 -0700 huffman arrange everything related to ordered_euclidean_space class together
Thu, 25 Aug 2011 16:06:50 -0700 huffman generalize and shorten proof of basis_orthogonal
Thu, 25 Aug 2011 15:35:54 -0700 huffman remove dot_lsum and dot_rsum in favor of inner_setsum_{left,right}
Thu, 25 Aug 2011 14:26:38 -0700 huffman merged
Thu, 25 Aug 2011 14:25:19 -0700 huffman generalize lemma finite_imp_compact_convex_hull and related lemmas
Thu, 25 Aug 2011 13:48:11 -0700 huffman generalize some lemmas
Thu, 25 Aug 2011 12:52:10 -0700 huffman generalize lemma convex_cone_hull
Thu, 25 Aug 2011 12:43:55 -0700 huffman rename subset_{interior,closure} to {interior,closure}_mono;
Thu, 25 Aug 2011 11:57:42 -0700 huffman simplify many proofs about subspace and span;
Thu, 25 Aug 2011 11:56:20 -0700 huffman remove duplicate simp declaration
Thu, 25 Aug 2011 09:17:02 -0700 huffman simplify definition of 'interior';
Wed, 24 Aug 2011 16:08:21 -0700 huffman add lemma closure_union;
Wed, 24 Aug 2011 15:32:40 -0700 huffman minimize imports
Wed, 24 Aug 2011 15:06:13 -0700 huffman move everything related to 'norm' method into new theory file Norm_Arith.thy
Wed, 24 Aug 2011 12:39:42 -0700 huffman remove unused lemmas dimensionI, dimension_eq
Wed, 24 Aug 2011 11:56:57 -0700 huffman move geometric progression lemmas from Linear_Algebra.thy to Integration.thy where they are used
Fri, 26 Aug 2011 22:53:04 +0900 Cezary Kaliszyk merge
Fri, 26 Aug 2011 09:31:56 +0900 Cezary Kaliszyk FSet: Explicit proof without mem_def
Fri, 26 Aug 2011 14:54:41 +0200 nipkow merged
Fri, 26 Aug 2011 11:22:47 +0200 nipkow added lemma
Fri, 26 Aug 2011 10:25:13 +0200 blanchet added a component in generated file names reflecting whether the minimizer is used -- needed for evaluation to keep these files separated from the main problem files
Fri, 26 Aug 2011 10:12:17 +0200 blanchet comment
Fri, 26 Aug 2011 01:18:48 +0200 blanchet disable TFF for Vampire 1.8 until they've fixed the soundness issues and it's back on SystemOnTPTP
Fri, 26 Aug 2011 01:14:49 +0200 blanchet improve completeness of polymorphic encodings
Fri, 26 Aug 2011 00:19:25 +0200 blanchet mangle tag bound declarations properly
Fri, 26 Aug 2011 00:05:45 +0200 blanchet fixed inverted logic and improve precision when handling monotonic types in polymorphic encodings
Thu, 25 Aug 2011 23:55:21 +0200 blanchet make sure that if slicing is disabled, a non-SOS slice is chosen
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);
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
Sat, 20 Aug 2011 09:59:28 -0700 huffman add lemma power2_eq_iff
Sat, 20 Aug 2011 07:09:44 -0700 huffman remove some over-specific rules from the simpset
Sat, 20 Aug 2011 06:35:43 -0700 huffman merged
Sat, 20 Aug 2011 06:34:51 -0700 huffman redefine constant 'trivial_limit' as an abbreviation
Sun, 21 Aug 2011 13:23:29 +0200 wenzelm purely functional task_queue.ML -- moved actual interrupt_unsynchronized to future.ML;
Sun, 21 Aug 2011 13:10:48 +0200 wenzelm refined Task_Queue.cancel: passive tasks are considered running due to pending abort operation;
Sat, 20 Aug 2011 23:36:18 +0200 wenzelm odd workaround for odd problem of load order in HOL/ex/ROOT.ML (!??);
Sat, 20 Aug 2011 23:35:30 +0200 wenzelm refined Graph implementation: more abstract/scalable Graph.Keys instead of plain lists -- order of adjacency is now standardized wrt. Key.ord;
Sat, 20 Aug 2011 22:46:19 +0200 wenzelm clarified get_imports -- should not rely on accidental order within graph;
Sat, 20 Aug 2011 22:28:53 +0200 wenzelm tuned Table.delete_safe: avoid potentially expensive attempt of delete;
Sat, 20 Aug 2011 20:24:12 +0200 wenzelm discontinued "Interrupt", which could disturb administrative tasks of the document model;
Sat, 20 Aug 2011 20:00:55 +0200 wenzelm more direct balanced version Ord_List.unions;
Sat, 20 Aug 2011 19:21:03 +0200 wenzelm reverted to join_bodies/join_proofs based on fold_body_thms to regain performance (escpecially of HOL-Proofs) -- see also aa9c1e9ef2ce and 4e2abb045eac;
Sat, 20 Aug 2011 18:11:17 +0200 wenzelm tuned future priorities (again);
Sat, 20 Aug 2011 16:06:27 +0200 wenzelm clarified fulfill_norm_proof: no join_thms yet;
Sat, 20 Aug 2011 15:52:29 +0200 wenzelm added Future.joins convenience;
Sat, 20 Aug 2011 09:42:34 +0200 haftmann merged
Sat, 20 Aug 2011 09:42:12 +0200 haftmann deactivated »unknown« nitpick example
Sat, 20 Aug 2011 09:30:23 +0200 haftmann merged
Sat, 20 Aug 2011 01:40:22 +0200 haftmann tuned proof
Sat, 20 Aug 2011 01:39:27 +0200 haftmann more uniform formatting of specifications
Sat, 20 Aug 2011 01:33:58 +0200 haftmann compatibility layer
Sat, 20 Aug 2011 01:21:22 +0200 haftmann merged
Fri, 19 Aug 2011 19:33:31 +0200 haftmann more concise definition for Inf, Sup on bool
Thu, 18 Aug 2011 13:37:41 +0200 noschinl do not call ghc with -fglasgow-exts
Fri, 19 Aug 2011 19:01:00 -0700 huffman remove some redundant simp rules about sqrt
Fri, 19 Aug 2011 18:42:41 -0700 huffman move sin_coeff and cos_coeff lemmas to Transcendental.thy; simplify some proofs
Fri, 19 Aug 2011 18:08:05 -0700 huffman remove unused lemma DERIV_sin_add
Fri, 19 Aug 2011 18:06:27 -0700 huffman remove redundant lemma lemma_DERIV_subst in favor of DERIV_cong
Fri, 19 Aug 2011 17:59:19 -0700 huffman remove redundant lemma exp_ln_eq in favor of ln_unique
Fri, 19 Aug 2011 16:55:43 -0700 huffman merged
Fri, 19 Aug 2011 15:54:43 -0700 huffman Lim.thy: legacy theorems
Fri, 19 Aug 2011 15:07:10 -0700 huffman SEQ.thy: legacy theorem names
Fri, 19 Aug 2011 14:46:45 -0700 huffman delete unused lemmas about limits
Fri, 19 Aug 2011 14:17:28 -0700 huffman Transcendental.thy: add tendsto_intros lemmas;
Fri, 19 Aug 2011 11:49:53 -0700 huffman add lemma isCont_tendsto_compose
Fri, 19 Aug 2011 23:48:18 +0200 wenzelm merged
Fri, 19 Aug 2011 10:46:54 -0700 huffman Transcendental.thy: remove several unused lemmas and simplify some proofs
Fri, 19 Aug 2011 08:40:15 -0700 huffman remove unused lemmas
Fri, 19 Aug 2011 08:39:43 -0700 huffman fold definitions of sin_coeff and cos_coeff in Maclaurin lemmas
Fri, 19 Aug 2011 07:45:22 -0700 huffman remove some redundant simp rules
Fri, 19 Aug 2011 23:25:47 +0200 wenzelm maintain recent future proofs at transaction boundaries;
Fri, 19 Aug 2011 21:40:52 +0200 wenzelm incremental Proofterm.join_body, with join_thms step in fulfill_norm_proof -- avoid full graph traversal of former Proofterm.join_bodies;
Fri, 19 Aug 2011 18:01:23 +0200 wenzelm tuned;
Fri, 19 Aug 2011 17:39:37 +0200 wenzelm tuned signature (again);
Fri, 19 Aug 2011 16:13:26 +0200 wenzelm tuned signature -- treat structure Task_Queue as private to implementation;
Fri, 19 Aug 2011 15:56:26 +0200 wenzelm refined Future.cancel: explicit future allows to join actual cancellation;
Fri, 19 Aug 2011 14:01:20 +0200 wenzelm Future.promise: explicit abort operation (like uninterruptible future job);
Fri, 19 Aug 2011 13:55:32 +0200 wenzelm editable raw text areas: allow user to clear content;
Fri, 19 Aug 2011 13:32:27 +0200 wenzelm more robust use of set_exn_serial, which is based on PolyML.raiseWithLocation internally;
Fri, 19 Aug 2011 12:51:14 +0200 wenzelm more focused use of Multithreading.interrupted: retain interrupts within task group boundary, without loss of information;
Fri, 19 Aug 2011 12:03:44 +0200 wenzelm clarified Future.cond_forks: more uniform handling of exceptional situations;
Fri, 19 Aug 2011 17:05:10 +0900 Cezary Kaliszyk Quotient_Examples: Cset, List_Cset: Lift Inf and Sup directly.
Thu, 18 Aug 2011 22:32:19 -0700 huffman merged
Thu, 18 Aug 2011 22:31:52 -0700 huffman define complex exponential 'expi' as abbreviation for 'exp'
Thu, 18 Aug 2011 21:23:31 -0700 huffman remove more bounded_linear locale interpretations (cf. f0de18b62d63)
Thu, 18 Aug 2011 19:53:03 -0700 huffman optimize some proofs
Thu, 18 Aug 2011 18:10:23 -0700 huffman add Multivariate_Analysis dependencies
Thu, 18 Aug 2011 18:08:43 -0700 huffman import Library/Sum_of_Squares instead of reloading positivstellensatz.ML
Thu, 18 Aug 2011 17:32:02 -0700 huffman declare euclidean_component_zero[simp] at the point it is proved
Fri, 19 Aug 2011 10:23:16 +0900 Cezary Kaliszyk Quotient Package: Regularization: do not fail if no progress is made, leave the subgoal to the user. Injection: try assumptions before extensionality to avoid looping.
Thu, 18 Aug 2011 23:43:22 +0200 wenzelm merged;
Thu, 18 Aug 2011 14:08:39 -0700 huffman merged
Thu, 18 Aug 2011 13:36:58 -0700 huffman remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
Thu, 18 Aug 2011 22:50:28 +0200 haftmann merged
Thu, 18 Aug 2011 22:50:17 +0200 haftmann merged
Thu, 18 Aug 2011 14:01:06 +0200 haftmann avoid duplicated simp add option
Thu, 18 Aug 2011 13:55:26 +0200 haftmann observe distinction between sets and predicates more properly
Thu, 18 Aug 2011 13:25:17 +0200 haftmann moved fundamental lemma fun_eq_iff to theory HOL; tuned whitespace
Thu, 18 Aug 2011 13:10:24 +0200 haftmann avoid case-sensitive name for example theory
Thu, 18 Aug 2011 17:42:35 +0200 nipkow merged
Thu, 18 Aug 2011 17:42:18 +0200 nipkow case_names NEWS
Thu, 18 Aug 2011 17:00:15 +0200 bulwahn adding documentation about simps equation in the inductive package
Thu, 18 Aug 2011 12:06:17 +0200 bulwahn activating narrowing-based quickcheck by default
Thu, 18 Aug 2011 18:07:40 +0200 wenzelm more precise treatment of exception nesting and serial numbers;
Thu, 18 Aug 2011 17:53:32 +0200 wenzelm more careful treatment of exception serial numbers, with propagation to message channel;
Thu, 18 Aug 2011 17:30:47 +0200 wenzelm updated sequential version (cf. b94951f06e48);
Thu, 18 Aug 2011 16:07:58 +0200 wenzelm tuned comments;
Thu, 18 Aug 2011 15:51:34 +0200 wenzelm tuned document;
Thu, 18 Aug 2011 15:39:00 +0200 wenzelm clarified Par_Exn.release_first: prefer plain exn, before falling back on full pack of parallel exceptions;
Thu, 18 Aug 2011 15:37:01 +0200 wenzelm export Par_List.managed_results, to enable specific treatment of results apart from default Par_Exn.release_first;
Thu, 18 Aug 2011 15:15:43 +0200 wenzelm tune Par_Exn.make: balance merge;
Thu, 18 Aug 2011 16:52:19 +0900 Cezary Kaliszyk Quotient_Examples/DList: explicit proof of remdups_eq_member_eq needed for explicit set type.
Wed, 17 Aug 2011 15:12:34 -0700 huffman merged
Wed, 17 Aug 2011 15:03:30 -0700 huffman HOL-IMP: respect set/pred distinction
Wed, 17 Aug 2011 15:02:17 -0700 huffman Determinants.thy: avoid using mem_def/Collect_def
Wed, 17 Aug 2011 14:42:59 -0700 huffman Wfrec.thy: respect set/pred distinction
Thu, 18 Aug 2011 00:02:44 +0200 wenzelm follow updates of Isabelle/Pure;
Wed, 17 Aug 2011 23:41:47 +0200 wenzelm merged
Wed, 17 Aug 2011 14:32:48 -0700 huffman IsaMakefile: target HOLCF-Library now compiles HOL/HOLCF/Library instead of HOL/Library
Wed, 17 Aug 2011 13:10:49 -0700 huffman merged
Wed, 17 Aug 2011 13:10:11 -0700 huffman Lim.thy: generalize and simplify proofs of LIM/LIMSEQ theorems
Wed, 17 Aug 2011 11:39:09 -0700 huffman add lemma tendsto_compose_eventually; use it to shorten some proofs
Wed, 17 Aug 2011 11:07:32 -0700 huffman Topology_Euclidean_Space.thy: simplify some proofs
Wed, 17 Aug 2011 11:06:39 -0700 huffman add lemma metric_tendsto_imp_tendsto
Wed, 17 Aug 2011 09:59:10 -0700 huffman simplify proofs of lemmas open_interval, closed_interval
Wed, 17 Aug 2011 23:37:23 +0200 wenzelm identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
Wed, 17 Aug 2011 22:25:00 +0200 wenzelm clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
Wed, 17 Aug 2011 22:14:22 +0200 wenzelm more systematic handling of parallel exceptions;
Wed, 17 Aug 2011 20:08:36 +0200 wenzelm tuned signature;
Wed, 17 Aug 2011 18:52:21 +0200 haftmann merged
Wed, 17 Aug 2011 18:51:27 +0200 haftmann merged
Wed, 17 Aug 2011 07:13:13 +0200 haftmann merged
Tue, 16 Aug 2011 19:47:50 +0200 haftmann avoid Collect_def in proof
Wed, 17 Aug 2011 18:05:31 +0200 wenzelm modernized signature of Term.absfree/absdummy;
Wed, 17 Aug 2011 16:46:58 +0200 wenzelm improved default context for ML toplevel pretty-printing;
Wed, 17 Aug 2011 16:30:38 +0200 wenzelm less verbosity for 'function' and 'fun': observe "int" flag more carefully (cf. a32ca9165928);
Wed, 17 Aug 2011 16:01:27 +0200 wenzelm some convenience actions/shortcuts for control symbols;
Wed, 17 Aug 2011 15:14:48 +0200 wenzelm export Function_Fun.fun_config for user convenience;
Wed, 17 Aug 2011 13:14:20 +0200 wenzelm moved theory Nested_Environment to HOL-Unix (a bit too specific for HOL-Library);
Wed, 17 Aug 2011 10:03:58 +0200 blanchet distinguish THF syntax with and without choice (Satallax vs. LEO-II)
Tue, 16 Aug 2011 15:02:20 -0700 huffman merged
Tue, 16 Aug 2011 09:31:23 -0700 huffman add simp rules for isCont
Tue, 16 Aug 2011 23:39:58 +0200 wenzelm updated keywords -- old codegen is no longer in Pure;
Tue, 16 Aug 2011 23:39:30 +0200 wenzelm include HOL-Library keywords for the sake of recdef;
Tue, 16 Aug 2011 23:25:02 +0200 wenzelm merged
Tue, 16 Aug 2011 13:07:52 -0700 huffman Multivariate_Analysis includes Determinants.thy, but doesn't import it by default
Tue, 16 Aug 2011 07:56:17 -0700 huffman get Multivariate_Analysis/Determinants.thy compiled and working again
Tue, 16 Aug 2011 07:06:54 -0700 huffman get Library/Permutations.thy compiled and working again
Tue, 16 Aug 2011 23:17:26 +0200 wenzelm workaround for Cygwin, to make it work in the important special case without extra files;
Tue, 16 Aug 2011 22:48:31 +0200 wenzelm more robust Thy_Header.base_name, with minimal assumptions about path syntax;
Tue, 16 Aug 2011 21:54:06 +0200 wenzelm tuned message;
Tue, 16 Aug 2011 21:50:53 +0200 wenzelm more robust treatment of node dependencies in incremental edits;
Tue, 16 Aug 2011 21:13:52 +0200 wenzelm use full .thy file name as node name, which makes MiscUtilities.resolveSymlinks/File.getCanonicalPath more predictable;
Tue, 16 Aug 2011 12:06:49 +0200 wenzelm omit MiscUtilities.resolveSymlinks for now -- odd effects on case-insensible file-system;
Mon, 15 Aug 2011 19:42:52 -0700 huffman merged
Mon, 15 Aug 2011 18:35:36 -0700 huffman generalize lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq to class topological_space
Mon, 15 Aug 2011 16:48:05 -0700 huffman add lemma tendsto_compose
Mon, 15 Aug 2011 16:18:13 -0700 huffman remove extraneous subsection heading
Mon, 15 Aug 2011 15:11:55 -0700 huffman generalized lemma closed_Collect_eq
Mon, 15 Aug 2011 14:50:24 -0700 huffman remove duplicate lemma disjoint_iff
Mon, 15 Aug 2011 14:29:17 -0700 huffman Library/Product_Vector.thy: class instances for t0_space, t1_space, and t2_space
Mon, 15 Aug 2011 14:09:39 -0700 huffman add lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq;
Mon, 15 Aug 2011 12:18:34 -0700 huffman generalize lemma continuous_uniform_limit to class metric_space
Mon, 15 Aug 2011 12:13:46 -0700 huffman remove duplicate lemmas eventually_conjI, eventually_and, eventually_false
Mon, 15 Aug 2011 10:49:48 -0700 huffman Topology_Euclidean_Space.thy: organize section headings
Mon, 15 Aug 2011 09:08:17 -0700 huffman simplify some proofs
Sun, 14 Aug 2011 13:04:57 -0700 huffman generalize lemma convergent_subseq_convergent
Sun, 14 Aug 2011 11:44:12 -0700 huffman locale-ize some definitions, so perfect_space and heine_borel can inherit from the proper superclasses
Sun, 14 Aug 2011 10:47:47 -0700 huffman locale-ize some constant definitions, so complete_space can inherit from metric_space
Sun, 14 Aug 2011 10:25:43 -0700 huffman generalize constant 'lim' and limit uniqueness theorems to class t2_space
Tue, 16 Aug 2011 07:17:15 +0900 Cezary Kaliszyk Quotient Package: make quotient_type work with separate set type
Mon, 15 Aug 2011 22:31:17 +0200 wenzelm updated README;
Mon, 15 Aug 2011 21:54:32 +0200 wenzelm touch descendants of edited nodes;
Mon, 15 Aug 2011 21:05:30 +0200 wenzelm parellel scheduling of node edits and execution;
Mon, 15 Aug 2011 20:38:16 +0200 wenzelm tuned error message;
Mon, 15 Aug 2011 20:19:41 +0200 wenzelm retrieve imports from document state, with fall-back on theory loader for preloaded theories;
Mon, 15 Aug 2011 19:27:55 +0200 wenzelm explicit check of finished evaluation;
Mon, 15 Aug 2011 16:38:42 +0200 wenzelm refined Document.edit: less stateful update via Graph.schedule;
Mon, 15 Aug 2011 14:54:36 +0200 wenzelm simplified exec: eliminated unused status flag;
Sun, 14 Aug 2011 08:45:38 -0700 huffman consistently use variable name 'F' for filters
Sun, 14 Aug 2011 07:54:24 -0700 huffman generalize lemmas about LIM and LIMSEQ to tendsto
Sat, 13 Aug 2011 18:10:14 -0700 huffman HOL-Nominal-Examples: respect distinction between sets and functions
Sat, 13 Aug 2011 22:04:07 +0200 wenzelm less verbosity in batch mode -- spam reduction and notable performance improvement;
Sat, 13 Aug 2011 21:28:01 +0200 wenzelm merged
Sat, 13 Aug 2011 07:56:55 -0700 huffman HOL-Hahn_Banach: use Set_Algebras library
Sat, 13 Aug 2011 07:39:35 -0700 huffman ex/Quickcheck_Examples.thy: respect distinction between sets and functions
Sat, 13 Aug 2011 21:06:01 +0200 wenzelm clarified Toplevel.end_theory;
Sat, 13 Aug 2011 20:49:41 +0200 wenzelm simplified Toplevel.init_theory: discontinued special name argument;
Sat, 13 Aug 2011 20:41:29 +0200 wenzelm simplified Toplevel.init_theory: discontinued special master argument;
Sat, 13 Aug 2011 20:20:36 +0200 wenzelm provide node header via Scala layer;
Sat, 13 Aug 2011 16:07:26 +0200 wenzelm reduced verbosity;
Sat, 13 Aug 2011 16:04:28 +0200 wenzelm tuned signature;
Sat, 13 Aug 2011 15:59:26 +0200 wenzelm clarified node header -- exclude master_dir;
Sat, 13 Aug 2011 13:48:26 +0200 wenzelm tuned;
Sat, 13 Aug 2011 13:42:35 +0200 wenzelm maintain node header;
Sat, 13 Aug 2011 12:23:51 +0200 kleing removed unused lemma; removed old-style ;
Sat, 13 Aug 2011 12:05:52 +0200 kleing point isatest-statistics to the right afp log files
Sat, 13 Aug 2011 11:57:13 +0200 kleing IMP/Util distinguishes between sets and functions again; imported only where used.
Fri, 12 Aug 2011 20:55:22 -0700 huffman remove redundant lemma setsum_norm in favor of norm_setsum;
Fri, 12 Aug 2011 16:47:53 -0700 huffman merged
Fri, 12 Aug 2011 14:45:50 -0700 huffman make more HOL theories work with separate set type
Sat, 13 Aug 2011 00:34:54 +0200 wenzelm immediate fork of initial workers -- avoid 5 ticks (250ms) for adaptive scheme (a07558eb5029);
Fri, 12 Aug 2011 23:29:28 +0200 wenzelm merged
Fri, 12 Aug 2011 09:17:30 -0700 huffman merged
Fri, 12 Aug 2011 09:17:24 -0700 huffman make Multivariate_Analysis work with separate set type
Fri, 12 Aug 2011 07:18:28 -0700 huffman make HOLCF work with separate set type
Fri, 12 Aug 2011 07:13:12 -0700 huffman merged
Thu, 11 Aug 2011 14:24:05 -0700 huffman avoid duplicate rule warnings
Thu, 11 Aug 2011 13:05:56 -0700 huffman modify euclidean_space class to include basis set
Thu, 11 Aug 2011 09:11:15 -0700 huffman remove lemma stupid_ext
Fri, 12 Aug 2011 17:01:30 +0200 nipkow documented extended version of case_names attribute
Fri, 12 Aug 2011 22:10:49 +0200 wenzelm normalized theory dependencies wrt. file_store;
Fri, 12 Aug 2011 20:32:25 +0200 wenzelm general Graph.schedule;
Fri, 12 Aug 2011 15:30:12 +0200 wenzelm allow "$" within basic path elements (NB: initial "$" refers to path variable);
Fri, 12 Aug 2011 15:28:30 +0200 wenzelm clarified document model header: master_dir (native wrt. editor, potentially URL) and node_name (full canonical path);
Fri, 12 Aug 2011 12:03:17 +0200 wenzelm simplified class Thy_Header;
Fri, 12 Aug 2011 11:41:26 +0200 wenzelm clarified Exn.message;
Thu, 11 Aug 2011 20:32:44 +0200 wenzelm uniform treatment of header edits as document edits;
Thu, 11 Aug 2011 18:01:28 +0200 wenzelm explicit datatypes for document node edits;
Thu, 11 Aug 2011 13:24:49 +0200 wenzelm tuned;
Thu, 11 Aug 2011 13:22:22 +0200 wenzelm disentangled nested ML files;
Thu, 11 Aug 2011 13:05:23 +0200 wenzelm minimal script to run raw Poly/ML with concurrency library;
Thu, 11 Aug 2011 12:53:41 +0200 wenzelm somewhat more uniform THIS;
Thu, 11 Aug 2011 12:49:14 +0200 wenzelm more trimming;
Thu, 11 Aug 2011 12:30:41 +0200 wenzelm recovered some ML toplevel pp;
Thu, 11 Aug 2011 12:24:10 +0200 wenzelm some trimming;
Thu, 11 Aug 2011 12:11:50 +0200 wenzelm prefix of Pure/ROOT.ML required for concurrency within the ML runtime;
Thu, 11 Aug 2011 11:40:25 +0200 wenzelm redundant use of misc_legacy.ML;
Thu, 11 Aug 2011 10:36:34 +0200 krauss eliminated use of recdef
Thu, 11 Aug 2011 09:41:21 +0200 krauss removed obsolete recdef-related examples
Thu, 11 Aug 2011 09:15:45 +0200 krauss removed unused material, which does not really belong here
Wed, 10 Aug 2011 18:07:32 -0700 huffman merged
Wed, 10 Aug 2011 18:02:16 -0700 huffman avoid warnings about duplicate rules
Wed, 10 Aug 2011 17:02:03 -0700 huffman follow standard naming scheme for sgn_vec_def
Wed, 10 Aug 2011 16:35:50 -0700 huffman remove several redundant and unused theorems about derivatives
Wed, 10 Aug 2011 15:56:48 -0700 huffman remove redundant lemma
Wed, 10 Aug 2011 14:25:56 -0700 huffman simplify proof of lemma bounded_component
Wed, 10 Aug 2011 14:10:52 -0700 huffman simplify some proofs
Wed, 10 Aug 2011 13:13:37 -0700 huffman more uniform naming scheme for finite cartesian product type and related theorems
Wed, 10 Aug 2011 10:13:16 -0700 huffman move euclidean_space instance from Cartesian_Euclidean_Space.thy to Finite_Cartesian_Product.thy
Wed, 10 Aug 2011 21:24:26 +0200 wenzelm merged
Wed, 10 Aug 2011 09:23:42 -0700 huffman split Linear_Algebra.thy from Euclidean_Space.thy
Wed, 10 Aug 2011 08:42:26 -0700 huffman full import paths
Wed, 10 Aug 2011 01:36:53 -0700 huffman declare tendsto_const [intro] (accidentally removed in 230a8665c919)
Wed, 10 Aug 2011 00:31:51 -0700 huffman merged
Wed, 10 Aug 2011 00:29:31 -0700 huffman simplified definition of class euclidean_space;
Tue, 09 Aug 2011 13:09:35 -0700 huffman bounded_linear interpretation for euclidean_component
Tue, 09 Aug 2011 12:50:22 -0700 huffman lemma bounded_linear_intro
Tue, 09 Aug 2011 10:42:07 -0700 huffman avoid duplicate rewrite warnings
Tue, 09 Aug 2011 10:30:00 -0700 huffman mark some redundant theorems as legacy
Tue, 09 Aug 2011 08:53:12 -0700 huffman Derivative.thy: more sensible subsection headings
Tue, 09 Aug 2011 07:37:18 -0700 huffman Derivative.thy: clean up formatting
Mon, 08 Aug 2011 21:17:52 -0700 huffman instance real_basis_with_inner < perfect_space
Wed, 10 Aug 2011 20:53:43 +0200 wenzelm old term operations are legacy;
Wed, 10 Aug 2011 20:12:36 +0200 wenzelm moved old code generator to src/Tools/;
Wed, 10 Aug 2011 19:46:48 +0200 wenzelm avoid OldTerm operations -- with subtle changes of semantics;
Wed, 10 Aug 2011 19:45:57 +0200 wenzelm avoid OldTerm operations -- with subtle changes of semantics;
Wed, 10 Aug 2011 19:45:41 +0200 wenzelm avoid OldTerm operations -- with subtle changes of semantics;
Wed, 10 Aug 2011 19:21:28 +0200 wenzelm avoid OldTerm operations -- with subtle changes of semantics;
Wed, 10 Aug 2011 16:26:05 +0200 wenzelm tuned signature;
Wed, 10 Aug 2011 16:24:39 +0200 wenzelm Goal.forked: clarified handling of interrupts;
Wed, 10 Aug 2011 16:05:14 +0200 wenzelm future_job: explicit indication of interrupts;
Wed, 10 Aug 2011 15:17:24 +0200 wenzelm more explicit Simple_Thread.interrupt_unsynchronized, to emphasize its meaning;
Wed, 10 Aug 2011 14:28:55 +0200 wenzelm synchronized cancel and flushing of Multithreading.interrupted state, to ensure that interrupts stay within task boundaries;
Wed, 10 Aug 2011 14:04:45 +0200 wenzelm tuned source structure;
Wed, 10 Aug 2011 10:59:37 +0200 wenzelm bash_output_fifo blocks on Cygwin 1.7.x;
Tue, 09 Aug 2011 23:54:17 +0200 berghofe rename_bvs now avoids introducing name clashes between schematic variables
Tue, 09 Aug 2011 22:37:33 +0200 wenzelm merged
Tue, 09 Aug 2011 20:24:48 +0200 haftmann tuned proofs
Tue, 09 Aug 2011 18:52:18 +0200 haftmann merged
Tue, 09 Aug 2011 08:07:22 +0200 haftmann tuned header
Tue, 09 Aug 2011 08:06:15 +0200 haftmann more uniform naming scheme for Inf/INF and Sup/SUP lemmas
Tue, 09 Aug 2011 16:09:10 +0200 kleing removed "extremely ambigous" warning; has been ignored by everyone for years.
Tue, 09 Aug 2011 22:30:33 +0200 wenzelm misc tuning and clarification;
Tue, 09 Aug 2011 21:48:36 +0200 wenzelm tuned whitespace;
Tue, 09 Aug 2011 17:33:17 +0200 blanchet support local HOATPs
Tue, 09 Aug 2011 17:33:17 +0200 blanchet document local HOATPs
Tue, 09 Aug 2011 17:33:17 +0200 blanchet workaround THF parser limitation
Tue, 09 Aug 2011 17:33:17 +0200 blanchet LEO-II also supports FOF
Tue, 09 Aug 2011 15:50:13 +0200 wenzelm misc tuning and simplification;
Tue, 09 Aug 2011 15:41:00 +0200 wenzelm updated documentation of method "split" according to e6a4bb832b46;
Tue, 09 Aug 2011 09:39:49 +0200 blanchet updated references to CADE-23
Tue, 09 Aug 2011 09:33:50 +0200 blanchet renamed E wrappers for consistency with CASC conventions
Tue, 09 Aug 2011 09:33:01 +0200 blanchet updated Sledgehammer docs
Tue, 09 Aug 2011 09:24:34 +0200 blanchet add line number prefix to output file name
Tue, 09 Aug 2011 09:07:59 +0200 blanchet added "sound" option to Mirabelle
Tue, 09 Aug 2011 09:05:22 +0200 blanchet move lambda-lifting code to ATP encoding, so it can be used by Metis
Tue, 09 Aug 2011 09:05:21 +0200 blanchet load lambda-lifting structure earlier, so it can be used in Metis
Tue, 09 Aug 2011 07:44:17 +0200 haftmann merged
Mon, 08 Aug 2011 22:33:36 +0200 haftmann move legacy candiates to bottom; marked candidates for default simp rules
Mon, 08 Aug 2011 22:11:00 +0200 haftmann merged
Mon, 08 Aug 2011 19:30:18 +0200 haftmann dropped lemmas (Inf|Sup)_(singleton|binary)
Mon, 08 Aug 2011 19:21:11 +0200 haftmann dropped lemmas (Inf|Sup)_(singleton|binary)
Mon, 08 Aug 2011 19:26:53 -0700 huffman rename type 'a net to 'a filter, following standard mathematical terminology
Mon, 08 Aug 2011 18:36:32 -0700 huffman HOLCF: fix warnings about unreferenced identifiers
Mon, 08 Aug 2011 16:57:37 -0700 huffman remove duplicate lemmas
Mon, 08 Aug 2011 16:19:57 -0700 huffman merged
Mon, 08 Aug 2011 16:04:58 -0700 huffman fix perfect_space instance proof for finite cartesian product (cf. 5b970711fb39)
Mon, 08 Aug 2011 15:27:24 -0700 huffman generalize sequence lemmas
Mon, 08 Aug 2011 15:11:38 -0700 huffman generalize more lemmas about compactness
Mon, 08 Aug 2011 15:03:34 -0700 huffman generalize compactness equivalence lemmas
Mon, 08 Aug 2011 14:59:01 -0700 huffman lemma bolzano_weierstrass_imp_compact
Mon, 08 Aug 2011 14:44:20 -0700 huffman class perfect_space inherits from topological_space;
Mon, 08 Aug 2011 21:55:01 +0200 wenzelm merged
Mon, 08 Aug 2011 16:47:55 +0200 kleing import constant folding theory into IMP
Sat, 06 Aug 2011 15:48:08 +0200 kleing make syntax ambiguity warnings a config option
Mon, 08 Aug 2011 11:47:41 -0700 huffman add lemmas INF_image, SUP_image
Mon, 08 Aug 2011 11:25:18 -0700 huffman declare {INF,SUP}_empty [simp]
Mon, 08 Aug 2011 10:32:55 -0700 huffman rename Pair_fst_snd_eq to prod_eq_iff (keeping old name too)
Mon, 08 Aug 2011 10:26:26 -0700 huffman standard theorem naming scheme: complex_eqI, complex_eq_iff
Mon, 08 Aug 2011 09:52:09 -0700 huffman moved division ring stuff from Rings.thy to Fields.thy
Mon, 08 Aug 2011 08:55:49 -0700 huffman Library/Product_ord: wellorder instance for products
Mon, 08 Aug 2011 21:11:10 +0200 wenzelm modernized file proof_checker.ML;
Mon, 08 Aug 2011 20:47:12 +0200 wenzelm tuned thm_of_proof: build lookup table within closure;
Mon, 08 Aug 2011 20:21:49 +0200 wenzelm added Reconstruct.proof_of convenience;
Mon, 08 Aug 2011 19:59:35 +0200 wenzelm ship message in one piece;
Mon, 08 Aug 2011 17:23:15 +0200 wenzelm misc tuning -- eliminated old-fashioned rep_thm;
Mon, 08 Aug 2011 16:38:59 +0200 wenzelm modernized strcture Proof_Checker;
Mon, 08 Aug 2011 16:09:34 +0200 wenzelm less ambitious use of AttributedString, for proper caret painting within \<^sup>\<foobar>;
Mon, 08 Aug 2011 13:48:38 +0200 wenzelm updated imports;
Mon, 08 Aug 2011 13:40:24 +0200 wenzelm proper signature;
Mon, 08 Aug 2011 13:39:51 +0200 wenzelm made SML/NJ happy;
Mon, 08 Aug 2011 13:29:54 +0200 wenzelm slightly more uniform messages;
Mon, 08 Aug 2011 13:19:19 +0200 wenzelm avoid pointless completion of illegal control commands;
Mon, 08 Aug 2011 08:56:58 +0200 nipkow removed old expand_fun_eq
Mon, 08 Aug 2011 08:25:28 +0200 nipkow fixed index entry
Mon, 08 Aug 2011 07:35:42 +0200 nipkow removed old recdef and types usage
Mon, 08 Aug 2011 07:13:16 +0200 nipkow merged
Sat, 06 Aug 2011 14:16:23 +0200 nipkow extended user-level attribute case_names with names for case hypotheses
Mon, 01 Aug 2011 12:08:53 +0200 nipkow infrastructure for attaching names to hypothesis in cases; realised via the same tag mechanism as case names
Sun, 07 Aug 2011 23:08:07 +0200 wenzelm workaround for Java 1.7 where javax.swing.JComboBox<E> is generic;
Sun, 07 Aug 2011 23:05:50 +0200 wenzelm updated version information;
Sun, 07 Aug 2011 18:38:36 +0200 wenzelm fixed document;
Fri, 05 Aug 2011 23:06:54 +0200 haftmann tuned order: pushing INF and SUP to Inf and Sup
Fri, 05 Aug 2011 22:58:17 +0200 haftmann tuned order: pushing INF and SUP to Inf and Sup
Fri, 05 Aug 2011 22:45:57 +0200 haftmann generalized lemmas to complete lattices
Fri, 05 Aug 2011 17:22:28 +0200 Andreas Lochbihler merged
Fri, 05 Aug 2011 16:55:14 +0200 Andreas Lochbihler replace old SML code generator by new code generator in MicroJava/J
Thu, 04 Aug 2011 16:49:57 +0200 kleing new state syntax with less conflicts
Fri, 05 Aug 2011 14:16:44 +0200 Andreas Lochbihler replace old SML code generator by new code generator in MicroJava/JVM and /BV
Fri, 05 Aug 2011 00:14:08 +0200 haftmann merged
Thu, 04 Aug 2011 20:11:39 +0200 haftmann more fine-granular instantiation
Thu, 04 Aug 2011 19:29:52 +0200 haftmann solving duality problem for complete_distrib_lattice; tuned
Thu, 04 Aug 2011 23:21:04 +0200 berghofe merged
Thu, 04 Aug 2011 17:40:48 +0200 berghofe Pending FDL types may now be associated with Isabelle types as well.
Thu, 04 Aug 2011 07:33:08 +0200 haftmann tuned orthography
Thu, 04 Aug 2011 07:31:59 +0200 haftmann avoid yet unknown fact antiquotation
Thu, 04 Aug 2011 07:31:43 +0200 haftmann NEWS
Wed, 03 Aug 2011 23:21:53 +0200 haftmann more specific instantiation
Wed, 03 Aug 2011 23:21:52 +0200 haftmann tuned
Wed, 03 Aug 2011 23:21:52 +0200 haftmann class complete_distrib_lattice
Wed, 03 Aug 2011 16:08:02 +0200 bulwahn NEWS
Wed, 03 Aug 2011 14:24:23 +0200 bulwahn removing value invocations with the SML code generator
Wed, 03 Aug 2011 13:59:59 +0200 bulwahn removing the SML evaluator
Wed, 03 Aug 2011 11:09:12 +0200 kleing fixed wrong isubs in IMP/Types
Tue, 02 Aug 2011 08:28:34 -0700 huffman Extended_Nat.thy: renamed iSuc to eSuc, standardized theorem names
Tue, 02 Aug 2011 07:36:58 -0700 huffman NEWS: fix typo
Tue, 02 Aug 2011 13:07:00 +0200 krauss updated unchecked forward reference
Tue, 02 Aug 2011 12:27:24 +0200 krauss replaced Nitpick's hardwired basic_ersatz_table by context data
Tue, 02 Aug 2011 12:17:48 +0200 krauss NEWS
Tue, 02 Aug 2011 11:52:57 +0200 krauss moved recursion combinator to HOL/Library/Wfrec.thy -- it is so fundamental and well-known that it should survive recdef
Tue, 02 Aug 2011 10:36:50 +0200 krauss moved recdef package to HOL/Library/Old_Recdef.thy
Tue, 02 Aug 2011 10:03:14 +0200 krauss added dynamic ersatz_table to Nitpick's data slot
Tue, 02 Aug 2011 10:03:12 +0200 krauss eliminated obsolete recdef/wfrec related declarations
Mon, 01 Aug 2011 20:21:11 +0200 kleing more consistent naming in IMP/Comp_Rev
Mon, 01 Aug 2011 19:53:30 +0200 haftmann merged
Sat, 30 Jul 2011 08:24:46 +0200 haftmann tuned proofs
Fri, 29 Jul 2011 19:47:55 +0200 haftmann tuned proofs
Mon, 01 Aug 2011 09:31:10 -0700 huffman new theory HOL/Library/Product_Lattice.thy
Sun, 31 Jul 2011 11:13:38 -0700 huffman domain package: more informative error message for illegal indirect recursion
Thu, 28 Jul 2011 16:56:14 +0200 kleing compiler proof cleanup
Thu, 28 Jul 2011 16:32:49 +0200 blanchet added helpers for "All" and "Ex"
Thu, 28 Jul 2011 16:32:48 +0200 blanchet put parentheses around non-trivial metis call
Thu, 28 Jul 2011 16:32:39 +0200 blanchet no needless mangling
Thu, 28 Jul 2011 15:15:26 +0200 kleing resolved code_pred FIXME in IMP; clearer notation for exec_n
Thu, 28 Jul 2011 11:49:03 +0200 blanchet clean up temporary directory hack
Thu, 28 Jul 2011 11:43:45 +0200 blanchet tuning
Thu, 28 Jul 2011 11:43:45 +0200 blanchet fixed lambda concealing
Thu, 28 Jul 2011 11:43:45 +0200 blanchet make SML/NJ happy
Thu, 28 Jul 2011 10:42:24 +0200 hoelzl simplified definition of vector (also removed Cartesian_Euclidean_Space.from_nat which collides with Countable.from_nat)
Thu, 28 Jul 2011 05:52:28 -0200 noschinl document coercions
Wed, 27 Jul 2011 20:28:00 +0200 bulwahn rudimentary documentation of the quotient package in the isar reference manual
Wed, 27 Jul 2011 19:35:00 +0200 hoelzl to_nat is injective on arbitrary domains
Wed, 27 Jul 2011 19:34:30 +0200 hoelzl finite vimage on arbitrary domains
Tue, 26 Jul 2011 22:53:06 +0200 blanchet updated Sledgehammer documentation
Tue, 26 Jul 2011 22:53:06 +0200 blanchet renamed "preds" encodings to "guards"
Tue, 26 Jul 2011 18:11:38 +0200 bulwahn more precise dependencies
Tue, 26 Jul 2011 14:53:00 +0200 blanchet further worked around LEO-II parser limitation, with eta-expansion
Tue, 26 Jul 2011 14:53:00 +0200 blanchet use syntactic sugar whenever possible in THF problems, to work around current LEO-II parser limitation (bang bang and query query are not handled correctly)
Tue, 26 Jul 2011 14:53:00 +0200 blanchet no need for existential witnesses for sorts in TFF and THF formats
Tue, 26 Jul 2011 14:53:00 +0200 blanchet mangle "undefined"
Tue, 26 Jul 2011 14:53:00 +0200 blanchet tuning -- remove useless function (at this point combinators are already in)
Tue, 26 Jul 2011 14:53:00 +0200 blanchet remove spurious message
Tue, 26 Jul 2011 14:53:00 +0200 blanchet give E at least two seconds -- anything else risks causing too early timeouts in the minimizer, because of too conservative time computations in E and eproof scripts
Tue, 26 Jul 2011 14:50:15 +0200 Andreas Lochbihler merged
Tue, 26 Jul 2011 14:05:28 +0200 Andreas Lochbihler fixed code generator setup in List_Cset
Tue, 26 Jul 2011 13:50:03 +0200 hoelzl enat is a complete_linorder instance
Tue, 26 Jul 2011 12:44:36 +0200 Andreas Lochbihler merged
Tue, 26 Jul 2011 10:49:34 +0200 Andreas Lochbihler Add theory for setting up monad syntax for Cset
Tue, 26 Jul 2011 11:48:11 +0200 bulwahn merged
Tue, 26 Jul 2011 08:07:01 +0200 bulwahn removing expectations from quickcheck example
Tue, 26 Jul 2011 08:07:00 +0200 bulwahn adding remarks after static inspection of the invocation of the SML code generator
Tue, 26 Jul 2011 10:03:19 +0200 Andreas Lochbihler merged
Mon, 25 Jul 2011 16:55:48 +0200 Andreas Lochbihler added operations to Cset with code equations in backing implementations
Mon, 25 Jul 2011 23:27:20 +0200 haftmann merged
Mon, 25 Jul 2011 23:26:55 +0200 haftmann adjusted to tailored version of ball_simps
Sun, 24 Jul 2011 22:38:13 +0200 haftmann adjusted to tailored version of bex_simps
Sun, 24 Jul 2011 21:27:25 +0200 haftmann more coherent structure in and across theories
Mon, 25 Jul 2011 14:10:12 +0200 blanchet declare "undefined" constant
Mon, 25 Jul 2011 14:10:12 +0200 blanchet make compile
Mon, 25 Jul 2011 14:10:12 +0200 blanchet thread proper context through, to make sure that "using [[meson_max_clauses = 200]]" is not ignored when clausifying the conjecture
Mon, 25 Jul 2011 14:10:12 +0200 blanchet tuning
Mon, 25 Jul 2011 14:10:12 +0200 blanchet introduced hybrid lambda translation
Mon, 25 Jul 2011 14:10:12 +0200 blanchet avoid needless type args for lifted-lambdas
Mon, 25 Jul 2011 11:21:45 +0200 bulwahn replacing conversion function of old code generator by the current code generator in the reflection tactic
Mon, 25 Jul 2011 11:21:44 +0200 bulwahn fixed typo
Mon, 25 Jul 2011 10:43:14 +0200 bulwahn removing SML_Quickcheck
Mon, 25 Jul 2011 10:42:32 +0200 bulwahn NEWS
Mon, 25 Jul 2011 10:40:52 +0200 bulwahn added legacy warning to old code generation evaluation
Mon, 25 Jul 2011 10:40:51 +0200 bulwahn added legacy warning to old code generation commands
Sat, 23 Jul 2011 23:33:59 +0200 wenzelm merged
Sat, 23 Jul 2011 20:05:28 +0200 bulwahn correcting last example in Predicate_Compile_Examples
Sat, 23 Jul 2011 22:22:21 +0200 wenzelm make double-sure that interrupts are flushed before executing new work (cf. 22f8c2483bd2);
Sat, 23 Jul 2011 21:29:56 +0200 wenzelm more detailed tracing;
Sat, 23 Jul 2011 20:34:33 +0200 wenzelm defensive Term_Sharing, to avoid extending trusted code base of inference kernel;
Sat, 23 Jul 2011 20:11:18 +0200 wenzelm more precise parse_name according to XML standard;
Sat, 23 Jul 2011 17:22:28 +0200 wenzelm explicit structure ML_System;
Sat, 23 Jul 2011 16:37:17 +0200 wenzelm defer evaluation of Scan.message, for improved performance in the frequent situation where failure is handled later (e.g. via ||);
Sat, 23 Jul 2011 16:12:12 +0200 wenzelm tuned;
Fri, 22 Jul 2011 07:33:34 +0200 haftmann merged
Fri, 22 Jul 2011 07:33:29 +0200 haftmann dropped errorneous hint
Thu, 21 Jul 2011 22:47:13 +0200 haftmann moved some lemmas
Thu, 21 Jul 2011 21:56:24 +0200 haftmann merged
Thu, 21 Jul 2011 18:40:31 +0200 haftmann ereal is a complete_linorder instance
Wed, 20 Jul 2011 22:14:39 +0200 haftmann class complete_linorder
Thu, 21 Jul 2011 21:29:10 +0200 blanchet make "concealed" lambda translation sound
Thu, 21 Jul 2011 08:33:57 +0200 bulwahn deactivating all quickcheck invocations until parallel invocation works safely
Thu, 21 Jul 2011 08:31:35 +0200 bulwahn adapting two examples in Predicate_Compile_Examples
Wed, 20 Jul 2011 23:47:27 +0200 blanchet use a more robust naming convention for "polymorphic" frees -- the check is an overapproximation but that's fine as far as soundness is concerned
Wed, 20 Jul 2011 16:15:33 +0200 Cezary Kaliszyk merge
Wed, 20 Jul 2011 16:14:49 +0200 Cezary Kaliszyk Quotient Package: handle Bound variables in rep_abs_rsp_tac not only at top-level of the goal
Wed, 20 Jul 2011 15:42:23 +0200 hoelzl add code generator setup and tests for ereal
Wed, 20 Jul 2011 15:09:53 +0200 boehmes removed debugging facilities accidentally left in the committed code
Wed, 20 Jul 2011 13:29:54 +0200 boehmes more precise dependencies
Wed, 20 Jul 2011 13:27:01 +0200 boehmes merged
Wed, 20 Jul 2011 12:23:20 +0200 boehmes generalized lambda-lifting such that it is less specifically tailored for SMT (it does not anymore dependent on any SMT-specific code)
Wed, 20 Jul 2011 09:23:12 +0200 boehmes moved lambda-lifting on terms into a separate structure (for better re-use in tools other than SMT)
Wed, 20 Jul 2011 09:23:09 +0200 boehmes removed old (unused) SMT monomorphizer
Wed, 20 Jul 2011 13:24:49 +0200 krauss added UNION
Wed, 20 Jul 2011 10:48:00 +0200 hoelzl merged
Tue, 19 Jul 2011 14:38:48 +0200 hoelzl rename Fin to enat
Tue, 19 Jul 2011 14:38:29 +0200 hoelzl add ereal to typeclass infinity
Tue, 19 Jul 2011 14:37:49 +0200 hoelzl add nat => enat coercion
Tue, 19 Jul 2011 14:37:09 +0200 hoelzl Introduce infinity type class
Tue, 19 Jul 2011 14:36:12 +0200 hoelzl Rename extreal => ereal
Tue, 19 Jul 2011 14:35:44 +0200 hoelzl rename Nat_Infinity (inat) to Extended_Nat (enat)
Wed, 20 Jul 2011 10:11:08 +0200 Cezary Kaliszyk HOL/Import reorganization/cleaning. Factor 9 speedup. Remove Import XML parser in favor of much faster of Isabelle's XML parser. Remove ImportRecording since we can use Isabelle images.
Wed, 20 Jul 2011 08:46:17 +0200 kleing build an image for HOL-IMP
Wed, 20 Jul 2011 08:16:42 +0200 bulwahn deactivating quickcheck invocation in this example until the Interrupt issue is understood
Wed, 20 Jul 2011 08:16:41 +0200 bulwahn removing inner time limits in quickcheck
Wed, 20 Jul 2011 08:16:39 +0200 bulwahn updating documentation about quickcheck; adding information about try
Wed, 20 Jul 2011 08:16:38 +0200 bulwahn adapting example in Predicate_Compile_Examples
Wed, 20 Jul 2011 08:16:36 +0200 bulwahn exporting function in quickcheck; adapting mutabelle script
Wed, 20 Jul 2011 08:16:35 +0200 bulwahn more information for the user how to deactivate quickcheck_narrowing if he does not want to use it
Wed, 20 Jul 2011 08:16:33 +0200 bulwahn making messages more informative
Wed, 20 Jul 2011 08:16:32 +0200 bulwahn only use exhaustive testing in this quickcheck example
Wed, 20 Jul 2011 00:37:42 +0200 blanchet parse equalities correctly in Nitrox parser
Wed, 20 Jul 2011 00:37:42 +0200 blanchet pass type arguments to lambda-lifted Frees, to account for polymorphism
Wed, 20 Jul 2011 00:37:42 +0200 blanchet generate slightly less type information -- this should be sound since type arguments should keep things cleanly apart
Wed, 20 Jul 2011 00:37:42 +0200 blanchet avoid calling "Term.is_first_order" (indirectly) on a term with loose de Bruijns -- this is not necessary anyway because of the Abs check in "simple_translate_lambdas"
Wed, 20 Jul 2011 00:37:42 +0200 blanchet remove offset from Mirabelle output
Tue, 19 Jul 2011 11:15:38 +0200 krauss the HOL4PROOFS setting is actually HOL4_PROOFS
Tue, 19 Jul 2011 07:14:14 +0200 haftmann merged
Mon, 18 Jul 2011 21:52:34 +0200 haftmann proof tuning
Mon, 18 Jul 2011 21:49:39 +0200 haftmann generalization; various notation and proof tuning
Mon, 18 Jul 2011 21:34:01 +0200 haftmann avoid misunderstandable names
Mon, 18 Jul 2011 21:15:51 +0200 haftmann moved lemmas to appropriate theory
Tue, 19 Jul 2011 00:16:18 +0200 krauss forgotten qualifier
Tue, 19 Jul 2011 00:07:21 +0200 krauss values_timeout defaults to 600.0 on SML/NJ -- saves us from cluttering all theories equivalent declarations
Mon, 18 Jul 2011 23:48:28 +0200 krauss killed use of PolyML.makestring
Mon, 18 Jul 2011 23:35:50 +0200 krauss added experimental mira configuration for HOL Light importer
Mon, 18 Jul 2011 18:52:52 +0200 boehmes allow rules with premises to be declared as z3_rule (to circumvent incompleteness of Z3 proof reconstruction)
Mon, 18 Jul 2011 13:49:26 +0200 bulwahn unactivating narrowing-based quickcheck by default
Mon, 18 Jul 2011 13:48:35 +0200 bulwahn making active configuration public in narrowing-based quickcheck
Mon, 18 Jul 2011 11:38:14 +0200 bulwahn declare tester in this quickcheck example
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn adding code equations for partial_term_of for rational numbers
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn adapting an experimental setup to changes in quickcheck's infrastructure
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn adding narrowing instances for real and rational
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn adapting quickcheck based on the analysis of the predicate compiler
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn adapting prolog-based tester
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn quickcheck does not deactivate testers if none are given
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn adapting mutabelle to latest changes in quickcheck; removing unused code in mutabelle
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn renaming quickcheck_tester to quickcheck_batch_tester; tuned
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn changing parser in quickcheck to activate and deactivate the testers
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn adapting SML_Quickcheck to new quickcheck infrastructure
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn enabling parallel execution of testers but removing more informative quickcheck output
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn changed every tester to have a configuration in quickcheck; enabling parallel testing of different testers in quickcheck
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn removing generator registration
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn parametrized test_term functions in quickcheck
Mon, 18 Jul 2011 10:34:21 +0200 bulwahn adding random, exhaustive and SML quickcheck as testers
Sun, 17 Jul 2011 22:25:14 +0200 haftmann more on complement
Sun, 17 Jul 2011 22:24:08 +0200 haftmann more on complement
Sun, 17 Jul 2011 20:57:56 +0200 haftmann more consistent theorem names
Sun, 17 Jul 2011 20:46:51 +0200 haftmann more lemmas about SUP
Sun, 17 Jul 2011 20:29:54 +0200 haftmann structuring duals together
Sun, 17 Jul 2011 20:23:39 +0200 haftmann merged
Sun, 17 Jul 2011 20:23:33 +0200 haftmann more lemmas about Sup
Sun, 17 Jul 2011 19:55:17 +0200 haftmann generalized INT_anti_mono
Sun, 17 Jul 2011 19:48:02 +0200 haftmann moving UNIV = ... equations to their proper theories
Sun, 17 Jul 2011 15:15:58 +0200 haftmann further generalization from sets to complete lattices
Sun, 17 Jul 2011 14:21:19 +0200 blanchet fixed lambda-liftg: must ensure the formulas are in close form
Sun, 17 Jul 2011 14:12:45 +0200 blanchet ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
Sun, 17 Jul 2011 14:11:35 +0200 blanchet pass kind to lambda-translation function
Sun, 17 Jul 2011 14:11:35 +0200 blanchet more refactoring of preprocessing
Sun, 17 Jul 2011 14:11:35 +0200 blanchet more refactoring of preprocessing, so as to be able to centralize it
Sun, 17 Jul 2011 14:11:35 +0200 blanchet renamed internal data structure
Sun, 17 Jul 2011 14:11:35 +0200 blanchet simplify code -- there are no lambdas in helpers anyway
Sun, 17 Jul 2011 14:11:35 +0200 blanchet added lambda-lifting to Sledgehammer (rough)
Sun, 17 Jul 2011 14:11:34 +0200 blanchet move more lambda-handling logic to Sledgehammer, from ATP module, for formal dependency reasons
Sun, 17 Jul 2011 08:45:06 +0200 haftmann merged
Sat, 16 Jul 2011 22:28:35 +0200 haftmann generalized some lemmas
Sat, 16 Jul 2011 22:04:02 +0200 haftmann consolidated bot and top classes, tuned notation
Sat, 16 Jul 2011 21:53:50 +0200 haftmann tuned notation
Sat, 16 Jul 2011 22:17:27 +0200 wenzelm clarified bash_output_fifo;
Sat, 16 Jul 2011 20:52:41 +0200 wenzelm moved bash operations to Isabelle_System (cf. Scala version);
Sat, 16 Jul 2011 20:14:58 +0200 wenzelm access to process output stream via auxiliary fifo;
Sat, 16 Jul 2011 18:41:35 +0200 wenzelm some file and directory operations;
Sat, 16 Jul 2011 18:20:02 +0200 wenzelm more general bash_process, which allows to terminate background processes as well;
Sat, 16 Jul 2011 18:11:14 +0200 wenzelm updated to Poly/ML SVN 1328, which is considered 5.4.2;
Sat, 16 Jul 2011 17:11:49 +0200 wenzelm added File.fold_pages for streaming of large files;
Sat, 16 Jul 2011 16:51:12 +0200 wenzelm tuned;
Sat, 16 Jul 2011 00:01:17 +0200 Cezary Kaliszyk HOL/Import: Fix errors with _mk_list
Fri, 15 Jul 2011 16:51:01 +0200 wenzelm Element.activate: leave check of binding where actually applied to the context -- allow internal qualifications, or non-identifier fact names like "assumes *: A" (see also 1183951365de);
Fri, 15 Jul 2011 14:07:12 +0200 wenzelm simplified malformed YXML markup -- special controls are visible in IsabelleText font;
Fri, 15 Jul 2011 13:29:00 +0200 wenzelm less ambitious ProofGeneral markup, which occasionally breaks plain-old regexps in elisp;
Fri, 15 Jul 2011 13:28:16 +0200 wenzelm more robust Binding.pretty/print in typical error sitations with spaces etc. (NB: markup can only provide *additional* emphasis and is occasionally suppressed in TTY mode or tooltips);
Fri, 15 Jul 2011 00:49:38 +0200 wenzelm more visible printing of empty binding;
Fri, 15 Jul 2011 00:03:47 +0200 wenzelm do not check vacous bindings, which routinely occur in locale expressions and long theorem statements etc.;
Thu, 14 Jul 2011 23:05:25 +0200 wenzelm more quotes;
Thu, 14 Jul 2011 22:53:43 +0200 wenzelm merged
Thu, 14 Jul 2011 22:08:11 +0200 krauss added missing dependencies;
Thu, 14 Jul 2011 19:43:45 +0200 haftmann merged
Thu, 14 Jul 2011 17:15:24 +0200 haftmann merged
Thu, 14 Jul 2011 17:14:54 +0200 haftmann tuned notation and proofs
Thu, 14 Jul 2011 17:29:30 +0200 blanchet move error logic closer to user
Thu, 14 Jul 2011 17:29:30 +0200 blanchet allow lambda-lifting without triggers
Thu, 14 Jul 2011 16:50:05 +0200 blanchet move lambda translation option from ATP to Sledgehammer, to avoid accidentally breaking Metis (its reconstruction code can only deal with combinators)
Thu, 14 Jul 2011 16:50:05 +0200 blanchet added option to control which lambda translation to use (for experiments)
Thu, 14 Jul 2011 15:14:38 +0200 blanchet fix subtle type inference bug in Metis -- different occurrences of the same Skolem might need to be typed differently, using paramify_vars overconstraints the typing problem
Thu, 14 Jul 2011 15:14:38 +0200 blanchet use monomorphic encoding as fallback, since they tend to produce fewer type errors
Thu, 14 Jul 2011 15:14:38 +0200 blanchet don't generate Waldmeister problems with only a conjecture, since it makes it crash sometimes
Thu, 14 Jul 2011 15:14:37 +0200 blanchet clearer unsound message
Thu, 14 Jul 2011 15:14:37 +0200 blanchet clarify fine soundness point
Thu, 14 Jul 2011 15:14:37 +0200 blanchet always unfold "Let"s is Sledgehammer, Metis, and MESON
Thu, 14 Jul 2011 15:14:37 +0200 blanchet unbreak Nitrox's parsing
Thu, 14 Jul 2011 00:21:56 +0200 haftmann merged
Thu, 14 Jul 2011 00:20:43 +0200 haftmann tuned lemma positions and proofs
Thu, 14 Jul 2011 00:16:41 +0200 haftmann tuned notation
Wed, 13 Jul 2011 23:49:56 +0200 haftmann uniqueness lemmas for bot and top
Wed, 13 Jul 2011 23:41:13 +0200 haftmann adjusted to tightened specification of classes bot and top
Wed, 13 Jul 2011 19:43:12 +0200 haftmann moved lemmas bot_less and less_top to classes bot and top respectively
Wed, 13 Jul 2011 19:40:18 +0200 haftmann tightened specification of classes bot and top: uniqueness of top and bot elements
Wed, 13 Jul 2011 22:16:19 +0200 blanchet honor the TPTP environment variable as the root of include relative paths -- that's a weird convention but without it Nitrox will fail at CASC
Wed, 13 Jul 2011 22:16:19 +0200 blanchet better temp name creation for Nitrox -- still very hackish though, but should get us through CASC-23 and CASC-J6
Wed, 13 Jul 2011 22:16:19 +0200 blanchet more exhaustive testing in Nitrox
Wed, 13 Jul 2011 22:16:19 +0200 blanchet no timeout for Nitrox
Wed, 13 Jul 2011 22:16:19 +0200 blanchet avoid relying on piping to "isabelle tty", because this gives errors on some Linuxes about the standard input not being a tty
Wed, 13 Jul 2011 22:16:19 +0200 blanchet added arithmetic decision procedure to CASC setup
Wed, 13 Jul 2011 22:16:19 +0200 blanchet added some arithmetic functions, for THF with arithmetic
Wed, 13 Jul 2011 22:16:19 +0200 blanchet pull in arithmetic theories
Wed, 13 Jul 2011 22:16:19 +0200 blanchet cleanly separate TPTP related files from other examples
Wed, 13 Jul 2011 21:59:54 +0200 bulwahn increasing timeout to avoid spurious failures
Wed, 13 Jul 2011 18:36:11 +0200 haftmann merged
Wed, 13 Jul 2011 07:26:31 +0200 haftmann more generalization towards complete lattices
Wed, 13 Jul 2011 15:50:45 +0200 krauss experimental variants of Library/Cset.thy and Library/Dlist_Cset.thy defined via quotient package
Wed, 13 Jul 2011 04:00:32 +0900 Cezary Kaliszyk merge
Wed, 13 Jul 2011 11:31:36 +0900 Cezary Kaliszyk Tuned
Thu, 14 Jul 2011 22:30:31 +0200 wenzelm more precise integer Markup.properties/XML.attributes: disallow ML-style ~ minus;
Wed, 13 Jul 2011 22:05:55 +0200 wenzelm added term_sharing.ML;
Wed, 13 Jul 2011 21:44:15 +0200 wenzelm recovered some runtime sharing from d6b6c74a8bcf, without the global memory bottleneck;
Wed, 13 Jul 2011 20:36:18 +0200 wenzelm sub-structural sharing after Syntax.check phase, with global interning of logical entities (the latter is relevant when bypassing default parsing via YXML);
Wed, 13 Jul 2011 20:13:27 +0200 wenzelm low-level tuning;
Wed, 13 Jul 2011 16:42:14 +0200 wenzelm Table.lookup_key and Graph.get_entry allow to retrieve the original key, which is not necessarily identical to the given one;
Wed, 13 Jul 2011 10:57:09 +0200 wenzelm XML.pretty with depth limit;
Tue, 12 Jul 2011 23:22:22 +0200 wenzelm more thorough Variable.check_name: Binding.check for logical entities within the term language;
Tue, 12 Jul 2011 23:20:34 +0200 wenzelm tuned;
Tue, 12 Jul 2011 20:53:14 +0200 wenzelm merged
Wed, 13 Jul 2011 00:43:07 +0900 Cezary Kaliszyk Update HOLLightCompat
Wed, 13 Jul 2011 00:29:33 +0900 Cezary Kaliszyk Update files generated in HOL/Import/HOLLight
Wed, 13 Jul 2011 00:23:24 +0900 Cezary Kaliszyk HOL/Import for HOLLight revival: Proper theory headers, update generation scripts to SVN version of HOL Light, add some constant maps and compatibility theorems
Tue, 12 Jul 2011 20:11:11 +0200 wenzelm ML pp for XML.tree;
Tue, 12 Jul 2011 20:11:00 +0200 wenzelm made SML/NJ happy;
Tue, 12 Jul 2011 19:49:35 +0200 wenzelm clarified YXML.detect;
Tue, 12 Jul 2011 19:47:40 +0200 wenzelm retain some terminology of "XML attributes";
Tue, 12 Jul 2011 19:36:46 +0200 wenzelm more uniform Properties in ML and Scala;
Tue, 12 Jul 2011 18:00:05 +0200 wenzelm more uniform Term and Term_XML modules;
Tue, 12 Jul 2011 17:53:06 +0200 wenzelm more compact representation of XML data (notably sort/typ/term), using properties as vector of atomic values;
Tue, 12 Jul 2011 15:32:16 +0200 wenzelm tuned signature -- less cryptic ASCII names;
Tue, 12 Jul 2011 15:17:37 +0200 wenzelm discontinued obsolete Isabelle_Syntax and Parse_Value -- superseded by Outer_Syntax.quote_string and XML.Encode, Term_XML.Encode etc.;
Tue, 12 Jul 2011 15:12:50 +0200 wenzelm added Parse.properties (again) -- allow empty list like Parse_Value.properties but unlike Parse.properties of ef86de9c98aa;
Tue, 12 Jul 2011 14:54:29 +0200 wenzelm added Outer_Syntax.quote_string, which is conceptually a bit different from Token.unparse;
Tue, 12 Jul 2011 14:33:08 +0200 wenzelm more precise Symbol_Pos.quote_string;
Tue, 12 Jul 2011 13:45:05 +0200 wenzelm clarified YXML.embed_controls -- this is idempotent and cannot be nested;
Tue, 12 Jul 2011 13:39:29 +0200 wenzelm allow empty body for raw_message -- important for Invoke_Scala;
Tue, 12 Jul 2011 11:45:13 +0200 wenzelm Isabelle string syntax allows literal control characters;
Tue, 12 Jul 2011 11:19:42 +0200 wenzelm glyphs from DejaVu for ASCII control characters 5, 6, 7, 127, which have a special meaning in Isabelle or Poly/ML;
Tue, 12 Jul 2011 11:16:56 +0200 wenzelm more precise exceptions;
Tue, 12 Jul 2011 10:44:30 +0200 wenzelm tuned XML modules;
Tue, 12 Jul 2011 16:00:05 +0900 Cezary Kaliszyk Quotient example: Lists with distinct elements
Mon, 11 Jul 2011 23:20:40 +0200 wenzelm merged
Mon, 11 Jul 2011 18:44:58 +0200 haftmann explicit code equation for equality
Mon, 11 Jul 2011 23:15:27 +0200 wenzelm tuned error messages;
Mon, 11 Jul 2011 23:15:04 +0200 wenzelm tuned;
Mon, 11 Jul 2011 22:55:47 +0200 wenzelm tuned signature -- corresponding to Scala version;
Mon, 11 Jul 2011 22:50:29 +0200 wenzelm made SML/NJ happy;
Mon, 11 Jul 2011 22:19:11 +0200 wenzelm more uniform padded_markup, which is important for caret visibility despite absence of markup;
Mon, 11 Jul 2011 17:22:31 +0200 wenzelm merged
Mon, 11 Jul 2011 07:04:30 +0200 haftmann merged
Sun, 10 Jul 2011 22:42:53 +0200 haftmann tuned proofs
Sun, 10 Jul 2011 22:17:33 +0200 haftmann tuned notation
Sun, 10 Jul 2011 22:11:32 +0200 haftmann tuned notation
Sun, 10 Jul 2011 21:56:39 +0200 haftmann tuned notation
Mon, 11 Jul 2011 17:22:15 +0200 wenzelm NEWS;
Mon, 11 Jul 2011 17:14:30 +0200 wenzelm proper InvocationTargetException.getCause for indirect exceptions;
Mon, 11 Jul 2011 17:11:54 +0200 wenzelm tuned error message;
Mon, 11 Jul 2011 17:10:32 +0200 wenzelm tuned signature;
Mon, 11 Jul 2011 16:48:02 +0200 wenzelm JVM method invocation service via Scala layer;
Mon, 11 Jul 2011 15:56:30 +0200 wenzelm tuned signature;
Mon, 11 Jul 2011 11:13:33 +0200 wenzelm some support for raw messages, which bypass standard Symbol/YXML decoding;
Mon, 11 Jul 2011 10:27:50 +0200 wenzelm tuned XML.Cache parameters;
Sun, 10 Jul 2011 23:46:05 +0200 wenzelm some support to invoke Scala methods under program control;
Sun, 10 Jul 2011 21:46:41 +0200 wenzelm merged;
Sun, 10 Jul 2011 21:39:03 +0200 haftmann merged
Sun, 10 Jul 2011 15:45:35 +0200 haftmann tuned proofs and notation
Sun, 10 Jul 2011 14:26:07 +0200 haftmann more succinct proofs
Sun, 10 Jul 2011 14:14:19 +0200 haftmann more succinct proofs
Sun, 10 Jul 2011 19:33:27 +0200 bulwahn adding a very liberal timeout for values after a test case failed due to the restricted timeout
Sun, 10 Jul 2011 14:02:27 +0200 bulwahn improved NEWS
Sat, 09 Jul 2011 21:18:20 +0200 bulwahn NEWS
Sat, 09 Jul 2011 21:09:09 +0200 bulwahn standardized String.concat towards implode (cf. c37a1f29bbc0)
Sat, 09 Jul 2011 19:29:25 +0200 bulwahn adding quickcheck examples for evaluating floor and ceiling functions
Sat, 09 Jul 2011 19:28:33 +0200 bulwahn adding code equations to execute floor and ceiling on rational and real numbers
Sat, 09 Jul 2011 13:41:58 +0200 bulwahn adding a floor_ceiling type class for different instantiations of floor (changeset from Brian Huffman)
Sun, 10 Jul 2011 20:59:04 +0200 wenzelm inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
Sun, 10 Jul 2011 17:58:11 +0200 wenzelm lambda terms with XML data representation in Scala;
Sun, 10 Jul 2011 16:34:17 +0200 wenzelm XML data representation of lambda terms;
Sun, 10 Jul 2011 16:31:04 +0200 wenzelm YXML.string_of_body convenience;
Sun, 10 Jul 2011 16:13:37 +0200 wenzelm made SML/NJ happy;
Sun, 10 Jul 2011 16:09:08 +0200 wenzelm tuned signature;
Sun, 10 Jul 2011 15:48:15 +0200 wenzelm more abstract signature;
Sun, 10 Jul 2011 13:51:21 +0200 wenzelm simplified XML_Data;
Sun, 10 Jul 2011 13:00:22 +0200 wenzelm less currying in Scala;
Sun, 10 Jul 2011 00:21:19 +0200 wenzelm propagate header changes to prover process;
Sat, 09 Jul 2011 21:53:27 +0200 wenzelm echo prover input via raw_messages, for improved protocol tracing;
Sat, 09 Jul 2011 18:54:50 +0200 wenzelm tuned;
Sat, 09 Jul 2011 18:35:00 +0200 wenzelm tuned signature;
Sat, 09 Jul 2011 18:15:23 +0200 wenzelm clarified propagation of node name and header;
Sat, 09 Jul 2011 17:14:08 +0200 wenzelm more precise treatment of prover definedness;
Sat, 09 Jul 2011 16:53:19 +0200 wenzelm tuned source structure;
Sat, 09 Jul 2011 13:29:33 +0200 wenzelm some support for blobs (arbitrary text files) within document nodes;
Sat, 09 Jul 2011 12:56:51 +0200 wenzelm tuned signature;
Fri, 08 Jul 2011 22:00:53 +0200 wenzelm moved global state to structure Document (again);
Fri, 08 Jul 2011 21:44:47 +0200 wenzelm moved Outer_Syntax.load_thy to Thy_Load.load_thy;
Fri, 08 Jul 2011 20:27:09 +0200 wenzelm less stateful outer_syntax;
Fri, 08 Jul 2011 17:04:38 +0200 wenzelm discontinued odd Position.column -- left-over from attempts at PGIP implementation;
Fri, 08 Jul 2011 16:13:34 +0200 wenzelm discontinued special treatment of hard tabulators;
Fri, 08 Jul 2011 16:01:14 +0200 wenzelm eliminated hard tabs;
Fri, 08 Jul 2011 15:18:28 +0200 wenzelm merged
Fri, 08 Jul 2011 12:18:46 +0200 nipkow merged
Thu, 07 Jul 2011 21:53:53 +0200 nipkow added translation to fix critical pair between abbreviations for surj and ~=
Thu, 07 Jul 2011 23:33:14 +0200 bulwahn floor and ceiling definitions are not code equations -- this enables trivial evaluation of floor and ceiling
Fri, 08 Jul 2011 15:17:40 +0200 wenzelm standardized String.concat towards implode;
Fri, 08 Jul 2011 14:37:19 +0200 wenzelm more abstract Thy_Load.load_file/use_file for external theory resources;
Fri, 08 Jul 2011 13:59:54 +0200 wenzelm comment;
Fri, 08 Jul 2011 11:50:58 +0200 wenzelm clarified Thy_Load.digest_file -- read ML files only once;
Fri, 08 Jul 2011 11:13:21 +0200 wenzelm tuned signature;
Thu, 07 Jul 2011 23:55:15 +0200 wenzelm simplified make_option/dest_option;
Thu, 07 Jul 2011 22:04:30 +0200 wenzelm explicit Document.Node.Header, with master_dir and thy_name;
Thu, 07 Jul 2011 14:10:50 +0200 wenzelm explicit indication of type Symbol.Symbol;
Thu, 07 Jul 2011 13:48:30 +0200 wenzelm simplified Symbol based on lazy Symbol.Interpretation -- reduced odd "functorial style";
Wed, 06 Jul 2011 23:11:59 +0200 wenzelm merged
Wed, 06 Jul 2011 17:19:34 +0100 blanchet make SML/NJ happier
Wed, 06 Jul 2011 17:19:34 +0100 blanchet make SML/NJ happy + tuning
Wed, 06 Jul 2011 17:19:34 +0100 blanchet moved ATP dependencies to HOL-Plain, where they belong
Wed, 06 Jul 2011 17:19:34 +0100 blanchet better setup for experimental "z3_atp"
Wed, 06 Jul 2011 17:58:03 +0200 krauss 64bit versions of some mira configurations
Wed, 06 Jul 2011 17:56:58 +0200 krauss removed unused mira configuration
Wed, 06 Jul 2011 13:57:52 +0200 bulwahn merged
Wed, 06 Jul 2011 13:52:42 +0200 bulwahn tuning options to avoid spurious isabelle test failures
Wed, 06 Jul 2011 22:02:52 +0200 wenzelm clarified record syntax: fieldext excludes the "more" pseudo-field (unlike 2f885b7e5ba7), so that errors like (| x = a, more = b |) are reported less confusingly;
Wed, 06 Jul 2011 20:46:06 +0200 wenzelm prefer Synchronized.var;
Wed, 06 Jul 2011 20:14:13 +0200 wenzelm tuned errors;
Wed, 06 Jul 2011 13:31:12 +0200 wenzelm record package: proper configuration options;
Wed, 06 Jul 2011 11:37:29 +0200 wenzelm just one copy of split_args;
Wed, 06 Jul 2011 09:54:40 +0200 wenzelm merged
Tue, 05 Jul 2011 19:11:29 +0200 hoelzl rename lemma Infinite_Product_Measure.sigma_sets_subseteq, it hides Sigma_Algebra.sigma_sets_subseteq
Tue, 05 Jul 2011 17:09:59 +0100 nik improved translation of lambdas in THF
Tue, 05 Jul 2011 17:09:59 +0100 nik added generation of lambdas in THF
Tue, 05 Jul 2011 17:09:59 +0100 nik add support for lambdas in TPTP THF generator + killed an unsound type encoding (because the monotonicity calculus assumes first-order)
Tue, 05 Jul 2011 23:18:14 +0200 wenzelm simplified Symbol.iterator: produce strings, which are mostly preallocated;
Tue, 05 Jul 2011 22:43:18 +0200 wenzelm tuned comment (cf. e9f26e66692d);
Tue, 05 Jul 2011 22:39:15 +0200 wenzelm Thy_Info.dependencies: ignore already loaded theories, according to initial prover session status;
Tue, 05 Jul 2011 22:38:44 +0200 wenzelm theory name needs to conform to Path syntax;
Tue, 05 Jul 2011 21:53:59 +0200 wenzelm hard-wired print mode "xsymbols" increases chance that "iff" in HOL will print symbolic arrow;
Tue, 05 Jul 2011 21:32:48 +0200 wenzelm prefer space_explode/split_lines as in Isabelle/ML;
Tue, 05 Jul 2011 21:20:24 +0200 wenzelm Path.split convenience;
Tue, 05 Jul 2011 20:36:49 +0200 wenzelm get theory from last executation state;
Tue, 05 Jul 2011 19:45:59 +0200 wenzelm explicit exit_transaction with Theory.end_theory (which could include sanity checks as in HOL-SPARK for example);
Tue, 05 Jul 2011 11:45:48 +0200 wenzelm clarified cancel_execution/await_cancellation;
Tue, 05 Jul 2011 11:16:37 +0200 wenzelm tuned signature;
Tue, 05 Jul 2011 10:54:05 +0200 wenzelm tuned;
Tue, 05 Jul 2011 09:54:39 +0200 krauss re-check to explicitly propagate a given type constraint to lhs -- necessary to trigger type improvement in an instantiation target
Mon, 04 Jul 2011 22:25:33 +0200 wenzelm Document.no_id/new_id as in ML (new_id *could* be session-specific but it isn't right now);
Mon, 04 Jul 2011 22:11:32 +0200 wenzelm quasi-static Isabelle_System -- reduced tendency towards "functorial style";
Mon, 04 Jul 2011 20:18:19 +0200 wenzelm explicit class Counter;
Mon, 04 Jul 2011 16:54:58 +0200 wenzelm merged
Mon, 04 Jul 2011 10:23:46 +0200 hoelzl the borel probability measure is easier to handle with {0 ..< 1} (coverable by disjoint intervals {_ ..< _})
Mon, 04 Jul 2011 10:15:49 +0200 hoelzl equalities of subsets of atLeastLessThan
Sun, 03 Jul 2011 09:59:25 +0200 bulwahn adding documentation of the value antiquotation to the code generation manual
Sun, 03 Jul 2011 08:15:14 +0200 blanchet make SML/NJ happy
Sat, 02 Jul 2011 22:55:58 +0200 haftmann install case certificate for If after code_datatype declaration for bool
Sat, 02 Jul 2011 22:14:47 +0200 haftmann tuned typo
Mon, 04 Jul 2011 16:51:45 +0200 wenzelm pervasive Basic_Library in Scala;
Mon, 04 Jul 2011 16:27:11 +0200 wenzelm some support for theory files within Isabelle/Scala session;
Mon, 04 Jul 2011 13:43:10 +0200 wenzelm imitate exception ERROR of Isabelle/ML;
Sun, 03 Jul 2011 19:53:35 +0200 wenzelm eliminated null;
Sun, 03 Jul 2011 19:42:32 +0200 wenzelm more explicit edit_node vs. init_node;
Sun, 03 Jul 2011 15:10:17 +0200 wenzelm tuned signature;
Sat, 02 Jul 2011 23:31:07 +0200 wenzelm Thy_Header.read convenience;
Sat, 02 Jul 2011 23:04:19 +0200 wenzelm some support for Session.File_Store;
Sat, 02 Jul 2011 21:24:19 +0200 wenzelm tuned signature;
Sat, 02 Jul 2011 20:54:38 +0200 wenzelm eliminated redundant session_ready;
Sat, 02 Jul 2011 20:22:02 +0200 wenzelm tuned;
Sat, 02 Jul 2011 19:22:06 +0200 wenzelm uniform finish_thy -- always Global_Theory.join_proofs, even with sequential scheduling;
Sat, 02 Jul 2011 19:08:51 +0200 wenzelm misc tuning;
Sat, 02 Jul 2011 10:37:35 +0200 haftmann correction: do not assume that case const index covered all cases
Fri, 01 Jul 2011 23:31:23 +0200 haftmann remove illegal case combinators after merge
Fri, 01 Jul 2011 23:10:27 +0200 haftmann corrected misunderstanding what `old functions` are supposed to be
Fri, 01 Jul 2011 23:07:06 +0200 haftmann centralized deletion of equations for constructors; corrected misunderstanding what `old functions` are supposed to be
Fri, 01 Jul 2011 22:48:05 +0200 haftmann merged
Fri, 01 Jul 2011 19:57:41 +0200 haftmann index cases for constructors
Fri, 01 Jul 2011 19:42:07 +0200 noschinl cover induct's "arbitrary" more deeply
Fri, 01 Jul 2011 18:11:17 +0200 wenzelm merged;
Fri, 01 Jul 2011 17:44:04 +0200 blanchet enforce hard timeout on ATPs (esp. "z3_atp" on Linux) + remove obsolete failure codes
Fri, 01 Jul 2011 16:31:33 +0200 blanchet made minimizer informative output accurate
Fri, 01 Jul 2011 15:53:38 +0200 blanchet test a few more type encodings
Fri, 01 Jul 2011 15:53:38 +0200 blanchet further repair "mangled_tags", now that tags are also mangled
Fri, 01 Jul 2011 15:53:38 +0200 blanchet update documentation after "type_enc" renaming + fixed a few other out-of-date factlets
Fri, 01 Jul 2011 15:53:38 +0200 blanchet renamed "type_sys" to "type_enc", which is more accurate
Fri, 01 Jul 2011 15:53:37 +0200 blanchet document "simple_higher" type encoding
Fri, 01 Jul 2011 15:53:37 +0200 blanchet cleaner handling of higher-order simple types, so that it's also possible to use first-order simple types with LEO-II and company
Fri, 01 Jul 2011 15:53:37 +0200 blanchet mangle "ti" tags
Fri, 01 Jul 2011 15:53:37 +0200 blanchet tuning
Fri, 01 Jul 2011 17:36:25 +0200 wenzelm clarified Thy_Syntax.element;
Fri, 01 Jul 2011 16:05:38 +0200 wenzelm tuned layout;
Fri, 01 Jul 2011 15:16:03 +0200 wenzelm proper @{binding} antiquotations (relevant for formal references);
Fri, 01 Jul 2011 15:14:44 +0200 wenzelm tuned;
Fri, 01 Jul 2011 14:17:02 +0200 wenzelm merged
Fri, 01 Jul 2011 13:54:25 +0200 noschinl reverted 782991e4180d: fold_fields was never used
Fri, 01 Jul 2011 13:54:23 +0200 noschinl reverted ce00462f,b3759dce, 7a165592: unwanted generalisation
Fri, 01 Jul 2011 11:26:02 +0200 bulwahn improving actual dependencies
Fri, 01 Jul 2011 10:45:51 +0200 bulwahn adding a minimalistic documentation of the value antiquotation in the Isar reference manual
Fri, 01 Jul 2011 10:45:49 +0200 bulwahn adding a value antiquotation
Thu, 30 Jun 2011 19:24:09 +0200 wenzelm more general theory header parsing;
Thu, 30 Jun 2011 16:50:26 +0200 wenzelm back to sequential merge_data, reverting 741373421318 (NB: expensive Parser.merge_gram is already asynchronous since 3daff3cc2214);
Thu, 30 Jun 2011 16:07:30 +0200 wenzelm merged
Thu, 30 Jun 2011 10:15:46 +0200 krauss parse term in auxiliary context augmented with variable;
Wed, 29 Jun 2011 11:58:35 +0200 boehmes linarith counterexamples now provide only valuations for variables (which should restrict the number of linarith trace messages);
Thu, 30 Jun 2011 14:55:01 +0200 wenzelm prefer Isabelle path algebra;
Thu, 30 Jun 2011 14:51:32 +0200 wenzelm proper fold order;
Thu, 30 Jun 2011 14:03:31 +0200 wenzelm more Path operations;
Thu, 30 Jun 2011 13:59:55 +0200 wenzelm getenv_strict in ML;
Thu, 30 Jun 2011 13:21:41 +0200 wenzelm standardized use of Path operations;
Thu, 30 Jun 2011 11:15:36 +0200 wenzelm tuned comments;
Thu, 30 Jun 2011 00:09:57 +0200 wenzelm abstract algebra of file paths in Scala (cf. path.ML);
Thu, 30 Jun 2011 00:01:00 +0200 wenzelm proper Path.print;
Wed, 29 Jun 2011 23:43:48 +0200 wenzelm basic operations on lists and strings;
Wed, 29 Jun 2011 21:34:16 +0200 wenzelm tuned signature;
Wed, 29 Jun 2011 20:39:41 +0200 wenzelm simplified/unified Simplifier.mk_solver;
Wed, 29 Jun 2011 18:12:34 +0200 wenzelm modernized some simproc setup;
Wed, 29 Jun 2011 17:35:46 +0200 wenzelm modernized some simproc setup;
Wed, 29 Jun 2011 16:31:50 +0200 wenzelm print Path.T with some markup;
Wed, 29 Jun 2011 15:23:36 +0200 wenzelm HTML: render control symbols more like Isabelle/Scala/jEdit;
Tue, 28 Jun 2011 10:52:15 +0200 traytel collapse map functions with identity subcoercions to identities;
Tue, 28 Jun 2011 21:06:59 +0200 blanchet reenabled accidentally-disabled automatic minimization
Tue, 28 Jun 2011 20:42:29 +0200 wenzelm tuned markup;
Tue, 28 Jun 2011 17:13:32 +0100 paulson merged
Tue, 28 Jun 2011 17:12:50 +0100 paulson tidied messy proofs
Tue, 28 Jun 2011 16:43:44 +0200 bulwahn merged
Tue, 28 Jun 2011 14:36:43 +0200 bulwahn adding timeout to quickcheck narrowing
Tue, 28 Jun 2011 14:52:46 +0100 paulson simplified proofs using metis calls
Tue, 28 Jun 2011 12:48:00 +0100 paulson merged
Tue, 28 Jun 2011 12:47:32 +0100 paulson keyfree: The set of key-free messages (and associated theorems)
Mon, 27 Jun 2011 22:44:44 +0200 wenzelm merged
Mon, 27 Jun 2011 17:04:04 +0200 krauss new Datatype.info_of_constr with strict behaviour wrt. to overloaded constructors -- side effect: function package correctly identifies 0::int as a non-constructor;
Mon, 27 Jun 2011 14:56:39 +0200 blanchet added reference for MESON
Mon, 27 Jun 2011 14:56:37 +0200 blanchet document "meson" and "metis" in HOL specific section of the Isar ref manual
Mon, 27 Jun 2011 14:56:35 +0200 blanchet clarify minimizer output
Mon, 27 Jun 2011 14:56:33 +0200 blanchet don't export any metastrange or other nonatomizable formulas, since these don't help proving normal things, they are somewhat broken in the ATP output, and they are atypical
Mon, 27 Jun 2011 14:56:32 +0200 blanchet tweaked comment
Mon, 27 Jun 2011 14:56:31 +0200 blanchet document "sound" option
Mon, 27 Jun 2011 14:56:29 +0200 blanchet minor Sledgehammer news
Mon, 27 Jun 2011 14:56:28 +0200 blanchet added "sound" option to force Sledgehammer to be pedantically sound
Mon, 27 Jun 2011 14:56:26 +0200 blanchet removed "full_types" option from documentation
Mon, 27 Jun 2011 14:56:10 +0200 blanchet document changes to Sledgehammer and "try"
Mon, 27 Jun 2011 13:52:47 +0200 blanchet removed "full_types" option from Sledgehammer, now that virtually sound encodings are used as the default anyway
Mon, 27 Jun 2011 13:52:47 +0200 blanchet clarify warning message to avoid confusing beginners
Mon, 27 Jun 2011 13:52:47 +0200 blanchet remove experimental trimming feature -- it slowed down things on Linux for some reason
Mon, 27 Jun 2011 13:52:47 +0200 blanchet filter out some tautologies using an ATP, especially for those theories that are known for producing such things
Mon, 27 Jun 2011 22:23:44 +0200 wenzelm NEWS;
Mon, 27 Jun 2011 22:20:49 +0200 wenzelm document antiquotations are managed as theory data, with proper name space and entity markup;
Mon, 27 Jun 2011 17:51:28 +0200 wenzelm proper checking of @{ML_antiquotation};
Mon, 27 Jun 2011 17:20:24 +0200 wenzelm hide rather short auxiliary names, which can easily occur in user theories;
Mon, 27 Jun 2011 17:06:06 +0200 wenzelm updated generated file;
Mon, 27 Jun 2011 16:53:31 +0200 wenzelm ML antiquotations are managed as theory data, with proper name space and entity markup;
Mon, 27 Jun 2011 15:03:55 +0200 wenzelm old gensym is now legacy -- global state is out of fashion, and its result is not guaranteed to be fresh;
Mon, 27 Jun 2011 15:01:08 +0200 wenzelm parallel Syntax.parse, which is rather slow;
Mon, 27 Jun 2011 14:38:58 +0200 wenzelm markup binding like class, which is the only special markup where Proof General (including version 4.1) allows "isar-long-id-stuff";
Mon, 27 Jun 2011 09:42:46 +0200 hoelzl move conditional expectation to its own theory file
Sun, 26 Jun 2011 19:10:03 +0200 boehmes updated SMT certificates
Sun, 26 Jun 2011 19:10:02 +0200 boehmes generalized introduction of explicit application constant: consider more functions as possible witness/instance of quantifiers than before (a constant of type T1 -> T2 -> T3 should be considered to have a rank less or equal to 1 if variables of type T2 -> T3 occur bound in a problem);
Sat, 25 Jun 2011 20:03:07 +0200 wenzelm proper tokens only if session is ready;
Sat, 25 Jun 2011 19:38:35 +0200 wenzelm entity markup for "type", "constant";
Sat, 25 Jun 2011 19:19:13 +0200 wenzelm clarified Markup.CLASS vs. HTML.CLASS;
Sat, 25 Jun 2011 18:29:51 +0200 wenzelm tuned color, to avoid confusion with type variables;
Sat, 25 Jun 2011 18:24:52 +0200 wenzelm discontinued generic XML markup -- this is for XHTML with <span/> elements;
Sat, 25 Jun 2011 18:15:36 +0200 wenzelm type classes: entity markup instead of old-style token markup;
Sat, 25 Jun 2011 17:17:49 +0200 wenzelm clarified Binding.pretty/print: no quotes, only markup -- Binding.str_of is rendered obsolete;
Sat, 25 Jun 2011 15:08:58 +0200 wenzelm clarified Binding.str_of/print: show full prefix + qualifier, which is relevant for print_locale, for example;
Sat, 25 Jun 2011 15:02:12 +0200 wenzelm produce string constant directly;
Sat, 25 Jun 2011 14:28:43 +0200 wenzelm merged
Sat, 25 Jun 2011 12:19:54 +0200 ballarin While reading equations of an interpretation, already allow syntax provided by the interpretation base.
Sat, 25 Jun 2011 14:25:10 +0200 wenzelm removed very slow proof of unnamed/unused theorem from HOL/Quickcheck_Narrowing.thy (cf. 2dee03f192b7) -- can take seconds for main HOL and minutes for HOL-Proofs;
Sat, 25 Jun 2011 12:57:46 +0200 wenzelm clarified java.ext.dirs: putting Isabelle extensions first makes it work miraculously even on Cygwin with Java in "C:\Program Files\..." (with spaces in file name);
Sat, 25 Jun 2011 12:54:32 +0200 wenzelm CLASSPATH already converted in isabelle java wrapper;
Sat, 25 Jun 2011 11:51:50 +0200 wenzelm removed unused/broken Isabelle.exe for now -- needs update of Admin/launch4j;
Thu, 23 Jun 2011 23:12:00 +0200 wenzelm more robust join_results: join_work needs to be uninterruptible, otherwise the task being dequeued by join_next might be never executed/finished!
Thu, 23 Jun 2011 23:05:38 +0200 wenzelm clarified EXCEPTIONS [] (cf. Exn.is_interrupt and Runtime.exn_message);
Thu, 23 Jun 2011 20:30:48 +0200 wenzelm more robust concurrent builds;
Thu, 23 Jun 2011 10:08:35 -0700 huffman merged
Thu, 23 Jun 2011 10:07:16 -0700 huffman add countable_datatype method for proving countable class instances
Thu, 23 Jun 2011 18:32:13 +0200 wenzelm merged;
Thu, 23 Jun 2011 09:16:48 -0700 huffman instance inat :: number_semiring
Thu, 23 Jun 2011 09:04:20 -0700 huffman added number_semiring class, plus a few new lemmas;
Thu, 23 Jun 2011 16:31:20 +0200 blanchet merged
Thu, 23 Jun 2011 11:19:41 +0200 blanchet fiddle with remote ATP settings, based on Judgment Day
Thu, 23 Jun 2011 11:19:41 +0200 blanchet give slightly more time to server to respond, to avoid leaving too much garbage on Geoff's servers
Thu, 23 Jun 2011 12:02:54 +0200 ballarin Release notes should be written from the user's perspective. Don't assume the user has universal knowledge of the system.
Wed, 22 Jun 2011 15:58:55 -0700 huffman generalize lemmas power_number_of_even and power_number_of_odd
Wed, 22 Jun 2011 13:45:32 -0700 huffman merged
Wed, 22 Jun 2011 13:30:28 -0700 huffman add HOLCF/ex/Concurrency_Monad.thy, which contains resumption/state/powerdomain monad example from my PhD thesis
Thu, 23 Jun 2011 17:17:40 +0200 wenzelm simplified arrangement of jars;
Thu, 23 Jun 2011 16:34:29 +0200 wenzelm adapted to Cygwin;
Thu, 23 Jun 2011 16:10:22 +0200 wenzelm provide Isabelle/Scala environment as Java extension, instead of user classpath
Thu, 23 Jun 2011 14:52:32 +0200 wenzelm explicit import java.lang.System to prevent odd scope problems;
Thu, 23 Jun 2011 14:48:32 +0200 wenzelm ensure export of initial CLASSPATH;
Thu, 23 Jun 2011 13:23:00 +0200 wenzelm augment Java extension directories;
Thu, 23 Jun 2011 10:58:29 +0200 wenzelm basic setup for Isabelle charset;
Wed, 22 Jun 2011 23:56:44 +0200 wenzelm prefer actual charset over charset name;
Wed, 22 Jun 2011 21:54:35 +0200 wenzelm clarified default ML settings;
Wed, 22 Jun 2011 21:35:48 +0200 wenzelm lazy Isabelle_System.default supports implicit boot;
Wed, 22 Jun 2011 21:27:20 +0200 wenzelm clarified plugin start/stop;
Wed, 22 Jun 2011 20:56:18 +0200 wenzelm clarified init/exit procedure;
Wed, 22 Jun 2011 20:38:03 +0200 wenzelm clarified decoded control symbols;
Wed, 22 Jun 2011 20:25:35 +0200 wenzelm init/exit model/view synchronously within the swing thread -- EditBus.send in jedit-4.4.1 always runs there;
Wed, 22 Jun 2011 20:21:22 +0200 wenzelm prefer STIXGeneral -- hard to tell if better or worse;
Wed, 22 Jun 2011 16:35:31 +0200 wenzelm merged
Wed, 22 Jun 2011 15:07:03 +0200 boehmes export lambda-lifting code as there is potential use for it within Sledgehammer
Wed, 22 Jun 2011 16:32:36 +0200 wenzelm updated to jedit-4.4.1 and jedit_build-20110622;
Wed, 22 Jun 2011 16:01:30 +0200 wenzelm clarified chunk.offset, chunk.length;
Tue, 21 Jun 2011 23:08:16 +0200 wenzelm avoid fractional font metrics, which makes rendering really ugly (e.g. on Linux);
Tue, 21 Jun 2011 22:40:30 +0200 wenzelm some arrow symbols from DejaVuSansMono for bsub/esub/bsup/esup;
Tue, 21 Jun 2011 21:34:36 +0200 wenzelm more precise font transformations: shift sub/superscript, adjust size for user fonts;
Tue, 21 Jun 2011 17:17:39 +0200 blanchet don't change the way helpers are generated for the exporter's sake
Tue, 21 Jun 2011 17:17:39 +0200 blanchet provide appropriate type system and number of fact defaults for remote ATPs
Tue, 21 Jun 2011 17:17:39 +0200 blanchet order generated facts topologically
Tue, 21 Jun 2011 17:17:39 +0200 blanchet peel off two or more layers in exceptional cases where the proof term refers to the proved theorems twice with the same name (e.g., "Transitive_Closure.trancl_into_trancl")
Tue, 21 Jun 2011 17:17:39 +0200 blanchet tweaked E, SPASS, Vampire setup based on latest Judgment Day results
Tue, 21 Jun 2011 17:17:39 +0200 blanchet remove historical bloat -- another benefit of merging Metis's and Sledgehammer's translations
Tue, 21 Jun 2011 17:17:39 +0200 blanchet avoid double ASCII-fication
Tue, 21 Jun 2011 17:17:39 +0200 blanchet make sure that enough type information is generated -- because the exported "lemma"s are also used as "conjecture", we can't optimize type information based on polarity
Tue, 21 Jun 2011 17:17:39 +0200 blanchet generate type predicates for existentials/skolems, otherwise some problems might not be provable
Tue, 21 Jun 2011 17:17:38 +0200 blanchet insert rather than append special facts to make it less likely that they're truncated away
Tue, 21 Jun 2011 15:43:27 +0200 wenzelm hidden font: full height makes cursor more visible;
Tue, 21 Jun 2011 14:12:49 +0200 wenzelm more uniform treatment of recode_set/recode_map;
Tue, 21 Jun 2011 13:29:44 +0200 wenzelm tuned iteration over short symbols;
Tue, 21 Jun 2011 12:53:55 +0200 wenzelm Symbol.is_ctrl: handle decoded version as well;
Tue, 21 Jun 2011 01:08:15 +0200 wenzelm some support for user symbol fonts;
Mon, 20 Jun 2011 23:25:39 +0200 wenzelm removed obsolete font specification;
Mon, 20 Jun 2011 23:21:24 +0200 wenzelm more tolerant Symbol.decode;
Mon, 20 Jun 2011 23:19:38 +0200 wenzelm simplified/generalized ISABELLE_FONTS handling;
Mon, 20 Jun 2011 22:48:41 +0200 wenzelm updated to jedit_build-20110620;
Mon, 20 Jun 2011 22:43:56 +0200 wenzelm added SyntaxUtilities.StyleExtender hook, with actual functionality in Isabelle/Scala;
Mon, 20 Jun 2011 12:13:43 +0200 blanchet clean up SPASS FLOTTER hack
Mon, 20 Jun 2011 11:42:41 +0200 blanchet remove automatic recovery from (some) unsound proofs, now that we use sound encodings for all the interesting provers
Mon, 20 Jun 2011 10:41:02 +0200 blanchet only refer to facts found in TPTP file -- e.g. facts that simplify to true are excluded
Mon, 20 Jun 2011 10:41:02 +0200 blanchet slightly better setup for E
Mon, 20 Jun 2011 10:41:02 +0200 blanchet respect "really_all" argument, which is used by "ATP_Export"
Mon, 20 Jun 2011 10:41:02 +0200 blanchet slightly better setup for SPASS and Vampire as more results have come in
Mon, 20 Jun 2011 10:41:02 +0200 blanchet optimized SPASS and Vampire time slices, like E before
Mon, 20 Jun 2011 10:41:02 +0200 blanchet optimized E's time slicing, based on latest exhaustive Judgment Day results
Mon, 20 Jun 2011 10:41:02 +0200 blanchet deal with ATP time slices in a more flexible/robust fashion
Mon, 20 Jun 2011 09:19:31 +0200 wenzelm literal unicode in README.html allows to copy/paste from Lobo output;
Sun, 19 Jun 2011 22:53:37 +0200 wenzelm merged;
Sun, 19 Jun 2011 22:53:15 +0200 wenzelm explain special control symbols;
Sun, 19 Jun 2011 22:52:49 +0200 wenzelm accept control symbols;
Sun, 19 Jun 2011 18:12:49 +0200 blanchet fixed silly ATP exporter bug: if the proof of lemma A relies on B and C, and the proof of B relies on C, return {B, C}, not {B}, as the set of dependencies
Sun, 19 Jun 2011 18:12:49 +0200 blanchet recognize one more E failure message
Sun, 19 Jun 2011 18:12:49 +0200 blanchet tweaked TPTP formula kind for typing information used in the conjecture
Sun, 19 Jun 2011 18:12:49 +0200 blanchet more forceful message
Sun, 19 Jun 2011 21:53:04 +0200 wenzelm treat quotes as non-controllable, to reduce surprise in incremental editing;
Sun, 19 Jun 2011 21:47:14 +0200 wenzelm abbreviations for special control symbols;
Sun, 19 Jun 2011 21:43:41 +0200 wenzelm completion for control symbols;
Sun, 19 Jun 2011 21:38:48 +0200 wenzelm updated to jedit_build-20110619;
Sun, 19 Jun 2011 21:34:55 +0200 wenzelm support for bold style within text buffer;
Sun, 19 Jun 2011 15:31:16 +0200 wenzelm tuned;
Sun, 19 Jun 2011 15:22:58 +0200 wenzelm discontinued special treatment of \<^loc> (which was original meant as workaround for "local" syntax);
Sun, 19 Jun 2011 14:36:06 +0200 wenzelm added glyphs 21e0..21e4, 21e6..21e9, 2759 from DejaVuSansMono;
Sun, 19 Jun 2011 14:31:08 +0200 wenzelm names for control symbols without "^", which is relevant for completion;
Sun, 19 Jun 2011 14:11:06 +0200 wenzelm some unicode chars for special control symbols;
Sun, 19 Jun 2011 00:03:44 +0200 wenzelm tuned;
Sat, 18 Jun 2011 23:51:22 +0200 wenzelm tuned markup;
Sat, 18 Jun 2011 23:34:34 +0200 wenzelm avoid setTokenMarker fluctuation on buffer reload etc. via static isabelle_token_marker, which is installed by hijacking the jEdit ModeProvider;
Sat, 18 Jun 2011 22:01:22 +0200 wenzelm proper gfx.setColor;
Sat, 18 Jun 2011 21:26:47 +0200 wenzelm proper x1;
Sat, 18 Jun 2011 21:20:22 +0200 wenzelm convenience functions;
Sat, 18 Jun 2011 21:03:52 +0200 wenzelm more robust caret painting wrt. surrogate characters;
Sat, 18 Jun 2011 18:57:38 +0200 wenzelm do not control malformed symbols;
Sat, 18 Jun 2011 18:31:55 +0200 wenzelm Buffer.editSyntaxStyle: mask extended syntax styles;
Sat, 18 Jun 2011 18:17:08 +0200 wenzelm hardwired abbreviations for standard control symbols;
Sat, 18 Jun 2011 17:42:28 +0200 wenzelm updated to jedit_build-20110618, which is required for sub/superscript rendering;
Sat, 18 Jun 2011 17:33:27 +0200 wenzelm basic support for extended syntax styles: sub/superscript;
Sat, 18 Jun 2011 17:32:13 +0200 wenzelm tuned -- Map.empty serves as partial function;
Sat, 18 Jun 2011 17:30:44 +0200 wenzelm proper place for config files (cf. 55866987a7d9);
Sat, 18 Jun 2011 15:32:05 +0200 wenzelm tuned signature;
Sat, 18 Jun 2011 15:18:57 +0200 wenzelm merged
Fri, 17 Jun 2011 20:38:43 +0200 kleing IMP compiler with int, added reverse soundness direction
Sat, 18 Jun 2011 15:11:33 +0200 wenzelm proper place for config files;
Sat, 18 Jun 2011 15:07:16 +0200 wenzelm tuned markup;
Sat, 18 Jun 2011 14:48:56 +0200 wenzelm highlight via foreground painter, using alpha channel;
Sat, 18 Jun 2011 12:58:41 +0200 wenzelm tuned signature;
Sat, 18 Jun 2011 12:49:55 +0200 wenzelm tuned text;
Sat, 18 Jun 2011 12:37:42 +0200 wenzelm inner literal/delimiter corresponds to outer keyword/operator;
Sat, 18 Jun 2011 12:13:42 +0200 wenzelm tuned markup;
Sat, 18 Jun 2011 11:45:07 +0200 wenzelm more uniform treatment of "keyword" vs. "operator";
Sat, 18 Jun 2011 11:22:03 +0200 wenzelm simplified Line_Context (again);
Sat, 18 Jun 2011 00:05:29 +0200 wenzelm more robust treatment of partial range restriction;
Sat, 18 Jun 2011 00:03:58 +0200 wenzelm select_markup: no filtering here -- results may be distorted anyway;
Fri, 17 Jun 2011 23:20:34 +0200 wenzelm more explicit treatment of ranges after revert/convert, which may well distort the overall start/end positions;
Fri, 17 Jun 2011 23:18:22 +0200 wenzelm more explicit error message;
Fri, 17 Jun 2011 14:35:24 +0200 wenzelm merged
Thu, 16 Jun 2011 13:50:35 +0200 blanchet gave up an optimization that sometimes lead to unsound proofs -- in short, facts talking about a schematic type variable can encode a cardinality constraint and be consistent with HOL, e.g. "card (UNIV::?'a set) = 1 ==> ALL x y. x = y"
Thu, 16 Jun 2011 13:50:35 +0200 blanchet added missing case in pattern matching -- solves Waldmeister "Match" exceptions that have been plaguing some users
Thu, 16 Jun 2011 13:50:35 +0200 blanchet fixed soundness bug related to extensionality
(0) -30000 -10000 -1920 +1920 +10000 +30000 tip