src/HOL/Tools/Qelim/cooper.ML
Thu, 14 Oct 2021 16:03:20 +0200 wenzelm clarified signature;
Sat, 02 Oct 2021 12:04:14 +0200 wenzelm proper term operation Term.dest_abs;
Fri, 10 Sep 2021 14:59:19 +0200 wenzelm clarified signature: more scalable operations;
Fri, 09 Apr 2021 22:06:59 +0200 wenzelm support for ML special forms: modified evaluation similar to Scheme;
Tue, 16 Jun 2020 08:41:39 +0000 haftmann more specific thm reference
Fri, 04 Jan 2019 23:22:53 +0100 wenzelm isabelle update -u control_cartouches;
Mon, 24 Sep 2018 14:30:09 +0200 nipkow Prefix form of infix with * on either side no longer needs special treatment
Sun, 15 Jul 2018 10:40:45 +0100 paulson last bit of renaming
Thu, 01 Feb 2018 13:55:10 +0100 wenzelm clarified signature;
Thu, 11 Jan 2018 13:48:17 +0100 wenzelm uniform use of Standard ML op-infix -- eliminated warnings;
Wed, 10 Jan 2018 15:25:09 +0100 nipkow ran isabelle update_op on all sources
Sat, 02 Dec 2017 16:50:53 +0000 haftmann more simplification rules
Sat, 17 Dec 2016 15:22:14 +0100 haftmann reoriented congruence rules in non-explosive direction
Sat, 17 Dec 2016 15:22:13 +0100 haftmann tuned fact references
Sun, 16 Oct 2016 09:31:05 +0200 haftmann clarified theorem names
Sun, 16 Oct 2016 09:31:05 +0200 haftmann eliminated irregular aliasses
Sun, 16 Oct 2016 09:31:05 +0200 haftmann more standardized theorem names for facts involving the div and mod identity
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;
less more (0) -100 -60 tip