src/HOL/SetInterval.thy
Wed, 04 Mar 2009 10:45:52 +0100 Merge.
Mon, 23 Feb 2009 16:25:52 -0800 make proofs work whether or not One_nat_def is a simp rule; replace 1 with Suc 0 in the rhs of some simp rules
Wed, 18 Feb 2009 11:18:01 +0000 Syntactic support for products over set intervals
Sun, 15 Feb 2009 11:26:38 +0100 more finiteness
Mon, 02 Feb 2009 13:56:23 +0100 fixed proposition slip
Wed, 28 Jan 2009 16:29:16 +0100 Replaced group_ and ring_simps by algebra_simps;
Wed, 19 Nov 2008 17:54:55 +0100 Added new fold operator and renamed the old oe to fold_image.
Mon, 01 Sep 2008 19:16:40 +0200 cleaned up code generation for {.._} and {..<_}
Sat, 19 Jul 2008 19:27:13 +0200 added verification framework for the HeapMonad and quicksort as example for this framework
Thu, 21 Feb 2008 17:33:58 +0100 moved bij_betw from Library/FuncSet to Fun, redistributed some lemmas, and
Fri, 15 Feb 2008 16:09:12 +0100 <= and < on nat no longer depend on wellfounded relations
Tue, 15 Jan 2008 16:19:23 +0100 joined theories IntDef, Numeral, IntArith to theory Int
Thu, 06 Dec 2007 16:36:21 +0100 dropped legacy bindings
Tue, 16 Oct 2007 23:12:45 +0200 global class syntax
Fri, 05 Oct 2007 08:38:09 +0200 added lemmas
Sat, 29 Sep 2007 08:58:51 +0200 proper syntax during class specification
Mon, 24 Sep 2007 19:34:55 +0200 localized { .. } (but only a few thms)
Tue, 28 Aug 2007 15:34:15 +0200 added (code) lemmas for setsum and foldl
Wed, 15 Aug 2007 12:52:56 +0200 ATP blacklisting is now in theory data, attribute noatp
Mon, 25 Jun 2007 15:19:18 +0200 removed redundant lemmas
Sat, 23 Jun 2007 19:33:22 +0200 tuned and renamed group_eq_simps and ring_eq_simps
Wed, 20 Jun 2007 05:18:39 +0200 change simp rules for of_nat to work like int did previously (reorient of_nat_Suc, remove of_nat_mult [simp]); preserve original variable names in legacy int theorems
Sun, 17 Jun 2007 18:47:03 +0200 tuned laws for cancellation in divisions for fields.
Fri, 15 Jun 2007 15:10:32 +0200 made divide_self a simp rule
Wed, 06 Jun 2007 17:01:33 +0200 generalize class constraints on some lemmas
Mon, 16 Apr 2007 04:02:15 +0200 generalized type of lemma geometric_sum
Thu, 23 Nov 2006 20:34:21 +0100 prefer antiquotations over LaTeX macros;
Wed, 26 Jul 2006 19:23:04 +0200 linear arithmetic splits certain operators (e.g. min, max, abs)
Tue, 02 May 2006 20:42:34 +0200 actually removed old stuff;
Wed, 26 Apr 2006 07:01:33 +0200 moved arithmetic series to geometric series in SetInterval
Sun, 09 Apr 2006 14:20:23 +0200 Removed old set interval syntax.
Sun, 19 Feb 2006 13:21:32 +0100 * added Library/ASeries (sum of arithmetic series with instantiation to nat and int)
Sun, 12 Feb 2006 10:42:19 +0100 * moved ThreeDivides from Isar_examples to better suited HOL/ex
Thu, 29 Sep 2005 15:31:34 +0200 Added a few lemmas
Fri, 26 Aug 2005 10:01:06 +0200 Lemmas on dvd, power and finite summation added or strengthened.
Thu, 07 Jul 2005 12:39:17 +0200 linear arithmetic now takes "&" in assumptions apart.
Fri, 27 May 2005 16:24:48 +0200 Locale expressions: rename with optional mixfix syntax.
Mon, 23 May 2005 19:39:45 +0200 tuned setsum rewrites
Mon, 23 May 2005 11:06:41 +0200 simplifier trace info; Suc-intervals
Mon, 02 May 2005 18:59:50 +0200 turned 2 lemmas into simp rules
Wed, 02 Mar 2005 12:06:15 +0100 another reorganization of setsums and intervals
Tue, 01 Mar 2005 18:48:52 +0100 integrated Jeremy's FiniteLib
Mon, 21 Feb 2005 19:23:46 +0100 more fine tuniung
Mon, 21 Feb 2005 15:04:10 +0100 comprehensive cleanup, replacing sumr by setsum
Fri, 17 Dec 2004 10:15:46 +0100 removed two looping simplifications in SetInterval.thy; deleted the .ML file
Sun, 12 Dec 2004 16:25:47 +0100 REorganized Finite_Set
Tue, 19 Oct 2004 18:18:45 +0200 converted some induct_tac to induct
Wed, 18 Aug 2004 11:09:40 +0200 import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 New theory header syntax.
Fri, 16 Jul 2004 17:33:12 +0200 Fine-tuned sum syntax.
Fri, 16 Jul 2004 11:46:59 +0200 Added nice latex syntax.
Thu, 15 Jul 2004 15:39:40 +0200 more syntax
Thu, 15 Jul 2004 15:32:32 +0200 redefining sumr to be a translation to setsum
Thu, 15 Jul 2004 13:11:34 +0200 Moved to new m<..<n syntax for set intervals.
Wed, 14 Jul 2004 10:25:03 +0200 added {0::nat..n(} = {..n(}
Tue, 13 Jul 2004 12:32:01 +0200 Got rid of Summation and made it a translation into setsum instead.
Sat, 29 May 2004 16:47:06 +0200 \<^bsub>/\<^esub> syntax: unbreakable block;
Sat, 01 May 2004 22:04:14 +0200 improved subscript syntax;
Fri, 16 Apr 2004 04:07:10 +0200 tuned document;
Thu, 25 Mar 2004 10:32:21 +0100 new material from Avigad