src/HOL/Presburger.thy
Tue, 27 Mar 2012 19:21:05 +0200 huffman remove redundant lemmas
Tue, 27 Mar 2012 14:49:56 +0200 huffman remove redundant lemmas
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
Wed, 09 Nov 2011 17:08:40 +0100 wenzelm avoid inconsistent sort constraints;
Mon, 12 Sep 2011 07:55:43 +0200 nipkow new fastforce replacing fastsimp - less confusing name
Tue, 06 Sep 2011 19:03:41 -0700 huffman avoid using legacy theorem names
Mon, 10 May 2010 15:00:53 +0200 haftmann shorten names
Mon, 10 May 2010 14:57:04 +0200 haftmann updated references to ML files
Mon, 10 May 2010 14:55:06 +0200 haftmann only one module fpr presburger method
Mon, 10 May 2010 14:18:41 +0200 haftmann tuned theory text; dropped unused lemma
Mon, 10 May 2010 14:11:50 +0200 haftmann one structure is better than three
Mon, 10 May 2010 13:58:18 +0200 haftmann less complex organization of cooper source code
Fri, 07 May 2010 09:51:55 +0200 haftmann moved lemma zdvd_period to theory Int
Thu, 18 Feb 2010 14:21:44 -0800 huffman get rid of many duplicate simp rule warnings
Mon, 08 Feb 2010 17:12:38 +0100 haftmann renamed OrderedGroup to Groups; split theory Ring_and_Field into Rings Fields
Thu, 29 Oct 2009 11:41:36 +0100 haftmann moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
Thu, 10 Sep 2009 14:07:58 +0200 haftmann cleanedup theorems all_nat ex_nat
Wed, 24 Jun 2009 09:41:14 +0200 nipkow corrected and unified thm names
Mon, 23 Mar 2009 19:01:16 +0100 haftmann moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
Sun, 22 Mar 2009 20:46:12 +0100 haftmann moved import of module qelim to theory Presburger
Mon, 16 Mar 2009 18:24:30 +0100 wenzelm simplified method setup;
Fri, 13 Mar 2009 19:58:26 +0100 wenzelm unified type Proof.method and pervasive METHOD combinators;
Wed, 04 Mar 2009 11:05:29 +0100 blanchet Merge.
Wed, 04 Mar 2009 10:45:52 +0100 blanchet Merge.
Fri, 20 Feb 2009 23:46:03 +0100 nipkow Removed redundant lemmas
Fri, 20 Feb 2009 20:50:49 +0100 nipkow removed subsumed lemmas
Mon, 02 Feb 2009 13:56:22 +0100 haftmann dropped Id
Wed, 28 Jan 2009 16:29:16 +0100 nipkow Replaced group_ and ring_simps by algebra_simps;
Wed, 03 Dec 2008 21:50:36 -0800 huffman enable eq_bin_simps for simplifying equalities on numerals
Mon, 29 Sep 2008 12:31:59 +0200 haftmann clarified dependencies between arith tools
Thu, 18 Sep 2008 19:39:44 +0200 wenzelm simplified oracle interface;
Mon, 21 Jul 2008 13:36:59 +0200 chaieb Tuned and simplified proofs
Fri, 18 Jul 2008 18:25:53 +0200 haftmann moved op dvd to theory Ring_and_Field; generalized a couple of lemmas
Fri, 11 Jul 2008 09:02:22 +0200 haftmann separate class dvd for divisibility predicate
Wed, 02 Apr 2008 15:58:27 +0200 haftmann moved some code lemmas for Numerals to other theories
Wed, 27 Feb 2008 14:39:50 +0100 chaieb loads Tools/Qelim/qelim.ML
Sun, 17 Feb 2008 06:49:53 +0100 huffman New simpler representation of numerals, using Bit0 and Bit1 instead of BIT, B0, and B1
Sat, 16 Feb 2008 02:01:13 +0100 huffman added lemma lists {normalize,succ,pred,minus,add,mult}_bin_simps
Tue, 15 Jan 2008 16:19:23 +0100 haftmann joined theories IntDef, Numeral, IntArith to theory Int
Tue, 30 Oct 2007 08:45:54 +0100 haftmann continued localization
Fri, 12 Oct 2007 08:20:46 +0200 haftmann class div inherits from class times
Wed, 22 Aug 2007 17:13:42 +0200 chaieb tuned;
Tue, 31 Jul 2007 19:40:25 +0200 wenzelm proper context for cooper_tac within arith;
Tue, 31 Jul 2007 00:56:26 +0200 wenzelm arith method setup: proper context;
Thu, 19 Jul 2007 21:47:43 +0200 haftmann code lemma for of_int
Tue, 10 Jul 2007 09:23:11 +0200 haftmann moved lemma zdvd_period here
Sat, 23 Jun 2007 19:33:22 +0200 nipkow tuned and renamed group_eq_simps and ring_eq_simps
Thu, 21 Jun 2007 23:49:26 +0200 huffman section headings
Thu, 21 Jun 2007 20:48:47 +0200 wenzelm moved Presburger setup back to Presburger.thy;
Thu, 21 Jun 2007 15:42:14 +0200 wenzelm adapted tool setup;
Wed, 20 Jun 2007 17:28:55 +0200 huffman remove simp attribute from of_nat_diff, for backward compatibility with zdiff_int
Wed, 20 Jun 2007 05:06:56 +0200 huffman section headings
Sun, 17 Jun 2007 13:39:27 +0200 chaieb moved lemma all_not_ex to HOL.thy ; tuned proofs
Thu, 14 Jun 2007 22:59:39 +0200 chaieb Added some lemmas to default presburger simpset; tuned proofs
Thu, 14 Jun 2007 18:33:31 +0200 wenzelm tuned proofs: avoid implicit prems;
Wed, 13 Jun 2007 03:31:11 +0200 huffman removed constant int :: nat => int;
Tue, 12 Jun 2007 10:15:40 +0200 chaieb Method now takes theorems to be added or deleted from a simpset for simplificatio before the core method starts
Mon, 11 Jun 2007 11:06:00 +0200 chaieb A new and cleaned up Theory for QE. for Presburger arithmetic
Tue, 05 Jun 2007 16:26:06 +0200 wenzelm tuned comments;
Thu, 31 May 2007 18:16:52 +0200 wenzelm moved Integ files to canonical place;
less more (0) -60 tip