src/HOL/Finite_Set.thy
Fri, 29 Nov 2013 08:26:45 +0100 set_comprehension_pointfree simproc causes to many surprises if enabled by default
Sun, 24 Nov 2013 00:31:50 +0000 polished some ancient proofs
Tue, 12 Nov 2013 19:28:54 +0100 add finite_select_induct; move generic lemmas from MV_Analysis/Linear_Algebra to the HOL image
Fri, 18 Oct 2013 10:43:21 +0200 killed more "no_atp"s
Fri, 18 Oct 2013 10:43:20 +0200 killed most "no_atp", to make Sledgehammer more complete
Tue, 24 Sep 2013 13:35:27 +0200 added lemmas
Tue, 03 Sep 2013 01:12:40 +0200 tuned proofs -- clarified flow of facts wrt. calculation;
Tue, 13 Aug 2013 16:25:47 +0200 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
Thu, 04 Apr 2013 22:29:59 +0200 convenient induction rule
Wed, 03 Apr 2013 10:15:43 +0200 generalized lemma fold_image thanks to Peter Lammich
Tue, 26 Mar 2013 21:53:56 +0100 more uniform style for interpretation and sublocale declarations
Sat, 23 Mar 2013 20:50:39 +0100 fundamental revision of big operators on sets
Sat, 23 Mar 2013 17:11:06 +0100 locales for abstract orders
Wed, 27 Feb 2013 13:43:04 +0100 added lemma
Wed, 10 Oct 2012 16:19:52 +0200 merged
Wed, 10 Oct 2012 10:47:43 +0200 moving simproc from Finite_Set to more appropriate Product_Type theory
Tue, 09 Oct 2012 16:58:36 +0200 use Set.filter instead of Finite_Set.filter, which is removed then
Tue, 09 Oct 2012 16:57:58 +0200 rename Set.project to Set.filter - more appropriate name
Wed, 10 Oct 2012 15:39:01 +0200 added some ad-hoc namespace prefixes to avoid duplicate facts;
Mon, 08 Oct 2012 12:03:49 +0200 consolidated names of theorems on composition;
Sat, 06 Oct 2012 16:03:41 +0200 congruence rule for Finite_Set.fold
Sat, 06 Oct 2012 11:08:52 +0200 alternative simplification of ^^ to the righthand side;
Wed, 22 Aug 2012 22:55:41 +0200 prefer ML_file over old uses;
Wed, 01 Aug 2012 15:32:36 +0200 removed junk;
Tue, 31 Jul 2012 13:55:39 +0200 more set operations expressed by Finite_Set.fold
Tue, 03 Jul 2012 09:25:42 +0200 add finiteness lemmas for 'a * 'b and 'a set
Mon, 25 Jun 2012 18:21:18 +0200 merged, resolving conflict with 87c831e30f0a;
Mon, 25 Jun 2012 17:41:20 +0200 tuned proofs -- prefer direct "rotated" instead of old-style COMP;
Mon, 25 Jun 2012 15:14:07 +0200 ignore morphism more explicitly;
Mon, 25 Jun 2012 16:03:14 +0200 adding set comprehension simproc to code generation's preprocessing to generate code for some set comprehensions;
Wed, 20 Jun 2012 16:54:08 +0200 Integrated set comprehension pointfree simproc.
Fri, 01 Jun 2012 11:53:58 +0200 remove duplicate lemma card_unit in favor of Finite_Set.card_UNIV_unit
Fri, 30 Mar 2012 14:00:18 +0200 rephrase lemma card_Pow using '2' instead of 'Suc (Suc 0)'
Fri, 30 Mar 2012 08:04:28 +0200 move lemma card_UNIV_bool from Nat_Numeral.thy to Finite_Set.thy
Tue, 13 Mar 2012 13:31:26 +0100 tuned proofs -- eliminated pointless chaining of facts after 'interpret';
Fri, 06 Jan 2012 21:48:45 +0100 incorporated various theorems from theory More_Set into corpus
Thu, 29 Dec 2011 13:41:41 +0100 qualified Finite_Set.fold
Sat, 24 Dec 2011 15:53:08 +0100 finite type class instance for `set`
Tue, 18 Oct 2011 15:27:18 +0200 tuned
Wed, 14 Sep 2011 10:08:52 -0400 renamed Complete_Lattices lemmas, removed legacy names
Tue, 13 Sep 2011 16:22:01 +0200 tune proofs
Mon, 12 Sep 2011 07:55:43 +0200 new fastforce replacing fastsimp - less confusing name
Tue, 06 Sep 2011 22:04:14 +0200 merged
Mon, 05 Sep 2011 07:49:31 +0200 tuned
Tue, 06 Sep 2011 14:25:16 +0200 added new lemmas
Wed, 27 Jul 2011 19:34:30 +0200 finite vimage on arbitrary domains
Sun, 17 Jul 2011 19:48:02 +0200 moving UNIV = ... equations to their proper theories
Fri, 20 May 2011 12:35:44 +0200 tuned proofs
Fri, 20 May 2011 12:07:17 +0200 point-free characterization of operations on finite sets
Fri, 20 May 2011 11:44:16 +0200 names of fold_set locales resemble name of characteristic property more closely
Fri, 20 May 2011 08:16:56 +0200 use point-free characterization for locale fun_left_comm_idem
Sat, 14 May 2011 18:26:25 +0200 use pointfree characterisation for fold_set locale
Thu, 12 May 2011 11:03:48 +0200 more uniform naming of lemma
Thu, 07 Apr 2011 13:01:27 +0200 dropped unused lemmas; proper Isar proof
Sun, 03 Apr 2011 11:40:32 +0200 tuned proofs
Sat, 02 Apr 2011 18:07:29 +0200 tuned proof
Thu, 17 Mar 2011 09:58:13 +0100 tuned lemma
Wed, 16 Mar 2011 19:50:56 +0100 added lemmas
Fri, 21 Jan 2011 09:44:12 +0100 moved theorem
Fri, 21 Jan 2011 09:41:59 +0100 restructured theory;