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
Fri, 20 Nov 2009 14:35:55 -0800 huffman NEWS: HOLCF changes since the last release
Fri, 20 Nov 2009 22:28:39 +1100 kleing added NEWS item for wwwfind
Thu, 19 Nov 2009 11:57:30 +0100 hoelzl Added the contributions of Robert Himmelmann to CONTRIBUTIONS and NEWS
Fri, 13 Nov 2009 19:48:32 +0100 nipkow -
Thu, 12 Nov 2009 20:38:57 +0100 bulwahn added a tabled implementation of the reflexive transitive closure
Thu, 12 Nov 2009 17:21:48 +0100 hoelzl New list theorems; added map_map to simpset, this is the prefered direction; allow sorting by a key
Thu, 12 Nov 2009 09:11:31 +0100 bulwahn announcing the predicate compiler in NEWS and CONTRIBUTORS
Sun, 08 Nov 2009 21:00:05 +0100 wenzelm updated functor Theory_Data, Proof_Data, Generic_Data;
Fri, 06 Nov 2009 17:52:57 +0100 boehmes added documentation for local SMT solver setup and available SMT options,
Fri, 06 Nov 2009 14:42:42 +0100 krauss renamed method induct_scheme to induction_schema
Fri, 06 Nov 2009 13:49:19 +0100 krauss NEWS
Tue, 03 Nov 2009 17:54:24 +0100 boehmes added HOL-Boogie
Fri, 30 Oct 2009 14:00:43 +0100 haftmann combined former theories Divides and IntDiv to one theory Divides
Wed, 28 Oct 2009 12:21:38 +0000 paulson Probability tweaks
Wed, 28 Oct 2009 11:42:31 +0000 paulson New theory Probability, which contains a development of measure theory
Tue, 27 Oct 2009 14:46:03 +0000 paulson merged
Tue, 27 Oct 2009 12:59:57 +0000 paulson New theory SupInf of the supremum and infimum operators for sets of reals.
Mon, 26 Oct 2009 09:14:29 +0100 blanchet merged
Thu, 22 Oct 2009 14:51:47 +0200 blanchet added Nitpick's theory and ML files to Isabelle/HOL;
Fri, 23 Oct 2009 17:12:36 +0200 haftmann turned off old quickcheck
Thu, 22 Oct 2009 09:27:48 +0200 nipkow inv_onto -> inv_into
Tue, 20 Oct 2009 16:13:01 +0200 haftmann replaced old_style infixes eq_set, subset, union, inter and variants by generic versions
Tue, 20 Oct 2009 10:11:30 +0200 boehmes added proof reconstructon for Z3,
Sun, 18 Oct 2009 18:07:44 +0200 nipkow certificates for sos
Sun, 18 Oct 2009 12:07:56 +0200 nipkow merged
Sun, 18 Oct 2009 12:07:25 +0200 nipkow Inv -> inv_onto, inv abbr. inv_onto UNIV.
Sat, 17 Oct 2009 23:07:53 +0200 ballarin Merged.
Sat, 17 Oct 2009 22:58:18 +0200 ballarin Finished revisions of locales tutorial.
Sat, 17 Oct 2009 16:58:03 +0200 wenzelm operations of structure Skip_Proof (formerly SkipProof) no longer require quick_and_dirty mode;
Fri, 09 Oct 2009 10:00:47 +0200 haftmann term styles also cover antiquotations term_type and typeof
Thu, 08 Oct 2009 15:16:13 +0200 haftmann new generalized concept for term styles
Thu, 01 Oct 2009 20:49:46 +0200 ballarin News entry: inheritance of mixins; print_interps.
Wed, 30 Sep 2009 09:25:18 +0200 haftmann merged
Wed, 30 Sep 2009 08:28:23 +0200 haftmann mandatory prefix where appropriate
Tue, 29 Sep 2009 16:42:29 +0200 wenzelm Synchronized and Unsynchronized;
Fri, 25 Sep 2009 10:20:03 +0200 haftmann NEWS; corrected spelling
Tue, 22 Sep 2009 15:39:46 +0200 haftmann merged
Mon, 21 Sep 2009 15:35:14 +0200 haftmann added note on simp rules
Mon, 21 Sep 2009 11:01:49 +0200 haftmann merged
Sat, 19 Sep 2009 07:38:03 +0200 haftmann inter and union are mere abbreviations for inf and sup
Tue, 22 Sep 2009 15:36:55 +0200 haftmann be more cautious wrt. simp rules: inf_absorb1, inf_absorb2, sup_absorb1, sup_absorb2 are no simp rules by default any longer
Fri, 18 Sep 2009 18:13:19 +0200 boehmes added new method "smt": an oracle-based connection to external SMT solvers
Fri, 18 Sep 2009 14:09:38 +0200 haftmann INTER and UNION are mere abbreviations for INFI and SUPR
Fri, 18 Sep 2009 07:54:26 +0200 haftmann tuned NEWS, added CONTRIBUTORS
Thu, 17 Sep 2009 15:04:46 +0100 paulson NEWS: New method metisFT
Wed, 16 Sep 2009 13:43:07 +0200 haftmann Inter and Union are mere abbreviations for Inf and Sup; tuned
Tue, 01 Sep 2009 21:46:38 +0200 haftmann corrected spelling
Tue, 01 Sep 2009 15:39:33 +0200 haftmann some reorganization of number theory
Mon, 31 Aug 2009 20:34:48 +0200 krauss moved lemma Wellfounded.in_inv_image to Relation.thy
Fri, 28 Aug 2009 21:15:22 +0200 wenzelm discontinued Display.pretty_ctyp/cterm etc.;
Fri, 28 Aug 2009 11:31:49 +0200 wenzelm misc updates and tuning;
Fri, 21 Aug 2009 13:38:57 +0200 boehmes added Mirabelle to NEWS
Wed, 12 Aug 2009 00:26:01 +0200 wenzelm added PARALLEL_CHOICE, PARALLEL_GOALS;
Tue, 04 Aug 2009 16:13:16 +0200 wenzelm etc/components;
Wed, 29 Jul 2009 12:12:01 +0200 nipkow sos documentation
Tue, 28 Jul 2009 13:37:09 +0200 haftmann Set.UNIV and Set.empty are mere abbreviations for top and bot
Mon, 27 Jul 2009 21:47:41 +0200 krauss "more standard" argument order of relation composition (op O)
Mon, 27 Jul 2009 09:01:13 +0200 haftmann NEWS
Sun, 26 Jul 2009 22:33:32 +0200 wenzelm tacticals FOCUS and FOCUS_PARAMS;
Thu, 23 Jul 2009 18:44:10 +0200 wenzelm Proper context for simpset_of, claset_of, clasimpset_of.
Wed, 22 Jul 2009 14:21:52 +0200 haftmann merged
Wed, 22 Jul 2009 14:20:32 +0200 haftmann set intersection and union now named inter and union
Wed, 22 Jul 2009 11:23:09 +0200 wenzelm merged, resolving trivial conflict;
Wed, 22 Jul 2009 10:49:26 +0200 nipkow News
Tue, 21 Jul 2009 01:05:10 +0200 wenzelm Display.pretty_thm now requires a proper context;
Mon, 20 Jul 2009 13:52:27 +0200 wenzelm merged
Tue, 14 Jul 2009 15:55:27 +0200 haftmann merged
Tue, 14 Jul 2009 15:54:19 +0200 haftmann refinement of lattice classes
Sun, 19 Jul 2009 19:24:04 +0200 wenzelm parallel_proofs: more fine-grained control with optional parallel checking of nested Isar proofs;
Tue, 14 Jul 2009 10:53:44 +0200 haftmann NEWS and CONTRIBUTORS
Thu, 09 Jul 2009 22:01:41 +0200 wenzelm renamed functor TableFun to Table, and GraphFun to Graph;
Thu, 02 Jul 2009 17:33:36 +0200 wenzelm renamed NamedThmsFun to Named_Thms;
Thu, 02 Jul 2009 17:30:54 +0200 wenzelm misc tuning;
Tue, 30 Jun 2009 19:54:04 +0200 hoelzl NEWS updated
Mon, 29 Jun 2009 23:29:11 +0200 hoelzl Implemented taylor series expansion for approximation
Fri, 26 Jun 2009 19:44:39 +0200 nipkow lcm abs lemmas
Thu, 25 Jun 2009 20:26:17 +0200 hoelzl NEWS updated
Mon, 08 Jun 2009 18:37:35 +0200 hoelzl Added new evaluator "approximate"
Thu, 25 Jun 2009 14:59:29 +0200 haftmann arbitrary farewell
Wed, 24 Jun 2009 09:41:14 +0200 nipkow corrected and unified thm names
Tue, 23 Jun 2009 16:27:12 +0200 haftmann tuned interfaces of datatype module
Fri, 19 Jun 2009 21:08:07 +0200 haftmann merged
Fri, 19 Jun 2009 17:23:21 +0200 haftmann discontinued ancient tradition to suffix certain ML module names with "_package"
Fri, 19 Jun 2009 18:56:53 +0200 nipkow NewNumberTheory
Mon, 15 Jun 2009 16:13:19 +0200 haftmann authentic syntax for Pow and image
Sat, 13 Jun 2009 16:32:38 +0200 haftmann merged
Sat, 13 Jun 2009 10:01:00 +0200 haftmann quickcheck using generic code generator
Wed, 10 Jun 2009 11:31:36 +0200 wenzelm discontinued escaped symbols;
Mon, 08 Jun 2009 08:38:49 +0200 haftmann method linarith
Sun, 31 May 2009 15:49:35 +0200 wenzelm removed "compress" option from isabelle-process and isabelle usedir -- this is always enabled;
Sun, 31 May 2009 14:15:07 +0200 wenzelm discontinued support for Poly/ML 4.x versions;
Sat, 30 May 2009 15:53:19 +0200 wenzelm eliminated old Attrib.add_attributes (and Attrib.syntax);
Sat, 30 May 2009 15:00:23 +0200 wenzelm eliminated old Method.add_method(s);
Mon, 27 Apr 2009 10:11:44 +0200 haftmann cleaned up theory power further
Fri, 24 Apr 2009 17:45:15 +0200 haftmann funpow and relpow with shared "^^" syntax
Wed, 22 Apr 2009 19:16:02 +0200 haftmann dropped duplication
Wed, 22 Apr 2009 19:12:15 +0200 haftmann code_datatype and power
Mon, 20 Apr 2009 16:28:13 +0200 haftmann merged
Mon, 20 Apr 2009 09:52:16 +0200 haftmann changes in power operations
Fri, 17 Apr 2009 16:41:31 +0200 haftmann formal declaration of undefined parameters after class instantiation
Fri, 17 Apr 2009 15:57:26 +0200 haftmann separated funpow, relpow from power on monoids
Thu, 16 Apr 2009 10:11:34 +0200 haftmann tightended specification of class semiring_div
Mon, 20 Apr 2009 12:26:31 +0200 wenzelm back to non-release mode;
Thu, 02 Apr 2009 15:07:00 +0200 wenzelm some more HOL-Nominal news;
Thu, 02 Apr 2009 14:09:41 +0200 wenzelm some HOL-Nominal news;
Thu, 02 Apr 2009 14:02:34 +0200 wenzelm tuned;
Thu, 02 Apr 2009 13:41:02 +0200 wenzelm misc cleanup and rearrangements for Isabelle2009 release;
Fri, 27 Mar 2009 10:12:55 +0100 haftmann merged
less more (0) -1000 -240 tip