src/HOL/Integ/NatBin.thy
Thu, 24 May 2007 22:55:53 +0200 nipkow *** empty log message ***
Thu, 24 May 2007 16:52:54 +0200 obua Squared things out.
Thu, 24 May 2007 07:27:44 +0200 nipkow Introduced new classes monoid_add and group_add
Sun, 20 May 2007 17:30:21 +0200 huffman add lemma power2_eq_imp_eq
Tue, 08 May 2007 01:10:55 +0200 huffman add lemmas power2_le_imp_le and power2_less_imp_less
Thu, 26 Apr 2007 13:33:09 +0200 haftmann slightly tuned
Fri, 02 Mar 2007 15:43:24 +0100 haftmann simplified code generator setup
Wed, 14 Feb 2007 10:06:15 +0100 haftmann cleanup
Wed, 31 Jan 2007 16:05:10 +0100 haftmann dropped lemma duplicates in HOL.thy
Fri, 26 Jan 2007 10:24:12 +0100 paulson simplification of Suc/numeral combinations with min, max
Tue, 09 Jan 2007 19:08:56 +0100 haftmann named preprocessors
Fri, 17 Nov 2006 02:20:03 +0100 wenzelm more robust syntax for definition/abbreviation/notation;
Tue, 07 Nov 2006 11:47:57 +0100 wenzelm renamed 'const_syntax' to 'notation';
Tue, 07 Nov 2006 09:33:47 +0100 krauss * Added annihilation axioms ("x * 0 = 0") to axclass semiring_0.
Mon, 02 Oct 2006 23:00:51 +0200 haftmann tuned
Tue, 19 Sep 2006 15:21:58 +0200 haftmann improved numeral handling for nbe
Mon, 11 Sep 2006 14:28:47 +0200 haftmann hid succ, pred in Numeral.thy
Wed, 06 Sep 2006 13:48:02 +0200 haftmann got rid of Numeral.bin type
Tue, 08 Aug 2006 08:19:44 +0200 haftmann cleanup code generation for Numerals
Wed, 26 Jul 2006 19:23:04 +0200 webertj linear arithmetic splits certain operators (e.g. min, max, abs)
Wed, 12 Jul 2006 17:00:22 +0200 haftmann adaptions in codegen
Wed, 14 Jun 2006 12:12:37 +0200 haftmann slight refinements for code generator
Tue, 16 May 2006 21:33:01 +0200 wenzelm tuned concrete syntax -- abbreviation/const_syntax;
Tue, 09 May 2006 10:10:28 +0200 haftmann added codegen preprocessors for numerals
Sun, 09 Apr 2006 18:51:13 +0200 wenzelm tuned syntax/abbreviations;
Thu, 09 Feb 2006 12:14:39 +0100 paulson names for simprules
Wed, 08 Feb 2006 15:12:59 +0100 nipkow made "dvd" on numbers executable by simp.
Thu, 19 Jan 2006 21:22:08 +0100 wenzelm setup: theory -> theory;
Tue, 17 Jan 2006 16:36:57 +0100 haftmann substantial improvements in code generator
Thu, 29 Sep 2005 17:02:57 +0200 paulson simprules need names
Tue, 27 Sep 2005 12:16:06 +0200 berghofe nat_number_of is no longer declared as code lemma, since this turned
Wed, 21 Sep 2005 12:02:19 +0200 berghofe Declared nat_number_of as code lemma.
Tue, 16 Aug 2005 18:53:11 +0200 paulson more simprules now have names
Tue, 12 Jul 2005 17:56:03 +0200 avigad added lemmas to OrderedGroup.thy (reasoning about signs, absolute value, triangle inequalities)
Fri, 01 Jul 2005 14:08:53 +0200 berghofe Moved code generator setup from NatBin to IntDef.
Thu, 16 Jun 2005 19:51:04 +0200 paulson a few new integer lemmas
Mon, 16 May 2005 10:29:15 +0200 paulson Use of IntInf.int instead of int in most numeric simprocs; avoids
Wed, 04 May 2005 08:36:10 +0200 nipkow Fixing a problem with lin.arith.
Wed, 23 Mar 2005 12:09:18 +0100 paulson replaced bool by a new datatype "bit" for binary numerals
Sun, 13 Feb 2005 17:15:14 +0100 skalberg Deleted Library.option type.
Mon, 17 Jan 2005 15:21:40 +0100 nipkow Removed div/mod ML code because it fails for 0.
Fri, 14 Jan 2005 12:00:27 +0100 nipkow made diff_less a simp rule
Tue, 19 Oct 2004 18:18:45 +0200 paulson converted some induct_tac to induct
Thu, 07 Oct 2004 15:42:30 +0200 paulson simplification tweaks for better arithmetic reasoning
Wed, 18 Aug 2004 11:09:40 +0200 nipkow import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 nipkow New theory header syntax.
Mon, 16 Aug 2004 12:29:09 +0200 berghofe Replaced `div and `mod in consts_code section by div and mod.
Thu, 01 Jul 2004 12:29:53 +0200 paulson new treatment of binary numerals
Thu, 24 Jun 2004 17:52:02 +0200 paulson replaced monomorphic abs definitions by abs_if
Tue, 11 May 2004 20:11:08 +0200 obua changes made due to new Ring_and_Field theory
Mon, 15 Mar 2004 10:46:01 +0100 paulson new lemma
Mon, 08 Mar 2004 11:12:06 +0100 paulson generic theorems about exponentials; general tidying up
Thu, 04 Mar 2004 12:06:07 +0100 paulson new material from Avigad, and simplified treatment of division by 0
Sun, 29 Feb 2004 23:05:48 +0100 berghofe Added specific code generator for number_of.
Tue, 17 Feb 2004 10:41:59 +0100 paulson further tweaks to the numeric theories
Sun, 15 Feb 2004 10:46:37 +0100 paulson Polymorphic treatment of binary arithmetic using axclasses
Tue, 10 Feb 2004 12:02:11 +0100 paulson generic of_nat and of_int functions, and generalization of iszero
Tue, 27 Jan 2004 15:39:51 +0100 paulson replacing HOL/Real/PRat, PNat by the rational number development
Mon, 12 Jan 2004 16:51:45 +0100 paulson Added lemmas to Ring_and_Field with slightly modified simplification rules
Wed, 10 Dec 2003 15:59:34 +0100 paulson Moving some theorems from Real/RealArith0.ML
less more (0) -60 tip