src/HOL/Tools/Qelim/cooper.ML
Sat, 16 Aug 2014 16:45:39 +0200 wenzelm clarified order of arith rules;
Sat, 16 Aug 2014 14:32:26 +0200 wenzelm updated to named_theorems;
Sat, 05 Jul 2014 11:01:53 +0200 haftmann prefer ac_simps collections over separate name bindings for add and mult
Fri, 21 Mar 2014 20:33:56 +0100 wenzelm more qualified names;
Tue, 31 Dec 2013 14:29:16 +0100 wenzelm proper context for norm_hhf and derived operations;
Sat, 14 Dec 2013 17:28:05 +0100 wenzelm proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
Tue, 19 Nov 2013 10:05:53 +0100 haftmann eliminiated neg_numeral in favour of - (numeral _)
Fri, 24 May 2013 17:00:46 +0200 wenzelm tuned signature;
Fri, 17 May 2013 20:41:45 +0200 wenzelm proper option quick_and_dirty;
Sat, 11 May 2013 16:57:18 +0200 wenzelm prefer explicitly qualified exceptions, which is particular important for robust handlers;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Fri, 15 Feb 2013 08:31:31 +0100 haftmann two target language numeral types: integer and natural, as replacement for code_numeral;
Mon, 03 Dec 2012 18:13:23 +0100 hoelzl add check to Cooper's algorithm that left-hand of dvd is a numeral
Sat, 14 Apr 2012 23:34:18 +0200 wenzelm refined Cooper.tac / "presburger" method: Subgoal.FOCUS_PARAMS allows to solve more problems with outer quantifiers, e.g "!!x. [| 0 <= (x::int); x div 2 < f x |] ==> x < f x * 2";
Thu, 12 Apr 2012 18:39:19 +0200 wenzelm more standard method setup;
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, 15 Feb 2012 23:19:30 +0100 wenzelm renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in conformance with similar operations in structure Term and Logic;
Fri, 02 Dec 2011 14:54:25 +0100 wenzelm more antiquotations;
Wed, 23 Nov 2011 22:59:39 +0100 wenzelm modernized some old-style infix operations, which were left over from the time of ML proof scripts;
Wed, 19 Oct 2011 15:42:43 +0200 wenzelm inlined @{thms} (ML compile-time) allows to get rid of legacy zadd_ac as well (cf. 49e305100097);
Wed, 10 Aug 2011 20:53:43 +0200 wenzelm old term operations are legacy;
Wed, 29 Jun 2011 17:35:46 +0200 wenzelm modernized some simproc setup;
Thu, 09 Jun 2011 23:12:02 +0200 wenzelm renamed Drule.instantiate to Drule.instantiate_normalize to emphasize its meaning as opposed to plain Thm.instantiate;
Fri, 13 May 2011 22:55:00 +0200 wenzelm proper Proof.context for classical tactics;
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Fri, 08 Apr 2011 13:31:16 +0200 wenzelm explicit structure Syntax_Trans;
Sat, 08 Jan 2011 17:14:48 +0100 wenzelm misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
Mon, 06 Sep 2010 19:13:10 +0200 wenzelm more antiquotations;
Sat, 28 Aug 2010 16:14:32 +0200 haftmann formerly unnamed infix equality now named HOL.eq
Fri, 27 Aug 2010 17:59:40 +0200 wenzelm more antiquotations;
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
Thu, 19 Aug 2010 16:08:59 +0200 haftmann tuned quotes
Thu, 19 Aug 2010 11:02:14 +0200 haftmann use antiquotations for remaining unqualified constants in HOL
Tue, 08 Jun 2010 16:37:22 +0200 haftmann tuned quotes, antiquotations and whitespace
Tue, 25 May 2010 20:28:16 +0200 wenzelm eliminated various catch-all exception patterns, guessing at the concrete exeptions that are intended here;
Sat, 15 May 2010 21:50:05 +0200 wenzelm less pervasive names from structure Thm;
Tue, 11 May 2010 19:00:16 +0200 haftmann represent de-Bruin indices simply by position in list
Tue, 11 May 2010 18:46:03 +0200 haftmann tuned reification functions
Tue, 11 May 2010 18:31:36 +0200 haftmann tuned code; toward a tightended interface with generated code
Mon, 10 May 2010 15:33:32 +0200 haftmann tuned; dropped strange myassoc2
Mon, 10 May 2010 15:24:43 +0200 haftmann stylized COOPER exception
Mon, 10 May 2010 15:21:13 +0200 haftmann simplified oracle
Mon, 10 May 2010 15:00:53 +0200 haftmann shorten names
Mon, 10 May 2010 14:55:06 +0200 haftmann only one module fpr presburger method
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
Mon, 10 May 2010 12:25:49 +0200 haftmann dropped unused bindings; avoid open (documents dependency on generated code more explicitly)
Thu, 06 May 2010 19:27:51 +0200 haftmann merged
Thu, 06 May 2010 16:32:21 +0200 haftmann tuned whitespace; dropped superfluous open
Wed, 05 May 2010 18:25:34 +0200 haftmann farewell to old-style mem infixes -- type inference in situations with mem_int and mem_string should provide enough information to resolve the type of (op =)
Wed, 28 Apr 2010 21:41:05 +0200 haftmann modernized structure name
Sun, 28 Feb 2010 23:51:31 +0100 wenzelm more antiquotations;
Fri, 19 Feb 2010 14:47:01 +0100 haftmann moved remaning class operations from Algebras.thy to Groups.thy
Wed, 10 Feb 2010 14:12:04 +0100 haftmann moved less_eq, less to Orderings.thy; moved abs, sgn to Groups.thy
Mon, 08 Feb 2010 17:12:38 +0100 haftmann renamed OrderedGroup to Groups; split theory Ring_and_Field into Rings Fields
Thu, 28 Jan 2010 11:48:49 +0100 haftmann new theory Algebras.thy for generic algebraic structures
Wed, 21 Oct 2009 12:02:56 +0200 haftmann curried union as canonical list operation
Wed, 21 Oct 2009 08:16:25 +0200 haftmann merged
less more (0) -60 tip