src/HOL/Set.thy
Thu, 27 Feb 2014 16:07:21 +0000 paulson A bit of tidying up
Sat, 25 Jan 2014 22:06:07 +0100 wenzelm explicit eigen-context for attributes "where", "of", and corresponding read_instantiate, instantiate_tac;
Sun, 12 Jan 2014 14:32:22 +0100 wenzelm tuned signature;
Fri, 18 Oct 2013 10:43:20 +0200 blanchet killed most "no_atp", to make Sledgehammer more complete
Mon, 02 Sep 2013 17:12:59 +0200 nipkow added lemmas
Sat, 25 May 2013 15:37:53 +0200 wenzelm syntax translations always depend on context;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Fri, 12 Apr 2013 17:21:51 +0200 wenzelm modifiers for classical wrappers operate on Proof.context instead of claset;
Tue, 12 Mar 2013 07:51:10 +0100 nipkow extended set comprehension notation with {pttrn : A . P}
Tue, 05 Mar 2013 10:16:15 +0100 nipkow more lemmas about intervals
Sun, 17 Feb 2013 21:29:30 +0100 haftmann Sieve of Eratosthenes
Mon, 17 Dec 2012 17:19:21 +0100 nipkow made element and subset relations non-associative (just like all orderings)
Tue, 09 Oct 2012 16:57:58 +0200 kuncar rename Set.project to Set.filter - more appropriate name
Sat, 29 Sep 2012 18:23:46 +0200 wenzelm more explicit Syntax_Trans.mark_bound_abs/mark_bound_body: preserve type information for show_markup;
Fri, 06 Apr 2012 19:18:00 +0200 haftmann tuned
Mon, 12 Mar 2012 15:11:24 +0100 noschinl tuned simpset
Fri, 09 Mar 2012 21:50:27 +0100 haftmann beautified
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;
less more (0) -100 -60 tip