src/HOL/Set.thy
Thu, 16 Feb 2012 16:02:02 +0100 bulwahn removing unnecessary premise from diff_single_insert
Tue, 14 Feb 2012 17:11:33 +0100 wenzelm eliminated obsolete aliases;
Sat, 07 Jan 2012 20:44:23 +0100 haftmann massaging of code setup for sets
Fri, 06 Jan 2012 21:48:45 +0100 haftmann incorporated various theorems from theory More_Set into corpus
Fri, 06 Jan 2012 16:45:19 +0100 wenzelm tuned -- more direct @{type_name set} (NB: binder_tr' retains the original non-syntax type for the bound/free variable);
Sun, 01 Jan 2012 15:44:15 +0100 haftmann interaction of set operations for execution and membership predicate
Sun, 01 Jan 2012 11:28:45 +0100 haftmann cleanup of code declarations
Thu, 29 Dec 2011 14:23:40 +0100 haftmann fundamental theorems on Set.bind
Thu, 29 Dec 2011 10:47:54 +0100 haftmann semiring_numeral_0_eq_0, semiring_numeral_1_eq_1 now [simp], superseeding corresponding simp rules on type nat
Mon, 26 Dec 2011 18:32:43 +0100 haftmann moved various set operations to theory Set (resp. Product_Type)
Sat, 24 Dec 2011 15:53:07 +0100 haftmann `set` is now a proper type constructor; added operation for set monad
Sat, 17 Dec 2011 13:08:03 +0100 wenzelm tuned signature;
Sun, 27 Nov 2011 22:03:22 +0100 wenzelm just one data slot per module;
Thu, 24 Nov 2011 21:01:06 +0100 wenzelm modernized some old-style infix operations, which were left over from the time of ML proof scripts;
Sun, 20 Nov 2011 21:07:10 +0100 wenzelm eliminated obsolete "standard";
Sun, 16 Oct 2011 14:48:00 +0200 haftmann hide not_member as also member
Sun, 09 Oct 2011 08:30:48 +0200 huffman Set.thy: remove redundant [simp] declarations
Tue, 06 Sep 2011 14:25:16 +0200 nipkow added new lemmas
Thu, 25 Aug 2011 14:06:34 +0200 krauss lemma Compl_insert: "- insert x A = (-A) - {x}"
Wed, 17 Aug 2011 18:05:31 +0200 wenzelm modernized signature of Term.absfree/absdummy;
Sun, 24 Jul 2011 21:27:25 +0200 haftmann more coherent structure in and across theories
Mon, 18 Jul 2011 21:15:51 +0200 haftmann moved lemmas to appropriate theory
Sun, 17 Jul 2011 19:48:02 +0200 haftmann moving UNIV = ... equations to their proper theories
Thu, 14 Jul 2011 00:20:43 +0200 haftmann tuned lemma positions and proofs
Fri, 22 Apr 2011 15:05:04 +0200 wenzelm misc tuning and simplification;
Fri, 22 Apr 2011 14:30:32 +0200 wenzelm proper context for Quantifier1 simprocs (avoid bad ProofContext.init_global from abc655166d61);
Fri, 22 Apr 2011 13:58:13 +0200 wenzelm modernized Quantifier1 simproc setup;
Fri, 08 Apr 2011 14:20:57 +0200 wenzelm discontinued special treatment of structure Mixfix;
Fri, 08 Apr 2011 13:31:16 +0200 wenzelm explicit structure Syntax_Trans;
Wed, 30 Mar 2011 11:32:52 +0200 bulwahn renewing specifications in HOL: replacing types by type_synonym
Fri, 10 Dec 2010 16:10:50 +0100 haftmann moved most fundamental lemmas upwards
Wed, 08 Dec 2010 15:05:46 +0100 haftmann bot comes before top, inf before sup etc.
Wed, 08 Dec 2010 13:34:51 +0100 haftmann primitive definitions of bot/top/inf/sup for bool and fun are named with canonical suffix `_def` rather than `_eq`;
Thu, 02 Dec 2010 14:34:58 +0100 hoelzl Move SUP_commute, SUP_less_iff to HOL image;
Tue, 23 Nov 2010 14:14:17 +0100 hoelzl Move some missing lemmas from Andrei Popescus 'Ordinals and Cardinals' AFP entry to the HOL-image.
Fri, 01 Oct 2010 16:05:25 +0200 haftmann constant `contents` renamed to `the_elem`
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
Wed, 08 Sep 2010 10:45:55 +0200 nipkow put expand_(fun/set)_eq back in as synonyms, for compatibility
Tue, 07 Sep 2010 10:05:19 +0200 nipkow expand_fun_eq -> ext_iff
Sat, 28 Aug 2010 16:14:32 +0200 haftmann formerly unnamed infix equality now named HOL.eq
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 20:51:17 +0200 haftmann formerly unnamed infix impliciation now named HOL.implies
Wed, 25 Aug 2010 18:36:22 +0200 wenzelm renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
Mon, 23 Aug 2010 12:13:58 +0200 blanchet "no_atp" fact that leads to unsound proofs
Mon, 23 Aug 2010 11:56:30 +0200 blanchet "no_atp" a few facts that often lead to unsound proofs
Mon, 12 Jul 2010 10:48:37 +0200 haftmann dropped superfluous [code del]s
Thu, 01 Jul 2010 16:54:42 +0200 haftmann qualified constants Set.member and Set.Collect
Tue, 08 Jun 2010 16:37:19 +0200 haftmann qualified types "+" and nat; qualified constants Ball, Bex, Suc, curry; modernized some specifications
Sun, 28 Mar 2010 12:50:38 -0700 huffman use lattice theorems to prove set theorems
Thu, 18 Mar 2010 12:58:52 +0100 blanchet now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
Thu, 04 Mar 2010 15:44:06 +0100 hoelzl Added vimage_inter_cong
Mon, 01 Mar 2010 13:40:23 +0100 haftmann replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
Thu, 11 Feb 2010 23:00:22 +0100 wenzelm modernized translations;
Thu, 04 Feb 2010 14:45:08 +0100 hoelzl Changed 'bounded unique existential quantifiers' from a constant to syntax translation.
Thu, 28 Jan 2010 11:48:49 +0100 haftmann new theory Algebras.thy for generic algebraic structures
Wed, 30 Dec 2009 10:24:53 +0100 krauss killed a few warnings
Fri, 27 Nov 2009 16:26:23 +0100 berghofe Removed eq_to_mono2, added not_mono.
Mon, 09 Nov 2009 15:50:15 +0000 paulson New theory Probability/Borel.thy, and some associated lemmas
Wed, 21 Oct 2009 11:19:11 +0100 paulson merged
Tue, 20 Oct 2009 16:32:51 +0100 paulson Some new lemmas concerning sets
less more (0) -100 -60 tip