NEWS
Thu, 04 Nov 2010 09:54:16 +0100 haftmann merged
Wed, 03 Nov 2010 12:20:33 +0100 haftmann Theory Multiset provides stable quicksort implementation of sort_key.
Wed, 03 Nov 2010 22:26:53 +0100 blanchet standardize on seconds for Nitpick and Sledgehammer timeouts
Wed, 03 Nov 2010 11:33:51 +0100 wenzelm discontinued obsolete function sys_error and exception SYS_ERROR;
Sun, 31 Oct 2010 11:45:45 +0100 nipkow merged
Fri, 29 Oct 2010 17:57:36 +0200 nipkow Plus -> Sum_Type.Plus
Sat, 30 Oct 2010 21:08:20 +0200 wenzelm support for real valued preferences;
Sat, 30 Oct 2010 16:33:58 +0200 wenzelm support for real valued configuration options;
Fri, 29 Oct 2010 11:07:21 +0200 wenzelm merged
Fri, 29 Oct 2010 08:44:46 +0200 bulwahn NEWS
Thu, 28 Oct 2010 23:19:52 +0200 wenzelm discontinued obsolete ML antiquotation @{theory_ref};
Tue, 26 Oct 2010 15:06:36 +0200 krauss fixed typo
Tue, 26 Oct 2010 13:50:18 +0200 krauss NEWS
Tue, 26 Oct 2010 11:45:12 +0200 boehmes joined setup of SMT solvers in one place; turned Z3-specific options into SMT options (renamed configuration options from z3_* to smt_*); more detailed SMT exception; improved SMT filter interface
Mon, 25 Oct 2010 16:18:00 +0200 wenzelm merged
Mon, 25 Oct 2010 16:17:16 +0200 wenzelm significantly improved Isabelle/Isar implementation manual;
Mon, 25 Oct 2010 11:42:05 +0200 blanchet merged
Mon, 25 Oct 2010 10:30:46 +0200 blanchet introduced manual version of "Auto Solve" as "solve_direct"
Mon, 25 Oct 2010 11:16:23 +0200 wenzelm added ML antiquotation @{assert};
Sun, 24 Oct 2010 20:37:30 +0200 nipkow renamed nat_number
Fri, 22 Oct 2010 11:11:34 +0200 blanchet make Sledgehammer minimizer fully work with SMT
Thu, 21 Oct 2010 14:55:09 +0200 blanchet use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
Thu, 14 Oct 2010 12:40:14 +0200 krauss NEWS
Wed, 06 Oct 2010 17:44:21 +0200 blanchet merged
Tue, 05 Oct 2010 12:06:08 +0200 blanchet document latest changes to Meson/Metis/Sledgehammer
Mon, 04 Oct 2010 14:46:48 +0200 haftmann turned distinct and sorted into inductive predicates: yields nice induction principles for free
Fri, 01 Oct 2010 16:05:25 +0200 haftmann constant `contents` renamed to `the_elem`
Tue, 28 Sep 2010 15:33:56 +0200 haftmann NEWS
Tue, 28 Sep 2010 09:54:07 +0200 krauss no longer declare .psimps rules as [simp].
Fri, 24 Sep 2010 16:17:59 +0200 wenzelm clarified @{type} antiquotation: abbreviations and nonterminals count as "syntactic", disallow TFrees;
Thu, 23 Sep 2010 09:53:52 +0200 haftmann CONTRIBUTORS and NEWS
Wed, 22 Sep 2010 18:21:48 +0200 wenzelm renamed setmp_noncritical to Unsynchronized.setmp to emphasize its meaning;
Mon, 20 Sep 2010 16:05:25 +0200 wenzelm renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
Fri, 17 Sep 2010 22:17:57 +0200 wenzelm discontinued Output.debug, which belongs to early PGIP experiments (b6788dbd2ef9) and causes just too many problems (like spamming the message channel if it is used by more than one module);
Mon, 13 Sep 2010 14:55:21 +0200 haftmann merged
Mon, 13 Sep 2010 14:53:56 +0200 haftmann 'class' and 'type' are now antiquoations by default
Mon, 13 Sep 2010 11:13:15 +0200 nipkow renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
Mon, 13 Sep 2010 08:43:48 +0200 nipkow added and renamed lemmas
Fri, 10 Sep 2010 15:17:44 +0200 wenzelm merged
Thu, 09 Sep 2010 14:38:14 +0200 bulwahn changing String.literal to a type instead of a datatype
Thu, 09 Sep 2010 18:32:21 +0200 wenzelm NEWS: some notes on interrupts;
Wed, 08 Sep 2010 13:25:22 +0200 haftmann NEWS
Tue, 07 Sep 2010 12:04:18 +0200 nipkow renamed expand_*_eq in HOLCF as well
Mon, 06 Sep 2010 22:08:49 +0200 wenzelm ML_Context.thm and ML_Context.thms no longer pervasive;
Mon, 06 Sep 2010 12:38:45 +0200 wenzelm merged;
Sun, 05 Sep 2010 21:39:24 +0200 krauss removed duplicate lemma
Sun, 05 Sep 2010 23:16:21 +0200 wenzelm turned show_brackets into proper configuration option;
Sun, 05 Sep 2010 21:41:24 +0200 wenzelm turned show_sorts/show_types into proper configuration options;
Fri, 03 Sep 2010 23:54:48 +0200 wenzelm turned eta_contract into proper configuration option;
Fri, 03 Sep 2010 22:36:16 +0200 wenzelm configuration options Syntax.ambiguity_enabled (inverse of former Syntax.ambiguity_is_error), Syntax.ambiguity_level (with Isar attribute "syntax_ambiguity_level"), Syntax.ambiguity_limit;
Fri, 03 Sep 2010 21:13:53 +0200 wenzelm pretty_goals: turned some global references and function arguments into configuration options (goals_limit = 10, goals_total = true, show_main_goal = false) depending on the context;
Fri, 03 Sep 2010 12:01:47 +0200 wenzelm merged
Thu, 02 Sep 2010 18:45:23 +0200 hoelzl merged
Thu, 02 Sep 2010 13:32:17 +0200 hoelzl NEWS
Fri, 03 Sep 2010 11:21:58 +0200 wenzelm turned show_consts into proper configuration option;
Thu, 02 Sep 2010 00:48:07 +0200 wenzelm turned show_question_marks into proper configuration option;
Sat, 28 Aug 2010 16:14:32 +0200 haftmann formerly unnamed infix equality now named HOL.eq
Sat, 28 Aug 2010 11:42:33 +0200 haftmann merged
Fri, 27 Aug 2010 19:34:23 +0200 haftmann renamed class/constant eq to equal; tuned some instantiations
Fri, 27 Aug 2010 18:00:45 +0200 wenzelm merged
Fri, 27 Aug 2010 14:25:29 +0200 haftmann merged
Fri, 27 Aug 2010 14:25:07 +0200 haftmann official support for Scala
Fri, 27 Aug 2010 14:14:08 +0200 wenzelm structure Unsynchronized is never opened and set/reset/toggle have been discontinued;
Fri, 27 Aug 2010 12:57:55 +0200 wenzelm merged, resolving some minor conflicts in src/HOL/Tools/Predicate_Compile/code_prolog.ML;
Fri, 27 Aug 2010 10:56:46 +0200 haftmann formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
Thu, 26 Aug 2010 21:03:14 +0200 haftmann NEWS
Fri, 27 Aug 2010 12:40:20 +0200 wenzelm proper context for various Thy_Output options, via official configuration options in ML and Isar;
Wed, 25 Aug 2010 14:18:09 +0200 wenzelm discontinued obsolete 'global' and 'local' commands;
Mon, 23 Aug 2010 19:35:57 +0200 hoelzl Rewrite the Probability theory.
Mon, 23 Aug 2010 11:17:13 +0200 haftmann dropped type classes mult_mono and mult_mono1; tuned names of technical rule duplicates
Fri, 20 Aug 2010 17:48:30 +0200 haftmann split and enriched theory SetsAndFunctions
Thu, 19 Aug 2010 17:41:52 +0200 wenzelm merged
Thu, 19 Aug 2010 16:08:53 +0200 haftmann deglobalized named HOL constants
Wed, 18 Aug 2010 17:03:09 +0200 haftmann merged
Wed, 18 Aug 2010 17:01:12 +0200 haftmann NEWS
Wed, 18 Aug 2010 15:01:57 +0200 haftmann more helpful NEWS entry
Tue, 17 Aug 2010 16:44:21 +0200 haftmann preemptive NEWS
Wed, 18 Aug 2010 14:55:09 +0200 haftmann NEWS
Wed, 18 Aug 2010 12:26:48 +0200 haftmann deglobalization
Tue, 17 Aug 2010 18:41:55 +0200 wenzelm discontinued support for Poly/ML 5.0 and 5.1 versions;
Tue, 17 Aug 2010 14:33:39 +0200 haftmann NEWS and CONTRIBUTORS
Wed, 11 Aug 2010 14:31:40 +0200 haftmann NEWS
Tue, 03 Aug 2010 16:33:11 +0200 wenzelm theory loading: only the master source file is looked-up in the implicit load path;
Sat, 31 Jul 2010 23:32:05 +0200 ballarin Documentation of 'interpret' updated.
Thu, 22 Jul 2010 22:31:20 +0200 wenzelm discontinued special treatment of ML files -- no longer complete extensions on demand;
Wed, 21 Jul 2010 15:02:51 +0200 wenzelm ML antiquotations @{theory} and @{theory_ref} refer to the theory ancestry, not any accidental theory loader state;
Wed, 14 Jul 2010 14:53:44 +0200 haftmann export_code without file prints to standard output
Wed, 07 Jul 2010 08:25:22 +0200 bulwahn added NEWS entry
Fri, 02 Jul 2010 10:47:50 +0200 haftmann fixed spelling
Thu, 01 Jul 2010 16:55:05 +0200 haftmann "prod" and "sum" replace "*" and "+" respectively; qualified constants Set.member and Set.Collect
Thu, 01 Jul 2010 10:57:19 +0200 hoelzl Updated NEWS
Tue, 29 Jun 2010 07:55:18 +0200 haftmann merged
Mon, 28 Jun 2010 15:32:06 +0200 haftmann dropped ancient infix mem; refined code generation operations in List.thy
Mon, 28 Jun 2010 15:03:07 +0200 haftmann merged constants "split" and "prod_case"
Fri, 25 Jun 2010 11:48:37 +0200 wenzelm explicit treatment of UTF8 sequences as Isabelle symbols;
Mon, 21 Jun 2010 17:41:57 +0200 wenzelm merged, resolving conflicts in doc-src/IsarRef/Thy/HOL_Specific.thy;
Tue, 15 Jun 2010 14:28:22 +0200 haftmann added code_simp infrastructure
Tue, 15 Jun 2010 07:42:48 +0200 haftmann merged
Mon, 14 Jun 2010 12:01:30 +0200 haftmann NEWS
Mon, 14 Jun 2010 15:10:36 +0200 haftmann removed simplifier congruence rule of "prod_case"
Thu, 10 Jun 2010 12:24:01 +0200 haftmann qualified type "*"; qualified constants Pair, fst, snd, split
Tue, 08 Jun 2010 16:37:19 +0200 haftmann qualified types "+" and nat; qualified constants Ball, Bex, Suc, curry; modernized some specifications
Mon, 07 Jun 2010 17:39:32 +0200 wenzelm back to non-release mode;
Mon, 21 Jun 2010 11:24:19 +0200 wenzelm final tuning; Isabelle2009-2
Fri, 11 Jun 2010 13:25:28 +0200 wenzelm NEWS: IsabelleText font;
Mon, 07 Jun 2010 17:52:30 +0200 berghofe Documented changes in induct, cases, and nominal_induct method.
Mon, 07 Jun 2010 11:42:32 +0200 wenzelm more NEWS;
Mon, 07 Jun 2010 11:27:08 +0200 wenzelm more NEWS;
Fri, 04 Jun 2010 16:02:46 +0200 krauss NEWS (more strict internal axioms/defs format)
Fri, 04 Jun 2010 11:30:46 +0200 wenzelm spelling;
Thu, 03 Jun 2010 22:17:36 +0200 wenzelm diagnostic commands 'ML_val' and 'ML_command' may refer to antiquotations @{Isar.state} and @{Isar.goal};
Thu, 03 Jun 2010 16:39:50 +0200 krauss clarified
Thu, 03 Jun 2010 16:39:05 +0200 krauss mention unconstrain in NEWS
Wed, 02 Jun 2010 21:53:03 +0200 wenzelm improved parallelism of proof term normalization;
Tue, 01 Jun 2010 17:52:19 +0200 blanchet merged
Tue, 01 Jun 2010 17:52:00 +0200 blanchet update NEWS
Tue, 01 Jun 2010 15:38:47 +0200 blanchet removed "nitpick_intro" attribute -- Nitpick noew uses Spec_Rules instead
Tue, 01 Jun 2010 12:20:08 +0200 blanchet added "atoms" option to Nitpick (request from Karlsruhe) + wrap Refute. functions to "nitpick_util.ML"
Mon, 31 May 2010 22:08:40 +0200 wenzelm notes on Isabelle/jEdit;
Mon, 31 May 2010 21:06:57 +0200 wenzelm modernized some structure names, keeping a few legacy aliases;
Thu, 27 May 2010 21:37:42 +0200 wenzelm merged
Thu, 27 May 2010 16:30:26 +0200 boehmes merged
Thu, 27 May 2010 14:54:13 +0200 boehmes moved SMT into the HOL image
Thu, 27 May 2010 18:10:37 +0200 wenzelm renamed structure PrintMode to Print_Mode, keeping the old name as legacy alias for some time;
Thu, 27 May 2010 17:41:27 +0200 wenzelm renamed structure TypeInfer to Type_Infer, keeping the old name as legacy alias for some time;
Thu, 27 May 2010 15:28:23 +0200 wenzelm misc updates for release;
Thu, 27 May 2010 15:15:20 +0200 wenzelm constant Rat.normalize needs to be qualified;
Sat, 22 May 2010 17:44:12 -0700 huffman NEWS: removed fixrec_simp attribute
Thu, 20 May 2010 16:35:52 +0200 haftmann turned old-style mem into an input abbreviation
Tue, 18 May 2010 19:00:55 -0700 huffman remove several redundant lemmas about floor and ceiling
Tue, 18 May 2010 00:01:51 +0200 wenzelm merged
Mon, 17 May 2010 10:58:58 +0200 haftmann dropped old Library/Word.thy and toy example ex/Adder.thy
Tue, 18 May 2010 00:01:03 +0200 wenzelm do not open Legacy by default;
Mon, 17 May 2010 15:11:25 +0200 wenzelm renamed structure OuterLex to Token and type token to Token.T, keeping legacy aliases for some time;
Sat, 15 May 2010 23:40:00 +0200 wenzelm renamed structure OuterSyntax to Outer_Syntax, keeping the old name as alias for some time;
Sat, 15 May 2010 23:32:15 +0200 wenzelm renamed structure SpecParse to Parse_Spec, keeping the old name as alias for some time;
Sat, 15 May 2010 22:24:25 +0200 wenzelm renamed structure OuterKeyword to Keyword and OuterParse to Parse, keeping the old names as legacy aliases for some time;
Fri, 14 May 2010 23:32:48 +0200 blanchet added some Sledgehammer news
Fri, 14 May 2010 23:16:33 +0200 blanchet document Nitpick changes
Thu, 13 May 2010 14:34:05 +0200 nipkow Multiset: renamed, added and tuned lemmas;
Wed, 12 May 2010 13:34:24 +0200 wenzelm minor tuning;
Wed, 12 May 2010 13:21:23 +0200 wenzelm reverted parts of 7902dc7ea11d -- note that NEWS of published Isabelle releases are essentially read-only;
Wed, 12 May 2010 11:13:33 +0200 hoelzl clarified NEWS entry
Wed, 12 May 2010 11:08:15 +0200 hoelzl merged
Wed, 12 May 2010 11:07:46 +0200 hoelzl added NEWS entry
Tue, 11 May 2010 12:05:19 -0700 huffman removed lemma real_sq_order; use power2_le_imp_le instead
Tue, 11 May 2010 11:58:34 -0700 huffman fix spelling of 'superseded'
Tue, 11 May 2010 11:57:14 -0700 huffman NEWS: removed theory PReal
Tue, 11 May 2010 11:40:39 -0700 huffman collected NEWS updates for HOLCF
Tue, 11 May 2010 08:36:02 +0200 haftmann renamed former Int.int_induct to Int.int_of_nat_induct, former Presburger.int_induct to Int.int_induct: is more conservative and more natural than the intermediate solution
Tue, 11 May 2010 08:29:42 +0200 haftmann theorem Presburger.int_induct has been renamed to Int.int_bidirectional_induct
Thu, 06 May 2010 17:59:19 +0200 haftmann dropped duplicate comp_arith
Tue, 04 May 2010 14:44:30 +0200 wenzelm merged
Tue, 04 May 2010 08:55:34 +0200 haftmann NEWS
Mon, 03 May 2010 14:38:18 +0200 wenzelm old NEWS on global operations;
Thu, 29 Apr 2010 20:00:26 +0200 wenzelm removed some Emacs junk;
Thu, 29 Apr 2010 18:41:38 +0200 haftmann merged
Thu, 29 Apr 2010 15:00:39 +0200 haftmann NEWS: code_reflect
Thu, 29 Apr 2010 17:47:53 +0200 wenzelm allow concrete syntax for local entities within a proof body, either via regular mixfix annotations to 'fix' etc. or the separate 'write' command;
Wed, 28 Apr 2010 13:29:57 +0200 haftmann merged
Wed, 28 Apr 2010 13:29:39 +0200 haftmann empty class specifcations observe default sort
Wed, 28 Apr 2010 12:21:55 +0200 wenzelm command 'defaultsort' is renamed to 'default_sort', it works within a local theory context;
Wed, 28 Apr 2010 08:25:02 +0200 haftmann term_typ: print styled term
Tue, 27 Apr 2010 21:46:10 +0200 wenzelm monotonic sort certification: sorts are no longer minimized at the kernel boundary, only when reading input from the end-user;
Tue, 27 Apr 2010 10:42:41 +0200 haftmann NEWS and CONTRIBUTORS
Mon, 26 Apr 2010 21:45:08 +0200 wenzelm command 'example_proof' opens an empty proof body;
Mon, 26 Apr 2010 11:34:15 +0200 haftmann dropped group_simps, ring_simps, field_eq_simps; classes division_ring_inverse_zero, field_inverse_zero, linordered_field_inverse_zero
Fri, 23 Apr 2010 22:48:07 +0200 wenzelm explicit 'schematic_theorem' etc. for schematic theorem statements;
Fri, 23 Apr 2010 13:58:14 +0200 haftmann modernized abstract algebra theories
Mon, 19 Apr 2010 10:56:26 +0200 wenzelm polyml-platform script is superseded by ISABELLE_PLATFORM;
Fri, 16 Apr 2010 22:18:59 +0200 wenzelm keep localized 'types' as regular non-old-style version -- 'type_abbrev' as 'type' just causes too many problems, e.g. clash with "type" in translations or "type:" argument syntax;
Fri, 16 Apr 2010 22:15:09 +0200 wenzelm separate commands 'hide_class', 'hide_type', 'hide_const', 'hide_fact';
Fri, 16 Apr 2010 10:52:10 +0200 wenzelm added ML antiquotation @{make_string}, which produces proper pretty printed version in Poly/ML 5.3.0 or later;
Thu, 15 Apr 2010 12:27:14 +0200 haftmann theory RBT with abstract type of red-black trees backed by implementation RBT_Impl
Wed, 07 Apr 2010 19:17:10 +0200 ballarin Merged resolving conflicts NEWS and locale.ML.
Mon, 15 Feb 2010 01:34:08 +0100 ballarin Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
Tue, 30 Mar 2010 23:12:55 +0200 krauss NEWS
Sun, 28 Mar 2010 16:13:29 +0200 wenzelm configuration options admit dynamic default values;
Sat, 27 Mar 2010 21:34:28 +0100 boehmes re-introduce reference to control simplifier tracing (needed for ProofGeneral settings menu) (cf. 12bb31230550)
Fri, 26 Mar 2010 23:46:22 +0100 boehmes replaced references 'trace_simp' and 'debug_simp' by configuration options stored in the context
Sat, 20 Mar 2010 17:33:11 +0100 wenzelm renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
Wed, 17 Mar 2010 08:11:24 -0700 huffman NEWS: Nat_Bijection library
Sat, 13 Mar 2010 20:33:14 +0100 wenzelm local theory specifications handle hidden polymorphism implicitly;
Sat, 13 Mar 2010 17:19:12 +0100 wenzelm removed obsolete HOL/Library/Coinductive_List.thy, superceded by thys/Coinductive/Coinductive_List.thy in AFP/f2f5727b77d0;
Sat, 13 Mar 2010 15:12:47 +0100 wenzelm command 'typedef' now works within a local theory context;
Thu, 11 Mar 2010 15:52:33 +0100 haftmann NEWS
Thu, 11 Mar 2010 14:38:09 +0100 haftmann fixed typo
Tue, 09 Mar 2010 23:32:13 +0100 wenzelm localized typedecl;
Sat, 06 Mar 2010 15:39:16 +0100 wenzelm eliminated Args.bang_facts (legacy feature);
Wed, 03 Mar 2010 15:40:39 +0100 wenzelm authentic syntax for *all* logical entities;
Mon, 01 Mar 2010 17:09:42 +0100 wenzelm added type_notation command;
Sat, 27 Feb 2010 20:56:03 +0100 wenzelm clarified @{const_name} (only logical consts) vs. @{const_abbrev};
Sat, 27 Feb 2010 13:32:38 +0100 wenzelm ML antiquotations for type classes;
Fri, 26 Feb 2010 10:57:35 +0100 haftmann merged
Wed, 24 Feb 2010 14:34:40 +0100 haftmann renamed theory Rational to Rat
Thu, 25 Feb 2010 22:08:43 +0100 wenzelm more orthogonal antiquotations for type constructors;
Wed, 24 Feb 2010 20:37:01 +0100 wenzelm allow general mixfix syntax for type constructors;
Mon, 22 Feb 2010 16:03:48 +0100 haftmann NEWS
Mon, 22 Feb 2010 09:30:50 +0100 haftmann NEWS
Mon, 22 Feb 2010 09:17:49 +0100 haftmann merged
Mon, 22 Feb 2010 09:15:10 +0100 haftmann NEWS
Fri, 19 Feb 2010 16:56:39 +0100 haftmann NEWS
Fri, 19 Feb 2010 14:46:59 +0100 haftmann NEWS
Sun, 21 Feb 2010 21:41:29 +0100 wenzelm tuned;
Sun, 21 Feb 2010 21:33:11 +0100 wenzelm NEWS: authentic syntax for *all* term constants;
Mon, 15 Feb 2010 18:03:42 +0100 wenzelm renamed InfixName to Infix etc.;
Mon, 15 Feb 2010 17:17:51 +0100 wenzelm discontinued unnamed infix syntax;
Thu, 11 Feb 2010 22:03:37 +0100 wenzelm added ML antiquotation @{syntax_const};
Wed, 10 Feb 2010 19:37:34 +0100 wenzelm renamed Library/Quotient.thy to Library/Quotient_Type.thy to avoid clash with new theory Quotient in Main HOL;
Wed, 10 Feb 2010 14:12:30 +0100 haftmann NEWS
Wed, 10 Feb 2010 08:49:26 +0100 haftmann moved constants inverse and divide to Ring.thy
Mon, 08 Feb 2010 17:12:38 +0100 haftmann renamed OrderedGroup to Groups; split theory Ring_and_Field into Rings Fields
Mon, 08 Feb 2010 14:22:22 +0100 haftmann NEWS: ax_simps
Mon, 08 Feb 2010 14:08:32 +0100 haftmann merged
Mon, 08 Feb 2010 14:06:41 +0100 haftmann separate library theory for type classes combining lattices with various algebraic structures
Mon, 08 Feb 2010 11:13:30 +0100 haftmann merged
Mon, 08 Feb 2010 10:36:02 +0100 haftmann separate theory for index structures
Fri, 05 Feb 2010 14:33:31 +0100 haftmann more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
Sun, 07 Feb 2010 19:33:34 +0100 wenzelm renamed old-style Drule.standard to Drule.export_without_context, to emphasize that this is in no way a standard operation;
Sat, 06 Feb 2010 14:39:33 +0100 wenzelm misc tuning;
Thu, 28 Jan 2010 11:48:49 +0100 haftmann new theory Algebras.thy for generic algebraic structures
Fri, 22 Jan 2010 16:56:51 +0100 haftmann HOLogic.strip_psplits: types are ordered after syntactic appearance, not after corresponding de-Bruin index (closer correspondence to similar strip operations)
Fri, 22 Jan 2010 13:38:40 +0100 haftmann NEWS
Tue, 19 Jan 2010 16:52:01 +0100 hoelzl Add transpose to the List-theory.
Mon, 04 Jan 2010 23:20:35 +0100 wenzelm discontinued old TheoryDataFun, but retain Theory_Data_PP with is Pretty.pp argument to merge (still required in exotic situations -- hard to get rid of);
Mon, 04 Jan 2010 22:16:48 +0100 wenzelm discontinued old ISABELLE and ISATOOL environment settings;
Mon, 04 Jan 2010 11:55:23 +0100 wenzelm discontinued special HOL_USEDIR_OPTIONS;
Wed, 23 Dec 2009 08:31:14 +0100 haftmann reduced code generator cache to the baremost minimum; corrected spelling
Fri, 11 Dec 2009 20:44:15 +0100 wenzelm Subgoal.FOCUS (and variants): resulting goal state is normalized as usual for resolution;
Fri, 11 Dec 2009 14:32:24 +0100 haftmann NEWS
Sat, 05 Dec 2009 20:02:21 +0100 haftmann tuned lattices theory fragements; generlized some lemmas from sets to lattices
Fri, 04 Dec 2009 18:51:15 +0100 haftmann merged, resolving minor conflicts
Fri, 04 Dec 2009 18:43:42 +0100 haftmann NEWS
Fri, 04 Dec 2009 11:44:57 +0100 wenzelm back to after-release mode;
Mon, 23 Nov 2009 22:47:08 +0100 wenzelm more tuning for release;
Mon, 23 Nov 2009 16:15:18 +0100 haftmann tuned NEWS
Sun, 22 Nov 2009 17:02:46 +0100 haftmann more uniform view on various number theory refinement steps
Sun, 22 Nov 2009 14:49:36 +0100 wenzelm more NEWS, more tuning for release;
Sun, 22 Nov 2009 14:13:18 +0100 wenzelm misc tuning and updates for official release;
Sat, 21 Nov 2009 11:47:38 +1100 kleing wwwfind support currently for Linux only
less more (0) -1000 -240 tip