src/HOL/Nat.thy
Tue, 11 May 2004 20:11:08 +0200 changes made due to new Ring_and_Field theory
Sat, 01 May 2004 22:01:57 +0200 tuned instance statements;
Fri, 09 Jan 2004 10:46:18 +0100 Defining the type class "ringpower" and deleting superseded theorems for
Tue, 06 Jan 2004 10:40:15 +0100 Ring_and_Field now requires axiom add_left_imp_eq for semirings.
Sat, 27 Dec 2003 21:02:14 +0100 re-organized numeric lemmas
Fri, 19 Dec 2003 04:28:45 +0100 *** empty log message ***
Tue, 25 Nov 2003 10:37:03 +0100 More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
Mon, 24 Nov 2003 15:33:07 +0100 conversion of integers to use Ring_and_Field;
Fri, 21 Nov 2003 11:15:40 +0100 HOL: installation of Ring_and_Field as the basis for Naturals and Reals
Fri, 26 Sep 2003 10:34:57 +0200 misc tidying
Mon, 22 Sep 2003 16:02:51 +0200 Improved efficiency of code generated for + and -
Thu, 24 Jul 2003 18:23:00 +0200 declarations moved from PreList.thy
Mon, 30 Sep 2002 15:44:21 +0200 modified induct method
Thu, 26 Sep 2002 10:51:29 +0200 Converted Fun to Isar style.
Mon, 05 Aug 2002 14:27:42 +0200 - Converted to new theory format
Sat, 01 Dec 2001 18:52:32 +0100 renamed class "term" to "type" (actually "HOL.type");
Wed, 25 Jul 2001 13:13:01 +0200 partial restructuring to reduce dependence on Axiom of Choice
Tue, 22 May 2001 15:10:06 +0200 Inductive definitions are now introduced earlier in the theory hierarchy.
Thu, 15 Feb 2001 16:00:36 +0100 added nat as instance of new wellorder axclass
Fri, 10 Nov 2000 19:04:31 +0100 added axclass power (from HOL.thy);
Tue, 25 Jul 2000 00:06:46 +0200 rearranged setup of arithmetic procedures, avoiding global reference values;
Mon, 04 Oct 1999 21:44:28 +0200 removed DatatypePackage.setup;
Wed, 21 Oct 1998 17:38:47 +0200 Changed syntax of rep_datatype.
Fri, 18 Sep 1998 14:36:54 +0200 updated comments
Fri, 24 Jul 1998 13:34:59 +0200 Declaration of type 'nat' as a datatype (this allows usage of
Fri, 20 Feb 1998 17:56:39 +0100 Congruence rules use == in premises now.
Mon, 09 Feb 1998 18:09:35 +0100 Replaced ALLNEWSUBGOALS by THEN_ALL_NEW
Mon, 03 Nov 1997 21:12:21 +0100 nat datatype_info moved to Nat.thy;
Fri, 30 May 1997 15:19:58 +0200 Overloading of "^" requires new type class "power", with types "nat" and
Wed, 12 Feb 1997 18:53:59 +0100 New class "order" and accompanying changes.
Thu, 23 Jan 1997 12:55:31 +0100 removed \<mu> syntax;
Fri, 13 Dec 1996 18:40:50 +0100 adaptions for symbol font
Wed, 27 Nov 1996 16:45:57 +0100 moved "1", "2" to syntax section;
Tue, 25 Jun 1996 13:11:29 +0200 Changed argument order of nat_rec.
Tue, 23 Apr 1996 17:01:51 +0200 *** empty log message ***
Tue, 23 Apr 1996 16:58:21 +0200 repaired critical proofs depending on the order inside non-confluent SimpSets,
Wed, 17 Apr 1996 17:59:58 +0200 *** empty log message ***
Thu, 28 Mar 1996 12:25:55 +0100 Translations for 1 and 2 moved from Hoare/Examples.thy to Nat.thy
Tue, 05 Mar 1996 15:55:15 +0100 Converted TABs to spaces
Mon, 04 Mar 1996 14:37:33 +0100 Added a constant UNIV == {x.True}
Mon, 05 Feb 1996 21:27:16 +0100 expanded tabs; renamed subtype to typedef;
Wed, 29 Nov 1995 16:44:59 +0100 removed quotes from types in consts and syntax sections
Wed, 21 Jun 1995 15:47:10 +0200 removed \...\ inside strings
Fri, 24 Mar 1995 12:30:35 +0100 changed syntax of tuples from <..., ...> to (..., ...)
Fri, 03 Mar 1995 12:02:25 +0100 new version of HOL with curried function application