Wed, 06 Dec 2006 01:12:43 +0100 |
wenzelm |
added aliases for nat_recs/cases;
|
file |
diff |
annotate
|
Wed, 22 Nov 2006 10:20:16 +0100 |
haftmann |
cleanup
|
file |
diff |
annotate
|
Sat, 18 Nov 2006 00:20:18 +0100 |
haftmann |
power is now a class
|
file |
diff |
annotate
|
Wed, 08 Nov 2006 21:45:13 +0100 |
wenzelm |
removed obsolete nat_case_tr' (duplicates case_tr' in datatype_package.ML);
|
file |
diff |
annotate
|
Wed, 08 Nov 2006 13:48:29 +0100 |
wenzelm |
removed theory NatArith (now part of Nat);
|
file |
diff |
annotate
|
Mon, 06 Nov 2006 16:28:31 +0100 |
haftmann |
code generator module naming improved
|
file |
diff |
annotate
|
Mon, 16 Oct 2006 14:07:19 +0200 |
haftmann |
added explicit print translation for nat_case
|
file |
diff |
annotate
|
Mon, 02 Oct 2006 23:00:50 +0200 |
haftmann |
added code generator names for nat_rec and nat_case
|
file |
diff |
annotate
|
Tue, 26 Sep 2006 13:34:16 +0200 |
haftmann |
renamed 0 and 1 to HOL.zero and HOL.one respectivly; introduced corresponding syntactic classes
|
file |
diff |
annotate
|
Mon, 25 Sep 2006 17:04:15 +0200 |
haftmann |
refinements in codegen serializer
|
file |
diff |
annotate
|
Wed, 20 Sep 2006 12:24:11 +0200 |
haftmann |
name shifts
|
file |
diff |
annotate
|
Tue, 19 Sep 2006 15:21:42 +0200 |
haftmann |
added operational equality
|
file |
diff |
annotate
|
Mon, 14 Aug 2006 13:46:06 +0200 |
haftmann |
simplified code generator setup
|
file |
diff |
annotate
|
Tue, 08 Aug 2006 08:19:44 +0200 |
haftmann |
cleanup code generation for Numerals
|
file |
diff |
annotate
|
Wed, 14 Jun 2006 12:14:42 +0200 |
haftmann |
slight adaption for code generator
|
file |
diff |
annotate
|
Tue, 13 Jun 2006 15:07:58 +0200 |
paulson |
new results
|
file |
diff |
annotate
|
Fri, 05 May 2006 21:59:41 +0200 |
wenzelm |
axiomatization;
|
file |
diff |
annotate
|
Tue, 17 Jan 2006 16:36:57 +0100 |
haftmann |
substantial improvements in code generator
|
file |
diff |
annotate
|
Wed, 11 Jan 2006 10:59:55 +0100 |
paulson |
tidied, and giving theorems names
|
file |
diff |
annotate
|
Thu, 29 Sep 2005 00:58:55 +0200 |
wenzelm |
more finalconsts;
|
file |
diff |
annotate
|
Thu, 22 Sep 2005 23:56:15 +0200 |
nipkow |
renamed rules to iprover
|
file |
diff |
annotate
|
Wed, 13 Jul 2005 15:06:20 +0200 |
paulson |
generlization of some "nat" theorems
|
file |
diff |
annotate
|
Thu, 07 Jul 2005 12:39:17 +0200 |
nipkow |
linear arithmetic now takes "&" in assumptions apart.
|
file |
diff |
annotate
|
Fri, 01 Jul 2005 13:56:34 +0200 |
berghofe |
Moved some code lemmas from Main to Nat.
|
file |
diff |
annotate
|
Wed, 04 May 2005 08:36:10 +0200 |
nipkow |
Fixing a problem with lin.arith.
|
file |
diff |
annotate
|
Mon, 21 Feb 2005 15:04:10 +0100 |
nipkow |
comprehensive cleanup, replacing sumr by setsum
|
file |
diff |
annotate
|
Wed, 15 Dec 2004 17:32:40 +0100 |
paulson |
removal of archaic Abs/Rep proofs
|
file |
diff |
annotate
|
Mon, 29 Nov 2004 14:02:55 +0100 |
paulson |
converted to Isar script, simplifying some results
|
file |
diff |
annotate
|
Sat, 13 Nov 2004 07:47:34 +0100 |
nipkow |
More lemmas
|
file |
diff |
annotate
|
Tue, 19 Oct 2004 18:18:45 +0200 |
paulson |
converted some induct_tac to induct
|
file |
diff |
annotate
|
Wed, 18 Aug 2004 11:09:40 +0200 |
nipkow |
import -> imports
|
file |
diff |
annotate
|
Mon, 16 Aug 2004 14:22:27 +0200 |
nipkow |
New theory header syntax.
|
file |
diff |
annotate
|
Wed, 12 May 2004 10:00:56 +0200 |
nipkow |
fixed latex problems
|
file |
diff |
annotate
|
Tue, 11 May 2004 20:11:08 +0200 |
obua |
changes made due to new Ring_and_Field theory
|
file |
diff |
annotate
|
Sat, 01 May 2004 22:01:57 +0200 |
wenzelm |
tuned instance statements;
|
file |
diff |
annotate
|
Fri, 09 Jan 2004 10:46:18 +0100 |
paulson |
Defining the type class "ringpower" and deleting superseded theorems for
|
file |
diff |
annotate
|
Tue, 06 Jan 2004 10:40:15 +0100 |
paulson |
Ring_and_Field now requires axiom add_left_imp_eq for semirings.
|
file |
diff |
annotate
|
Sat, 27 Dec 2003 21:02:14 +0100 |
paulson |
re-organized numeric lemmas
|
file |
diff |
annotate
|
Fri, 19 Dec 2003 04:28:45 +0100 |
nipkow |
*** empty log message ***
|
file |
diff |
annotate
|
Tue, 25 Nov 2003 10:37:03 +0100 |
paulson |
More refinements to Ring_and_Field and numerics. Conversion of Divides_lemmas
|
file |
diff |
annotate
|
Mon, 24 Nov 2003 15:33:07 +0100 |
paulson |
conversion of integers to use Ring_and_Field;
|
file |
diff |
annotate
|
Fri, 21 Nov 2003 11:15:40 +0100 |
paulson |
HOL: installation of Ring_and_Field as the basis for Naturals and Reals
|
file |
diff |
annotate
|
Fri, 26 Sep 2003 10:34:57 +0200 |
paulson |
misc tidying
|
file |
diff |
annotate
|
Mon, 22 Sep 2003 16:02:51 +0200 |
berghofe |
Improved efficiency of code generated for + and -
|
file |
diff |
annotate
|
Thu, 24 Jul 2003 18:23:00 +0200 |
paulson |
declarations moved from PreList.thy
|
file |
diff |
annotate
|
Mon, 30 Sep 2002 15:44:21 +0200 |
nipkow |
modified induct method
|
file |
diff |
annotate
|
Thu, 26 Sep 2002 10:51:29 +0200 |
paulson |
Converted Fun to Isar style.
|
file |
diff |
annotate
|
Mon, 05 Aug 2002 14:27:42 +0200 |
berghofe |
- Converted to new theory format
|
file |
diff |
annotate
|
Sat, 01 Dec 2001 18:52:32 +0100 |
wenzelm |
renamed class "term" to "type" (actually "HOL.type");
|
file |
diff |
annotate
|
Wed, 25 Jul 2001 13:13:01 +0200 |
paulson |
partial restructuring to reduce dependence on Axiom of Choice
|
file |
diff |
annotate
|
Tue, 22 May 2001 15:10:06 +0200 |
berghofe |
Inductive definitions are now introduced earlier in the theory hierarchy.
|
file |
diff |
annotate
|
Thu, 15 Feb 2001 16:00:36 +0100 |
oheimb |
added nat as instance of new wellorder axclass
|
file |
diff |
annotate
|
Fri, 10 Nov 2000 19:04:31 +0100 |
wenzelm |
added axclass power (from HOL.thy);
|
file |
diff |
annotate
|
Tue, 25 Jul 2000 00:06:46 +0200 |
wenzelm |
rearranged setup of arithmetic procedures, avoiding global reference values;
|
file |
diff |
annotate
|
Mon, 04 Oct 1999 21:44:28 +0200 |
wenzelm |
removed DatatypePackage.setup;
|
file |
diff |
annotate
|
Wed, 21 Oct 1998 17:38:47 +0200 |
berghofe |
Changed syntax of rep_datatype.
|
file |
diff |
annotate
|
Fri, 18 Sep 1998 14:36:54 +0200 |
paulson |
updated comments
|
file |
diff |
annotate
|
Fri, 24 Jul 1998 13:34:59 +0200 |
berghofe |
Declaration of type 'nat' as a datatype (this allows usage of
|
file |
diff |
annotate
|
Fri, 20 Feb 1998 17:56:39 +0100 |
nipkow |
Congruence rules use == in premises now.
|
file |
diff |
annotate
|
Mon, 09 Feb 1998 18:09:35 +0100 |
nipkow |
Replaced ALLNEWSUBGOALS by THEN_ALL_NEW
|
file |
diff |
annotate
|