haftmann [Fri, 23 Feb 2007 08:39:23 +0100] rev 22350
slightly tuned
haftmann [Fri, 23 Feb 2007 08:39:22 +0100] rev 22349
slight cleanup
haftmann [Fri, 23 Feb 2007 08:39:21 +0100] rev 22348
adjusted code lemmas
haftmann [Fri, 23 Feb 2007 08:39:20 +0100] rev 22347
continued
haftmann [Fri, 23 Feb 2007 08:39:19 +0100] rev 22346
dropped diagnostic switch
paulson [Thu, 22 Feb 2007 10:25:14 +0100] rev 22345
Improved handling of situation when theorem in cache disagrees with theorem supplied: new clauses
are now returned, fixing a bug in the metis method.
krauss [Wed, 21 Feb 2007 13:51:12 +0100] rev 22344
Fixed print translations for quantifiers a la "ALL x>=t. P x". These used
to fail when the other term in the comparison was itself a bound variable,
as in "EX y. ALL x>=y. P x".
kleing [Wed, 21 Feb 2007 02:30:06 +0100] rev 22343
prevent quadratic time removal of duplicates if filter list is empty (likely to have too many results)
kleing [Tue, 20 Feb 2007 00:53:18 +0100] rev 22342
added missing \
kleing [Tue, 20 Feb 2007 00:23:58 +0100] rev 22341
updated docs with new with_dups syntax for find_theorems
kleing [Tue, 20 Feb 2007 00:14:33 +0100] rev 22340
Remove duplicates from printed theorems in find_theorems
(still pretty slow, needs optimising).
Added syntax "find_theorems (..) with_dups .." to switch off removal.
schirmer [Mon, 19 Feb 2007 16:44:08 +0100] rev 22339
more precise error message in parameter unification
aspinall [Sat, 17 Feb 2007 18:01:22 +0100] rev 22338
Updated
aspinall [Sat, 17 Feb 2007 18:00:59 +0100] rev 22337
Fix <pgipquit>. Remove unused pgmlatomsN. Make showid match askids. Use string functions for showid, avoiding printwrap kludge.
aspinall [Sat, 17 Feb 2007 17:22:53 +0100] rev 22336
<idvalue>: add name attribute to allow unsolicited updates.
aspinall [Sat, 17 Feb 2007 17:19:59 +0100] rev 22335
pretty_full_theory: expose in signature.
aspinall [Sat, 17 Feb 2007 17:18:47 +0100] rev 22334
Clarify comment
wenzelm [Fri, 16 Feb 2007 22:46:03 +0100] rev 22333
unified arity parser/arguments;
wenzelm [Fri, 16 Feb 2007 22:13:16 +0100] rev 22332
ML text: informative Output.debug only;
wenzelm [Fri, 16 Feb 2007 22:13:15 +0100] rev 22331
unified arity parser/arguments;
berghofe [Fri, 16 Feb 2007 19:19:19 +0100] rev 22330
Replaced "raise RecError" by "primrec_err" in function
gen_primrec_i to prevent error message from being suppressed.
schirmer [Fri, 16 Feb 2007 11:01:16 +0100] rev 22329
added example for print-mode Axiom
schirmer [Fri, 16 Feb 2007 11:00:47 +0100] rev 22328
added print-mode Axiom to print theorems without premises with a rule on top.
krauss [Fri, 16 Feb 2007 09:04:23 +0100] rev 22327
updated Makefile
narboux [Thu, 15 Feb 2007 18:18:21 +0100] rev 22326
start adding the attribute eqvt to some lemmas of the nominal library
krauss [Thu, 15 Feb 2007 17:35:19 +0100] rev 22325
changed termination goal to use object quantifier
krauss [Thu, 15 Feb 2007 12:14:34 +0100] rev 22324
added congruence rule for function composition
krauss [Thu, 15 Feb 2007 12:02:11 +0100] rev 22323
beta_eta_contract specification befor processing. These normal forms avoid unpleasant surprises later on.
haftmann [Wed, 14 Feb 2007 10:07:17 +0100] rev 22322
continued
haftmann [Wed, 14 Feb 2007 10:06:17 +0100] rev 22321
class package now using Locale.interpretation_i
haftmann [Wed, 14 Feb 2007 10:06:16 +0100] rev 22320
clarified explanation
haftmann [Wed, 14 Feb 2007 10:06:15 +0100] rev 22319
cleanup