src/HOL/Groebner_Basis.thy
Mon, 04 Nov 2013 20:10:10 +0100 dropped dead code
Wed, 22 Aug 2012 22:55:41 +0200 prefer ML_file over old uses;
Thu, 12 Apr 2012 18:39:19 +0200 more standard method setup;
Tue, 27 Mar 2012 19:21:05 +0200 remove redundant lemmas
Tue, 27 Mar 2012 15:34:36 +0200 remove duplicate [algebra] declarations
Tue, 27 Mar 2012 15:34:04 +0200 generalize more div/mod lemmas
Tue, 27 Mar 2012 15:27:49 +0200 generalize some theorems about div/mod
Tue, 27 Mar 2012 14:49:56 +0200 remove redundant lemmas
Fri, 28 Oct 2011 23:41:16 +0200 tuned Named_Thms: proper binding;
Fri, 07 May 2010 16:12:25 +0200 delete Groebner_Basis directory -- only one file left
Fri, 07 May 2010 15:05:52 +0200 split of semiring normalization from Groebner theory; moved field_comp_conv to Numeral_Simproces
Thu, 06 May 2010 23:11:57 +0200 proper sublocales; no free-floating ML sections
Thu, 06 May 2010 18:16:07 +0200 moved generic lemmas to appropriate places
Thu, 06 May 2010 17:59:19 +0200 dropped duplicate comp_arith
Thu, 06 May 2010 17:55:11 +0200 avoid references to groebner bases in names which have no references to groebner bases
Thu, 06 May 2010 16:40:02 +0200 moved presimplification rules for algebraic methods into named thms functor
Thu, 06 May 2010 16:32:20 +0200 dropped auxiliary method sring_norm; integrated normalizer.ML and normalizer_data.ML
Wed, 05 May 2010 16:53:21 +0200 moved nat_arith ot Nat_Numeral: clarified normalizer setup
Wed, 05 May 2010 16:46:19 +0200 dropped unused file
Mon, 26 Apr 2010 15:37:50 +0200 use new classes (linordered_)field_inverse_zero
Mon, 26 Apr 2010 11:34:17 +0200 class division_ring_inverse_zero
Fri, 23 Apr 2010 15:17:59 +0200 dequalified fact name
Sun, 28 Feb 2010 23:51:31 +0100 more antiquotations;
Thu, 18 Feb 2010 14:21:44 -0800 get rid of many duplicate simp rule warnings
Wed, 10 Feb 2010 14:12:04 +0100 moved less_eq, less to Orderings.thy; moved abs, sgn to Groups.thy
Wed, 10 Feb 2010 08:49:26 +0100 moved constants inverse and divide to Ring.thy
Mon, 08 Feb 2010 17:12:38 +0100 renamed OrderedGroup to Groups; split theory Ring_and_Field into Rings Fields
Thu, 28 Jan 2010 11:48:49 +0100 new theory Algebras.thy for generic algebraic structures
Fri, 30 Oct 2009 14:00:43 +0100 combined former theories Divides and IntDiv to one theory Divides
Wed, 28 Oct 2009 19:09:47 +0100 moved theory Divides after theory Nat_Numeral; tuned some proof texts
Wed, 24 Jun 2009 09:41:14 +0200 corrected and unified thm names
Fri, 08 May 2009 09:48:07 +0200 modules numeral_simprocs, nat_numeral_simprocs; proper structures for numeral simprocs
Tue, 28 Apr 2009 15:50:30 +0200 stripped class recpower further
Wed, 15 Apr 2009 15:30:39 +0200 theory NatBin now named Nat_Numeral
Sun, 05 Apr 2009 19:21:51 +0100 More precise treatement of rational constants by the normalizer for fields
Sun, 05 Apr 2009 05:07:10 +0100 now deals with devision in fields
Thu, 26 Mar 2009 20:08:55 +0100 interpretation/interpret: prefixes are mandatory by default;
Sun, 22 Mar 2009 20:46:11 +0100 dropped theory Arith_Tools
Mon, 16 Mar 2009 18:24:30 +0100 simplified method setup;
Fri, 13 Mar 2009 19:58:26 +0100 unified type Proof.method and pervasive METHOD combinators;
Wed, 04 Mar 2009 11:05:29 +0100 Merge.
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
Sat, 21 Feb 2009 20:52:30 +0100 Removed subsumed lemmas
Sat, 21 Feb 2009 09:58:26 +0100 removed redundant thms
Fri, 20 Feb 2009 23:46:03 +0100 Removed redundant lemmas
Fri, 20 Feb 2009 20:50:49 +0100 removed subsumed lemmas
Wed, 28 Jan 2009 16:29:16 +0100 Replaced group_ and ring_simps by algebra_simps;
Sun, 14 Dec 2008 18:45:51 +0100 Ported HOL and HOL-Library to new locales.
Fri, 12 Dec 2008 20:10:22 +0100 Merged.
Thu, 11 Dec 2008 18:30:26 +0100 Conversion of HOL-Main and ZF to new locales.
Tue, 09 Dec 2008 20:36:20 -0800 separate neg_simps from rel_simps
Thu, 04 Dec 2008 16:05:45 -0800 remove duplicated lemmas
Thu, 04 Dec 2008 13:30:09 -0800 include iszero_simps in lemmas comp_arith
Thu, 20 Nov 2008 00:03:47 +0100 Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
Mon, 17 Nov 2008 17:00:55 +0100 tuned unfold_locales invocation
Tue, 28 Oct 2008 11:03:07 +0100 Removed 'includes meta_term_syntax' and 'includes meta_conjunction_syntax'.
Mon, 29 Sep 2008 12:31:59 +0200 clarified dependencies between arith tools
Mon, 21 Jul 2008 13:36:39 +0200 Relevant rules added to algebra's context
Fri, 28 Mar 2008 19:43:54 +0100 avoid rebinding of existing facts;