src/HOL/Tools/Qelim/cooper.ML
Mon, 26 Sep 2016 07:56:54 +0200 haftmann syntactic type class for operation mod named after mod;
Wed, 17 Feb 2016 21:51:57 +0100 haftmann dropped various legacy fact bindings
Sun, 13 Dec 2015 21:56:15 +0100 wenzelm more general types Proof.method / context_tactic;
Tue, 17 Nov 2015 12:32:08 +0000 paulson Removed some legacy theorems; minor adjustments to simplification rules; new material on homotopic paths
Sun, 18 Oct 2015 21:30:01 +0200 wenzelm tuned signature;
Sun, 06 Sep 2015 22:14:52 +0200 haftmann formally regenerated
Tue, 01 Sep 2015 17:25:36 +0200 wenzelm tuned -- avoid slightly odd @{cpat};
Mon, 27 Jul 2015 17:44:55 +0200 wenzelm tuned signature;
Sat, 18 Jul 2015 20:47:08 +0200 wenzelm prefer tactics with explicit context;
Sun, 05 Jul 2015 15:02:30 +0200 wenzelm simplified Thm.instantiate and derivatives: the LHS refers to non-certified variables -- this merely serves as index into already certified structures (or is ignored);
Mon, 01 Jun 2015 18:59:21 +0200 haftmann separate class for division operator, with particular syntax added in more specific classes
Sun, 29 Mar 2015 23:08:03 +0200 wenzelm clarified equality of formal entities;
Mon, 09 Mar 2015 11:32:32 +0100 wenzelm eliminated unused arith "verbose" flag -- tools that need options can use the context;
Fri, 06 Mar 2015 15:58:56 +0100 wenzelm Thm.cterm_of and Thm.ctyp_of operate on local context;
Wed, 04 Mar 2015 22:05:01 +0100 wenzelm clarified signature;
Wed, 04 Mar 2015 19:53:18 +0100 wenzelm tuned signature -- prefer qualified names;
Tue, 03 Mar 2015 19:08:04 +0100 traytel eliminated some clones of Proof_Context.cterm_of
Wed, 26 Nov 2014 20:05:34 +0100 wenzelm renamed "pairself" to "apply2", in accordance to @{apply 2};
Wed, 29 Oct 2014 14:40:14 +0100 wenzelm modernized setup;
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
less more (0) -100 -60 tip