src/HOL/Library/Multiset.thy
Mon, 12 Jul 2010 08:58:13 +0200 haftmann dropped superfluous [code del]s
Fri, 09 Jul 2010 08:11:10 +0200 haftmann nicer xsymbol syntax for fcomp and scomp
Tue, 01 Jun 2010 14:14:02 +0200 blanchet honor xsymbols in Nitpick
Thu, 27 May 2010 16:42:03 +0200 blanchet make Nitpick "show_all" option behave less surprisingly
Mon, 24 May 2010 13:48:57 +0200 haftmann more lemmas
Sat, 22 May 2010 10:12:49 +0200 haftmann localized properties_for_sort
Thu, 13 May 2010 14:34:05 +0200 nipkow Multiset: renamed, added and tuned lemmas;
Wed, 12 May 2010 15:25:02 +0200 nipkow simplified proof
Tue, 04 May 2010 08:55:43 +0200 haftmann locale predicates of classes carry a mandatory "class" prefix
Fri, 16 Apr 2010 21:28:09 +0200 wenzelm replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
Thu, 11 Mar 2010 15:33:45 +0100 blanchet added a mechanism to Nitpick to support custom rendering of terms, and used it for multisets
Sat, 27 Feb 2010 20:57:08 +0100 wenzelm clarified @{const_name} vs. @{const_abbrev};
Wed, 24 Feb 2010 21:55:46 +0100 wenzelm observe standard convention for syntax consts;
Tue, 23 Feb 2010 08:08:23 +0100 haftmann mind the "s"
Mon, 22 Feb 2010 09:15:11 +0100 haftmann ascii syntax for multiset order
Fri, 19 Feb 2010 16:52:00 +0100 haftmann switched notations for pointwise and multiset order
Fri, 05 Feb 2010 14:33:50 +0100 haftmann more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
Fri, 22 Jan 2010 13:38:28 +0100 haftmann cleanup of Multiset.thy: less duplication, tuned and simplified a couple of proofs, less historical organization of sections, conversion from associations lists to multisets, rudimentary code generation
Sun, 25 Oct 2009 00:00:53 +0200 wenzelm adapted Function_Lib (cf. b8cdd3d73022);
Sat, 17 Oct 2009 14:43:18 +0200 wenzelm eliminated hard tabulators, guessing at each author's individual tab-width;
Fri, 28 Aug 2009 19:35:49 +0200 nipkow tuned proofs
Thu, 26 Mar 2009 20:08:55 +0100 wenzelm interpretation/interpret: prefixes are mandatory by default;
Mon, 23 Mar 2009 08:14:24 +0100 haftmann Main is (Complex_Main) base entry point in library theories
Thu, 19 Mar 2009 22:05:00 +0100 wenzelm proper spacing before ML antiquotations -- note that @ may be part of symbolic ML identifiers;
Wed, 11 Mar 2009 08:45:46 +0100 haftmann explicitly delete some code equations
Fri, 13 Feb 2009 23:55:04 +0100 nipkow finiteness lemmas
Fri, 16 Jan 2009 14:58:11 +0100 haftmann migrated class package to new locale implementation
Tue, 30 Dec 2008 11:10:01 +0100 ballarin Merged.
Sun, 14 Dec 2008 18:45:51 +0100 ballarin Ported HOL and HOL-Library to new locales.
Tue, 16 Dec 2008 08:46:07 +0100 krauss method "sizechange" proves termination of functions; added more infrastructure for termination proofs
Mon, 17 Nov 2008 17:00:55 +0100 haftmann tuned unfold_locales invocation
Wed, 29 Oct 2008 11:33:40 +0100 haftmann explicit check for pattern discipline before code translation
Fri, 10 Oct 2008 06:45:53 +0200 haftmann `code func` now just `code`
Fri, 25 Jul 2008 12:03:34 +0200 haftmann added class preorder
Tue, 15 Jul 2008 16:50:09 +0200 ballarin Removed uses of context element includes.
Mon, 07 Jul 2008 08:47:17 +0200 haftmann absolute imports of HOL/*.thy theories
Thu, 26 Jun 2008 10:07:01 +0200 haftmann established Plain theory and image
Tue, 10 Jun 2008 15:30:56 +0200 haftmann removed some dubious code lemmas
Wed, 07 May 2008 10:59:33 +0200 berghofe Instantiated rule expand_fun_eq in proof of set_of_eq_empty_iff, to avoid that
Mon, 07 Apr 2008 15:37:34 +0200 haftmann instantiation replacing primitive instance plus overloaded defs; more conservative type arities
Thu, 28 Feb 2008 14:04:29 +0100 nipkow tuned
Thu, 28 Feb 2008 12:56:31 +0100 wenzelm tuned syntax declaration;
Tue, 26 Feb 2008 16:10:54 +0100 wenzelm tuned document;
Tue, 26 Feb 2008 11:18:43 +0100 bulwahn Added useful general lemmas from the work with the HeapMonad
Fri, 01 Feb 2008 18:01:06 +0100 nipkow modified MCollect syntax
Wed, 30 Jan 2008 17:34:21 +0100 nipkow added multiset comprehension
Wed, 02 Jan 2008 04:10:47 +0100 kleing renamed foldM to fold_mset on general request
Thu, 13 Dec 2007 22:35:45 +0100 kleing removed syntax in locale left_commutative
Thu, 13 Dec 2007 07:09:23 +0100 haftmann changed order in class parameters
Thu, 13 Dec 2007 06:51:22 +0100 kleing a fold operation for multisets + more lemmas
Mon, 10 Dec 2007 11:24:12 +0100 haftmann switched import from Main to List
Fri, 07 Dec 2007 15:07:59 +0100 haftmann instantiation target rather than legacy instance
Fri, 30 Nov 2007 11:51:22 +0100 nipkow added {#.,.,...#}
Fri, 26 Oct 2007 21:22:19 +0200 haftmann changed order of class parameters
Tue, 23 Oct 2007 23:27:23 +0200 nipkow went back to >0
Sun, 21 Oct 2007 22:33:35 +0200 nipkow More changes from >0 to ~=0::nat
Sun, 21 Oct 2007 14:53:44 +0200 nipkow Eliminated most of the neq0_conv occurrences. As a result, many
Sun, 29 Jul 2007 14:29:49 +0200 wenzelm simplified ResAtpset via NamedThmsFun;
Wed, 11 Jul 2007 11:24:36 +0200 berghofe Restored set notation.
Fri, 06 Jul 2007 23:26:13 +0200 nipkow more interpretations
less more (0) -100 -60 tip