src/HOL/Nat.thy
Mon, 14 Aug 2006 13:46:06 +0200 haftmann simplified code generator setup
Tue, 08 Aug 2006 08:19:44 +0200 haftmann cleanup code generation for Numerals
Wed, 14 Jun 2006 12:14:42 +0200 haftmann slight adaption for code generator
Tue, 13 Jun 2006 15:07:58 +0200 paulson new results
Fri, 05 May 2006 21:59:41 +0200 wenzelm axiomatization;
Tue, 17 Jan 2006 16:36:57 +0100 haftmann substantial improvements in code generator
Wed, 11 Jan 2006 10:59:55 +0100 paulson tidied, and giving theorems names
Thu, 29 Sep 2005 00:58:55 +0200 wenzelm more finalconsts;
Thu, 22 Sep 2005 23:56:15 +0200 nipkow renamed rules to iprover
Wed, 13 Jul 2005 15:06:20 +0200 paulson generlization of some "nat" theorems
Thu, 07 Jul 2005 12:39:17 +0200 nipkow linear arithmetic now takes "&" in assumptions apart.
Fri, 01 Jul 2005 13:56:34 +0200 berghofe Moved some code lemmas from Main to Nat.
Wed, 04 May 2005 08:36:10 +0200 nipkow Fixing a problem with lin.arith.
Mon, 21 Feb 2005 15:04:10 +0100 nipkow comprehensive cleanup, replacing sumr by setsum
Wed, 15 Dec 2004 17:32:40 +0100 paulson removal of archaic Abs/Rep proofs
Mon, 29 Nov 2004 14:02:55 +0100 paulson converted to Isar script, simplifying some results
Sat, 13 Nov 2004 07:47:34 +0100 nipkow More lemmas
Tue, 19 Oct 2004 18:18:45 +0200 paulson converted some induct_tac to induct
Wed, 18 Aug 2004 11:09:40 +0200 nipkow import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 nipkow New theory header syntax.
Wed, 12 May 2004 10:00:56 +0200 nipkow fixed latex problems
Tue, 11 May 2004 20:11:08 +0200 obua changes made due to new Ring_and_Field theory
Sat, 01 May 2004 22:01:57 +0200 wenzelm tuned instance statements;
Fri, 09 Jan 2004 10:46:18 +0100 paulson Defining the type class "ringpower" and deleting superseded theorems for
Tue, 06 Jan 2004 10:40:15 +0100 paulson Ring_and_Field now requires axiom add_left_imp_eq for semirings.
Sat, 27 Dec 2003 21:02:14 +0100 paulson re-organized numeric lemmas
Fri, 19 Dec 2003 04:28:45 +0100 nipkow *** empty log message ***
Tue, 25 Nov 2003 10:37:03 +0100 paulson More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
Mon, 24 Nov 2003 15:33:07 +0100 paulson conversion of integers to use Ring_and_Field;
Fri, 21 Nov 2003 11:15:40 +0100 paulson HOL: installation of Ring_and_Field as the basis for Naturals and Reals
Fri, 26 Sep 2003 10:34:57 +0200 paulson misc tidying
Mon, 22 Sep 2003 16:02:51 +0200 berghofe Improved efficiency of code generated for + and -
Thu, 24 Jul 2003 18:23:00 +0200 paulson declarations moved from PreList.thy
Mon, 30 Sep 2002 15:44:21 +0200 nipkow modified induct method
Thu, 26 Sep 2002 10:51:29 +0200 paulson Converted Fun to Isar style.
Mon, 05 Aug 2002 14:27:42 +0200 berghofe - Converted to new theory format
Sat, 01 Dec 2001 18:52:32 +0100 wenzelm renamed class "term" to "type" (actually "HOL.type");
Wed, 25 Jul 2001 13:13:01 +0200 paulson partial restructuring to reduce dependence on Axiom of Choice
Tue, 22 May 2001 15:10:06 +0200 berghofe Inductive definitions are now introduced earlier in the theory hierarchy.
Thu, 15 Feb 2001 16:00:36 +0100 oheimb added nat as instance of new wellorder axclass
Fri, 10 Nov 2000 19:04:31 +0100 wenzelm added axclass power (from HOL.thy);
Tue, 25 Jul 2000 00:06:46 +0200 wenzelm rearranged setup of arithmetic procedures, avoiding global reference values;
Mon, 04 Oct 1999 21:44:28 +0200 wenzelm removed DatatypePackage.setup;
Wed, 21 Oct 1998 17:38:47 +0200 berghofe Changed syntax of rep_datatype.
Fri, 18 Sep 1998 14:36:54 +0200 paulson updated comments
Fri, 24 Jul 1998 13:34:59 +0200 berghofe Declaration of type 'nat' as a datatype (this allows usage of
Fri, 20 Feb 1998 17:56:39 +0100 nipkow Congruence rules use == in premises now.
Mon, 09 Feb 1998 18:09:35 +0100 nipkow Replaced ALLNEWSUBGOALS by THEN_ALL_NEW
Mon, 03 Nov 1997 21:12:21 +0100 wenzelm nat datatype_info moved to Nat.thy;
Fri, 30 May 1997 15:19:58 +0200 paulson Overloading of "^" requires new type class "power", with types "nat" and
Wed, 12 Feb 1997 18:53:59 +0100 nipkow New class "order" and accompanying changes.
Thu, 23 Jan 1997 12:55:31 +0100 wenzelm removed \<mu> syntax;
Fri, 13 Dec 1996 18:40:50 +0100 oheimb adaptions for symbol font
Wed, 27 Nov 1996 16:45:57 +0100 wenzelm moved "1", "2" to syntax section;
Tue, 25 Jun 1996 13:11:29 +0200 berghofe Changed argument order of nat_rec.
Tue, 23 Apr 1996 17:01:51 +0200 oheimb *** empty log message ***
Tue, 23 Apr 1996 16:58:21 +0200 oheimb repaired critical proofs depending on the order inside non-confluent SimpSets,
Wed, 17 Apr 1996 17:59:58 +0200 oheimb *** empty log message ***
Thu, 28 Mar 1996 12:25:55 +0100 paulson Translations for 1 and 2 moved from Hoare/Examples.thy to Nat.thy
Tue, 05 Mar 1996 15:55:15 +0100 paulson Converted TABs to spaces
less more (0) -60 tip