Tue, 19 Sep 2006 15:22:29 +0200 removed
haftmann [Tue, 19 Sep 2006 15:22:29 +0200] rev 20603
removed
Tue, 19 Sep 2006 15:22:29 +0200 moved part of normalization oracle here
haftmann [Tue, 19 Sep 2006 15:22:29 +0200] rev 20602
moved part of normalization oracle here
Tue, 19 Sep 2006 15:22:28 +0200 classical arity syntax
haftmann [Tue, 19 Sep 2006 15:22:28 +0200] rev 20601
classical arity syntax
Tue, 19 Sep 2006 15:22:26 +0200 added codegen_data
haftmann [Tue, 19 Sep 2006 15:22:26 +0200] rev 20600
added codegen_data
Tue, 19 Sep 2006 15:22:24 +0200 moved base setup for evaluation oracle hier
haftmann [Tue, 19 Sep 2006 15:22:24 +0200] rev 20599
moved base setup for evaluation oracle hier
Tue, 19 Sep 2006 15:22:21 +0200 added OperationalEquality.thy
haftmann [Tue, 19 Sep 2006 15:22:21 +0200] rev 20598
added OperationalEquality.thy
Tue, 19 Sep 2006 15:22:05 +0200 code generation 2 adjustments
haftmann [Tue, 19 Sep 2006 15:22:05 +0200] rev 20597
code generation 2 adjustments
Tue, 19 Sep 2006 15:22:03 +0200 (void)
haftmann [Tue, 19 Sep 2006 15:22:03 +0200] rev 20596
(void)
Tue, 19 Sep 2006 15:21:58 +0200 improved numeral handling for nbe
haftmann [Tue, 19 Sep 2006 15:21:58 +0200] rev 20595
improved numeral handling for nbe
Tue, 19 Sep 2006 15:21:55 +0200 added suspensions in Pure
haftmann [Tue, 19 Sep 2006 15:21:55 +0200] rev 20594
added suspensions in Pure
Tue, 19 Sep 2006 15:21:52 +0200 added some stuff for code generation 2
haftmann [Tue, 19 Sep 2006 15:21:52 +0200] rev 20593
added some stuff for code generation 2
Tue, 19 Sep 2006 15:21:51 +0200 dropped error-prone code generation 2 for wfrec
haftmann [Tue, 19 Sep 2006 15:21:51 +0200] rev 20592
dropped error-prone code generation 2 for wfrec
Tue, 19 Sep 2006 15:21:48 +0200 text cleanup
haftmann [Tue, 19 Sep 2006 15:21:48 +0200] rev 20591
text cleanup
Tue, 19 Sep 2006 15:21:44 +0200 introduced syntactic classes; moved some setup to Pure/codegen, Pure/nbe or OperationalEquality.thy
haftmann [Tue, 19 Sep 2006 15:21:44 +0200] rev 20590
introduced syntactic classes; moved some setup to Pure/codegen, Pure/nbe or OperationalEquality.thy
Tue, 19 Sep 2006 15:21:43 +0200 explicit divmod algorithm for code generation
haftmann [Tue, 19 Sep 2006 15:21:43 +0200] rev 20589
explicit divmod algorithm for code generation
Tue, 19 Sep 2006 15:21:42 +0200 added operational equality
haftmann [Tue, 19 Sep 2006 15:21:42 +0200] rev 20588
added operational equality
Tue, 19 Sep 2006 15:21:41 +0200 added section on code generation 2
haftmann [Tue, 19 Sep 2006 15:21:41 +0200] rev 20587
added section on code generation 2
Tue, 19 Sep 2006 15:21:39 +0200 code_gen now peek keyword
haftmann [Tue, 19 Sep 2006 15:21:39 +0200] rev 20586
code_gen now peek keyword
Tue, 19 Sep 2006 15:19:38 +0200 cleanupdiff
haftmann [Tue, 19 Sep 2006 15:19:38 +0200] rev 20585
cleanupdiff
Tue, 19 Sep 2006 06:22:26 +0200 added classes real_div_algebra and real_field; added lemmas
huffman [Tue, 19 Sep 2006 06:22:26 +0200] rev 20584
added classes real_div_algebra and real_field; added lemmas
Tue, 19 Sep 2006 05:54:17 +0200 add Real/RealVector.thy
huffman [Tue, 19 Sep 2006 05:54:17 +0200] rev 20583
add Real/RealVector.thy
Mon, 18 Sep 2006 19:40:14 +0200 * Pure: 'class_deps' command visualizes the subclass relation;
wenzelm [Mon, 18 Sep 2006 19:40:14 +0200] rev 20582
* Pure: 'class_deps' command visualizes the subclass relation;
Mon, 18 Sep 2006 19:39:14 +0200 added class_deps;
wenzelm [Mon, 18 Sep 2006 19:39:14 +0200] rev 20581
added class_deps;
Mon, 18 Sep 2006 19:39:11 +0200 added dest_arg, i.e. a tuned version of #2 o dest_comb;
wenzelm [Mon, 18 Sep 2006 19:39:11 +0200] rev 20580
added dest_arg, i.e. a tuned version of #2 o dest_comb;
Mon, 18 Sep 2006 19:39:07 +0200 Thm.dest_arg;
wenzelm [Mon, 18 Sep 2006 19:39:07 +0200] rev 20579
Thm.dest_arg;
Mon, 18 Sep 2006 19:12:50 +0200 Present.display_graph;
wenzelm [Mon, 18 Sep 2006 19:12:50 +0200] rev 20578
Present.display_graph;
Mon, 18 Sep 2006 19:12:49 +0200 added display_graph (from thm_deps.ML);
wenzelm [Mon, 18 Sep 2006 19:12:49 +0200] rev 20577
added display_graph (from thm_deps.ML);
Mon, 18 Sep 2006 19:12:48 +0200 output: uninterpreted raw symbols -- these are usually LaTeX macros;
wenzelm [Mon, 18 Sep 2006 19:12:48 +0200] rev 20576
output: uninterpreted raw symbols -- these are usually LaTeX macros;
Mon, 18 Sep 2006 19:12:47 +0200 pretty_thm: graceful treatment of ProtoPure.thy;
wenzelm [Mon, 18 Sep 2006 19:12:47 +0200] rev 20575
pretty_thm: graceful treatment of ProtoPure.thy;
Mon, 18 Sep 2006 19:12:46 +0200 added class_deps;
wenzelm [Mon, 18 Sep 2006 19:12:46 +0200] rev 20574
added class_deps;
Mon, 18 Sep 2006 19:12:45 +0200 classes: maintain serial number;
wenzelm [Mon, 18 Sep 2006 19:12:45 +0200] rev 20573
classes: maintain serial number;
Mon, 18 Sep 2006 19:12:44 +0200 tuned;
wenzelm [Mon, 18 Sep 2006 19:12:44 +0200] rev 20572
tuned;
Mon, 18 Sep 2006 19:12:43 +0200 isatool browser: renamed option -d to -c (cf. isatool tool)
wenzelm [Mon, 18 Sep 2006 19:12:43 +0200] rev 20571
isatool browser: renamed option -d to -c (cf. isatool tool)
Mon, 18 Sep 2006 19:12:42 +0200 PRIVATE_FILE: slightly more robust way to create and dispose;
wenzelm [Mon, 18 Sep 2006 19:12:42 +0200] rev 20570
PRIVATE_FILE: slightly more robust way to create and dispose;
Mon, 18 Sep 2006 19:12:41 +0200 renamed option -d to -c (cf. isatool display);
wenzelm [Mon, 18 Sep 2006 19:12:41 +0200] rev 20569
renamed option -d to -c (cf. isatool display); operate on PRIVATE_FILE;
Mon, 18 Sep 2006 19:12:40 +0200 updated;
wenzelm [Mon, 18 Sep 2006 19:12:40 +0200] rev 20568
updated;
Mon, 18 Sep 2006 16:21:24 +0200 Bug fix to prevent exception dest_Free from escaping
paulson [Mon, 18 Sep 2006 16:21:24 +0200] rev 20567
Bug fix to prevent exception dest_Free from escaping
Mon, 18 Sep 2006 16:00:19 +0200 Added the max_new parameter, which is a cap on how many clauses may be admitted per round.
paulson [Mon, 18 Sep 2006 16:00:19 +0200] rev 20566
Added the max_new parameter, which is a cap on how many clauses may be admitted per round. Also various tidying up.
Mon, 18 Sep 2006 15:11:31 +0200 replaced implodeable_Ext by set_like
obua [Mon, 18 Sep 2006 15:11:31 +0200] rev 20565
replaced implodeable_Ext by set_like
Mon, 18 Sep 2006 10:09:57 +0200 Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb [Mon, 18 Sep 2006 10:09:57 +0200] rev 20564
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n) instead of only ... = xs!n.
Mon, 18 Sep 2006 07:48:07 +0200 replace (x + - y) with (x - y)
huffman [Mon, 18 Sep 2006 07:48:07 +0200] rev 20563
replace (x + - y) with (x - y)
Sun, 17 Sep 2006 16:44:51 +0200 add type constraint to otherwise looping iff rule
huffman [Sun, 17 Sep 2006 16:44:51 +0200] rev 20562
add type constraint to otherwise looping iff rule
Sun, 17 Sep 2006 16:44:05 +0200 generalize type of (NS)LIM to work on functions with vector space domain types
huffman [Sun, 17 Sep 2006 16:44:05 +0200] rev 20561
generalize type of (NS)LIM to work on functions with vector space domain types
Sun, 17 Sep 2006 16:42:38 +0200 norm_one is now proved from other class axioms
huffman [Sun, 17 Sep 2006 16:42:38 +0200] rev 20560
norm_one is now proved from other class axioms
Sun, 17 Sep 2006 02:56:25 +0200 removed capprox, CFinite, CInfinite, CInfinitesimal, cmonad, and cgalaxy in favor of polymorphic constants
huffman [Sun, 17 Sep 2006 02:56:25 +0200] rev 20559
removed capprox, CFinite, CInfinite, CInfinitesimal, cmonad, and cgalaxy in favor of polymorphic constants
Sun, 17 Sep 2006 02:53:36 +0200 hcmod abbreviates hnorm :: hcomplex => hypreal
huffman [Sun, 17 Sep 2006 02:53:36 +0200] rev 20558
hcmod abbreviates hnorm :: hcomplex => hypreal
Sat, 16 Sep 2006 23:46:38 +0200 complex_of_real abbreviates of_real::real=>complex;
huffman [Sat, 16 Sep 2006 23:46:38 +0200] rev 20557
complex_of_real abbreviates of_real::real=>complex; cmod abbreviates norm::complex=>real; removed several redundant lemmas
Sat, 16 Sep 2006 19:14:37 +0200 add instance for real_algebra_1 and real_normed_div_algebra
huffman [Sat, 16 Sep 2006 19:14:37 +0200] rev 20556
add instance for real_algebra_1 and real_normed_div_algebra
Sat, 16 Sep 2006 19:12:54 +0200 add instances for real_vector and real_algebra
huffman [Sat, 16 Sep 2006 19:12:54 +0200] rev 20555
add instances for real_vector and real_algebra
Sat, 16 Sep 2006 19:12:03 +0200 define new constant of_real for class real_algebra_1;
huffman [Sat, 16 Sep 2006 19:12:03 +0200] rev 20554
define new constant of_real for class real_algebra_1; define set Reals as range of_real; add lemmas about of_real and Reals
Sat, 16 Sep 2006 18:04:14 +0200 int_diff_cases moved to Integ/IntDef.thy
huffman [Sat, 16 Sep 2006 18:04:14 +0200] rev 20553
int_diff_cases moved to Integ/IntDef.thy
Sat, 16 Sep 2006 02:40:00 +0200 generalized types of many constants to work over arbitrary vector spaces;
huffman [Sat, 16 Sep 2006 02:40:00 +0200] rev 20552
generalized types of many constants to work over arbitrary vector spaces; modified theorems using Rep_star to eliminate existential quantifiers
Sat, 16 Sep 2006 02:35:58 +0200 add theorem norm_diff_triangle_ineq
huffman [Sat, 16 Sep 2006 02:35:58 +0200] rev 20551
add theorem norm_diff_triangle_ineq
Sat, 16 Sep 2006 02:32:48 +0200 add required type annotation
huffman [Sat, 16 Sep 2006 02:32:48 +0200] rev 20550
add required type annotation
Fri, 15 Sep 2006 22:56:17 +0200 removed type aliases for theory/theory_ref;
wenzelm [Fri, 15 Sep 2006 22:56:17 +0200] rev 20549
removed type aliases for theory/theory_ref;
Fri, 15 Sep 2006 22:56:13 +0200 renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
wenzelm [Fri, 15 Sep 2006 22:56:13 +0200] rev 20548
renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
Fri, 15 Sep 2006 22:56:08 +0200 tuned;
wenzelm [Fri, 15 Sep 2006 22:56:08 +0200] rev 20547
tuned;
Fri, 15 Sep 2006 20:08:38 +0200 rrule: maintain 'extra' field for rule that contain extra vars outside elhs;
wenzelm [Fri, 15 Sep 2006 20:08:38 +0200] rev 20546
rrule: maintain 'extra' field for rule that contain extra vars outside elhs; rewrite_rule_extra_vars: tuned; rewritec: omit incr_indexes in most cases, which is a big performance gain;
Fri, 15 Sep 2006 20:08:37 +0200 instantiate: omit has_duplicates check, which is irrelevant for soundness;
wenzelm [Fri, 15 Sep 2006 20:08:37 +0200] rev 20545
instantiate: omit has_duplicates check, which is irrelevant for soundness;
Fri, 15 Sep 2006 18:06:51 +0200 trivial whitespace change
webertj [Fri, 15 Sep 2006 18:06:51 +0200] rev 20544
trivial whitespace change
Fri, 15 Sep 2006 16:49:41 +0200 tuned;
wenzelm [Fri, 15 Sep 2006 16:49:41 +0200] rev 20543
tuned;
Thu, 14 Sep 2006 22:48:37 +0200 more on theorems;
wenzelm [Thu, 14 Sep 2006 22:48:37 +0200] rev 20542
more on theorems;
Thu, 14 Sep 2006 21:42:21 +0200 generalized types of Infinitesimal, HFinite, and HInfinite to work over nonstandard extensions of any real normed vector space
huffman [Thu, 14 Sep 2006 21:42:21 +0200] rev 20541
generalized types of Infinitesimal, HFinite, and HInfinite to work over nonstandard extensions of any real normed vector space
Thu, 14 Sep 2006 21:36:26 +0200 add instance for class division_ring
huffman [Thu, 14 Sep 2006 21:36:26 +0200] rev 20540
add instance for class division_ring
Thu, 14 Sep 2006 20:31:10 +0200 removed duplicate lemmas
huffman [Thu, 14 Sep 2006 20:31:10 +0200] rev 20539
removed duplicate lemmas
Thu, 14 Sep 2006 19:18:10 +0200 fixed syntax clash with Real/RealVector
huffman [Thu, 14 Sep 2006 19:18:10 +0200] rev 20538
fixed syntax clash with Real/RealVector
Thu, 14 Sep 2006 15:51:20 +0200 *** empty log message ***
wenzelm [Thu, 14 Sep 2006 15:51:20 +0200] rev 20537
*** empty log message ***
Thu, 14 Sep 2006 15:27:08 +0200 Function package: Outside their domain functions now return "arbitrary".
krauss [Thu, 14 Sep 2006 15:27:08 +0200] rev 20536
Function package: Outside their domain functions now return "arbitrary".
Thu, 14 Sep 2006 15:25:23 +0200 updated makefile
krauss [Thu, 14 Sep 2006 15:25:23 +0200] rev 20535
updated makefile
Thu, 14 Sep 2006 15:25:05 +0200 Fixed Subscript Exception occurring with Higher-Order recursion
krauss [Thu, 14 Sep 2006 15:25:05 +0200] rev 20534
Fixed Subscript Exception occurring with Higher-Order recursion
Thu, 14 Sep 2006 03:25:17 +0200 remove conflicting norm syntax
huffman [Thu, 14 Sep 2006 03:25:17 +0200] rev 20533
remove conflicting norm syntax
Thu, 14 Sep 2006 00:23:02 +0200 made SML/NJ happy;
wenzelm [Thu, 14 Sep 2006 00:23:02 +0200] rev 20532
made SML/NJ happy;
Wed, 13 Sep 2006 21:41:31 +0200 added exists_type;
wenzelm [Wed, 13 Sep 2006 21:41:31 +0200] rev 20531
added exists_type;
Wed, 13 Sep 2006 21:41:25 +0200 renamed NameSpace.drop_base to NameSpace.qualifier;
wenzelm [Wed, 13 Sep 2006 21:41:25 +0200] rev 20530
renamed NameSpace.drop_base to NameSpace.qualifier;
Wed, 13 Sep 2006 12:40:39 +0200 Updated keyword file
krauss [Wed, 13 Sep 2006 12:40:39 +0200] rev 20529
Updated keyword file
Wed, 13 Sep 2006 12:37:13 +0200 Removed debugging code imports...
krauss [Wed, 13 Sep 2006 12:37:13 +0200] rev 20528
Removed debugging code imports...
Wed, 13 Sep 2006 12:21:35 +0200 Added the "theory_const" option. Only it is OFF because it's often harmful!
paulson [Wed, 13 Sep 2006 12:21:35 +0200] rev 20527
Added the "theory_const" option. Only it is OFF because it's often harmful!
Wed, 13 Sep 2006 12:20:21 +0200 Extended the blacklist with higher-order theorems. Restructured. Added checks to
paulson [Wed, 13 Sep 2006 12:20:21 +0200] rev 20526
Extended the blacklist with higher-order theorems. Restructured. Added checks to ensure that no higher-order clauses are output in first-order mode.
Wed, 13 Sep 2006 12:18:36 +0200 bug fix to abstractions: free variables in theorem can be abstracted over.
paulson [Wed, 13 Sep 2006 12:18:36 +0200] rev 20525
bug fix to abstractions: free variables in theorem can be abstracted over.
Wed, 13 Sep 2006 12:17:17 +0200 Tweaks to is_fol_term, the first-order test. We don't count "=" as a connective
paulson [Wed, 13 Sep 2006 12:17:17 +0200] rev 20524
Tweaks to is_fol_term, the first-order test. We don't count "=" as a connective since this test is applied to clause forms.
Wed, 13 Sep 2006 12:05:50 +0200 Major update to function package, including new syntax and the (only theoretical)
krauss [Wed, 13 Sep 2006 12:05:50 +0200] rev 20523
Major update to function package, including new syntax and the (only theoretical) ability to handle local contexts.
Wed, 13 Sep 2006 00:38:38 +0200 added instance rat :: recpower
huffman [Wed, 13 Sep 2006 00:38:38 +0200] rev 20522
added instance rat :: recpower
Tue, 12 Sep 2006 21:05:39 +0200 more on theorems;
wenzelm [Tue, 12 Sep 2006 21:05:39 +0200] rev 20521
more on theorems;
Tue, 12 Sep 2006 17:45:58 +0200 tuned;
wenzelm [Tue, 12 Sep 2006 17:45:58 +0200] rev 20520
tuned;
Tue, 12 Sep 2006 17:23:34 +0200 more on terms;
wenzelm [Tue, 12 Sep 2006 17:23:34 +0200] rev 20519
more on terms;
Tue, 12 Sep 2006 17:12:51 +0200 no_syntax norm -- clash with Real/RealVector.thy;
wenzelm [Tue, 12 Sep 2006 17:12:51 +0200] rev 20518
no_syntax norm -- clash with Real/RealVector.thy;
Tue, 12 Sep 2006 17:05:44 +0200 simplify some proofs, remove obsolete realpow_divide
huffman [Tue, 12 Sep 2006 17:05:44 +0200] rev 20517
simplify some proofs, remove obsolete realpow_divide
Tue, 12 Sep 2006 17:03:52 +0200 realpow_divide -> power_divide
huffman [Tue, 12 Sep 2006 17:03:52 +0200] rev 20516
realpow_divide -> power_divide
Tue, 12 Sep 2006 16:44:04 +0200 remove extra dependency
huffman [Tue, 12 Sep 2006 16:44:04 +0200] rev 20515
remove extra dependency
Tue, 12 Sep 2006 14:50:11 +0200 more on terms;
wenzelm [Tue, 12 Sep 2006 14:50:11 +0200] rev 20514
more on terms; tuned;
Tue, 12 Sep 2006 12:16:17 +0200 Efficient term substitution -- avoids copying.
wenzelm [Tue, 12 Sep 2006 12:16:17 +0200] rev 20513
Efficient term substitution -- avoids copying. moved here from term.ML; added instantiate_maxidx;
Tue, 12 Sep 2006 12:12:57 +0200 ctyp: maintain maxidx;
wenzelm [Tue, 12 Sep 2006 12:12:57 +0200] rev 20512
ctyp: maintain maxidx; cterm_match: tight maxidx for substitution; instantiate: determine maxidx from insts -- major performance improvement; moved term subst functions to TermSubst; tuned;
Tue, 12 Sep 2006 12:12:55 +0200 removed obsolete aconvs (use eq_list aconv);
wenzelm [Tue, 12 Sep 2006 12:12:55 +0200] rev 20511
removed obsolete aconvs (use eq_list aconv); tuned aconv --- more efficient on identical subterms; moved term subst functions to term_subst.ML;
Tue, 12 Sep 2006 12:12:53 +0200 tuned eq_list;
wenzelm [Tue, 12 Sep 2006 12:12:53 +0200] rev 20510
tuned eq_list;
Tue, 12 Sep 2006 12:12:46 +0200 moved term subst functions to TermSubst;
wenzelm [Tue, 12 Sep 2006 12:12:46 +0200] rev 20509
moved term subst functions to TermSubst;
Tue, 12 Sep 2006 12:12:39 +0200 intr/elim: use constant complexity thanks to tuned Thm.instantiate/implies_elim;
wenzelm [Tue, 12 Sep 2006 12:12:39 +0200] rev 20508
intr/elim: use constant complexity thanks to tuned Thm.instantiate/implies_elim;
Tue, 12 Sep 2006 12:12:33 +0200 added Pure/term_subst.ML;
wenzelm [Tue, 12 Sep 2006 12:12:33 +0200] rev 20507
added Pure/term_subst.ML;
Tue, 12 Sep 2006 12:12:25 +0200 added Gentzen:1935;
wenzelm [Tue, 12 Sep 2006 12:12:25 +0200] rev 20506
added Gentzen:1935;
Tue, 12 Sep 2006 07:49:07 +0200 import RealVector
huffman [Tue, 12 Sep 2006 07:49:07 +0200] rev 20505
import RealVector
Tue, 12 Sep 2006 06:44:45 +0200 formalization of vector spaces and algebras over the real numbers
huffman [Tue, 12 Sep 2006 06:44:45 +0200] rev 20504
formalization of vector spaces and algebras over the real numbers
Mon, 11 Sep 2006 21:35:19 +0200 induct method: renamed 'fixing' to 'arbitrary';
wenzelm [Mon, 11 Sep 2006 21:35:19 +0200] rev 20503
induct method: renamed 'fixing' to 'arbitrary';
Mon, 11 Sep 2006 14:35:30 +0200 updated;
wenzelm [Mon, 11 Sep 2006 14:35:30 +0200] rev 20502
updated;
Mon, 11 Sep 2006 14:35:25 +0200 more rules;
wenzelm [Mon, 11 Sep 2006 14:35:25 +0200] rev 20501
more rules;
Mon, 11 Sep 2006 14:28:47 +0200 hid succ, pred in Numeral.thy
haftmann [Mon, 11 Sep 2006 14:28:47 +0200] rev 20500
hid succ, pred in Numeral.thy
Mon, 11 Sep 2006 12:27:36 +0200 updated;
wenzelm [Mon, 11 Sep 2006 12:27:36 +0200] rev 20499
updated;
Mon, 11 Sep 2006 12:27:30 +0200 more rules;
wenzelm [Mon, 11 Sep 2006 12:27:30 +0200] rev 20498
more rules;
Mon, 11 Sep 2006 12:27:21 +0200 tuned;
wenzelm [Mon, 11 Sep 2006 12:27:21 +0200] rev 20497
tuned;
Sun, 10 Sep 2006 05:34:24 +0200 added axclass division_ring (like field without commutativity; includes e.g. quaternions) and generalized some theorems from field to division_ring
huffman [Sun, 10 Sep 2006 05:34:24 +0200] rev 20496
added axclass division_ring (like field without commutativity; includes e.g. quaternions) and generalized some theorems from field to division_ring
Sat, 09 Sep 2006 18:28:42 +0200 cleaned up
huffman [Sat, 09 Sep 2006 18:28:42 +0200] rev 20495
cleaned up
Fri, 08 Sep 2006 19:44:43 +0200 tuned;
wenzelm [Fri, 08 Sep 2006 19:44:43 +0200] rev 20494
tuned;
Fri, 08 Sep 2006 17:33:05 +0200 tuned;
wenzelm [Fri, 08 Sep 2006 17:33:05 +0200] rev 20493
tuned;
Fri, 08 Sep 2006 13:33:11 +0200 changed order of type classes and axclasses
haftmann [Fri, 08 Sep 2006 13:33:11 +0200] rev 20492
changed order of type classes and axclasses
Thu, 07 Sep 2006 20:12:08 +0200 tuned;
wenzelm [Thu, 07 Sep 2006 20:12:08 +0200] rev 20491
tuned;
Thu, 07 Sep 2006 15:16:51 +0200 updated;
wenzelm [Thu, 07 Sep 2006 15:16:51 +0200] rev 20490
updated;
Thu, 07 Sep 2006 15:16:41 +0200 tentative appendix C;
wenzelm [Thu, 07 Sep 2006 15:16:41 +0200] rev 20489
tentative appendix C;
Thu, 07 Sep 2006 15:16:26 +0200 tuned;
wenzelm [Thu, 07 Sep 2006 15:16:26 +0200] rev 20488
tuned;
Wed, 06 Sep 2006 22:48:36 +0200 read_instantiate: declare names of TVars as well (temporary workaround for no-freeze feature of type inference);
wenzelm [Wed, 06 Sep 2006 22:48:36 +0200] rev 20487
read_instantiate: declare names of TVars as well (temporary workaround for no-freeze feature of type inference);
Wed, 06 Sep 2006 17:39:52 +0200 rawsat_thm: mk_conjunction_list replaced by Conjunction.mk_conjunction_list
webertj [Wed, 06 Sep 2006 17:39:52 +0200] rev 20486
rawsat_thm: mk_conjunction_list replaced by Conjunction.mk_conjunction_list
Wed, 06 Sep 2006 13:48:02 +0200 got rid of Numeral.bin type
haftmann [Wed, 06 Sep 2006 13:48:02 +0200] rev 20485
got rid of Numeral.bin type
Wed, 06 Sep 2006 10:01:27 +0200 now using TypecopyPackage
haftmann [Wed, 06 Sep 2006 10:01:27 +0200] rev 20484
now using TypecopyPackage
(0) -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip