src/HOL/Tools/arith_data.ML
Sat, 16 Aug 2014 14:32:26 +0200 wenzelm updated to named_theorems;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Sat, 17 Nov 2012 17:55:52 +0100 wenzelm tuned signature;
Sat, 15 Sep 2012 20:13:25 +0200 haftmann dropped some unused identifiers
Fri, 20 Jul 2012 10:53:25 +0200 huffman make nat_cancel_sums simprocs robust in the presence of schematic variables; add regression tests
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
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;
Fri, 28 Oct 2011 23:41:16 +0200 wenzelm tuned Named_Thms: proper binding;
Sat, 17 Sep 2011 00:37:21 +0200 haftmann tuned
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Thu, 13 Jan 2011 20:54:07 +0100 wenzelm less verbosity -- avoid slightly odd tracing information on warning channel;
Wed, 25 Aug 2010 18:36:22 +0200 wenzelm renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
Sat, 13 Mar 2010 16:37:15 +0100 wenzelm reverted fe9b43a08187 -- "warning" is a perfectly normal way of tactics to emit spurious messages (although "arith" could be less chatty), while "priority" is a special Proof General protocol message;
Sun, 07 Mar 2010 09:57:30 -0800 huffman arith tactic uses 'priority' instead of 'warning' to print messages
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
Sun, 07 Feb 2010 19:33:34 +0100 wenzelm renamed old-style Drule.standard to Drule.export_without_context, to emphasize that this is in no way a standard operation;
Thu, 28 Jan 2010 11:48:49 +0100 haftmann new theory Algebras.thy for generic algebraic structures
Tue, 10 Nov 2009 18:11:23 +0100 wenzelm eliminated some unused/obsolete Args.bang_facts;
Sun, 08 Nov 2009 18:43:42 +0100 wenzelm adapted Theory_Data;
Fri, 30 Oct 2009 13:59:51 +0100 haftmann dedicated theory for loading numeral simprocs
Sat, 17 Oct 2009 00:52:37 +0200 wenzelm explicitly qualify Drule.standard;
Thu, 23 Jul 2009 23:12:21 +0200 wenzelm more @{theory} antiquotations;
Thu, 02 Jul 2009 17:34:14 +0200 wenzelm renamed NamedThmsFun to Named_Thms;
Mon, 06 Apr 2009 15:59:05 +0200 haftmann tuned comment
Thu, 26 Mar 2009 14:14:02 +0100 wenzelm simplified attribute and method setup: eliminating bottom-up styles makes it easier to keep things in one place, and also SML/NJ happy;
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
Fri, 13 Mar 2009 19:17:57 +0100 haftmann moved some generic nonsense to arith_data.ML
Thu, 12 Mar 2009 18:01:26 +0100 haftmann vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
Thu, 01 Jan 2009 23:31:49 +0100 wenzelm normalized some ML type/val aliases;
Wed, 03 Dec 2008 15:58:44 +0100 haftmann made repository layout more coherent with logical distribution structure; stripped some $Id$s
less more (0) tip