Mon, 26 Feb 2007 23:18:27 +0100 Further operations on type thm, outside the inference kernel.
wenzelm [Mon, 26 Feb 2007 23:18:27 +0100] rev 22362
Further operations on type thm, outside the inference kernel.
Mon, 26 Feb 2007 23:18:26 +0100 added more_thm.ML;
wenzelm [Mon, 26 Feb 2007 23:18:26 +0100] rev 22361
added more_thm.ML;
Mon, 26 Feb 2007 23:18:24 +0100 moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
wenzelm [Mon, 26 Feb 2007 23:18:24 +0100] rev 22360
moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
Mon, 26 Feb 2007 21:34:16 +0100 Added formalization of size-change principle (experimental).
krauss [Mon, 26 Feb 2007 21:34:16 +0100] rev 22359
Added formalization of size-change principle (experimental).
Mon, 26 Feb 2007 20:14:52 +0100 added theorems_of;
wenzelm [Mon, 26 Feb 2007 20:14:52 +0100] rev 22358
added theorems_of;
Mon, 26 Feb 2007 20:14:47 +0100 removed obsolete theorem_space;
wenzelm [Mon, 26 Feb 2007 20:14:47 +0100] rev 22357
removed obsolete theorem_space;
Mon, 26 Feb 2007 15:08:37 +0100 Added lemma lfp_const: "lfp (%x. t) = t
krauss [Mon, 26 Feb 2007 15:08:37 +0100] rev 22356
Added lemma lfp_const: "lfp (%x. t) = t
Fri, 23 Feb 2007 08:39:28 +0100 exported serializer parsers
haftmann [Fri, 23 Feb 2007 08:39:28 +0100] rev 22355
exported serializer parsers
Fri, 23 Feb 2007 08:39:27 +0100 proper treatment of -> as type constructor
haftmann [Fri, 23 Feb 2007 08:39:27 +0100] rev 22354
proper treatment of -> as type constructor
Fri, 23 Feb 2007 08:39:26 +0100 tuned
haftmann [Fri, 23 Feb 2007 08:39:26 +0100] rev 22353
tuned
Fri, 23 Feb 2007 08:39:25 +0100 add_path for naming in proof contexts
haftmann [Fri, 23 Feb 2007 08:39:25 +0100] rev 22352
add_path for naming in proof contexts
Fri, 23 Feb 2007 08:39:24 +0100 locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann [Fri, 23 Feb 2007 08:39:24 +0100] rev 22351
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
Fri, 23 Feb 2007 08:39:23 +0100 slightly tuned
haftmann [Fri, 23 Feb 2007 08:39:23 +0100] rev 22350
slightly tuned
Fri, 23 Feb 2007 08:39:22 +0100 slight cleanup
haftmann [Fri, 23 Feb 2007 08:39:22 +0100] rev 22349
slight cleanup
Fri, 23 Feb 2007 08:39:21 +0100 adjusted code lemmas
haftmann [Fri, 23 Feb 2007 08:39:21 +0100] rev 22348
adjusted code lemmas
Fri, 23 Feb 2007 08:39:20 +0100 continued
haftmann [Fri, 23 Feb 2007 08:39:20 +0100] rev 22347
continued
Fri, 23 Feb 2007 08:39:19 +0100 dropped diagnostic switch
haftmann [Fri, 23 Feb 2007 08:39:19 +0100] rev 22346
dropped diagnostic switch
Thu, 22 Feb 2007 10:25:14 +0100 Improved handling of situation when theorem in cache disagrees with theorem supplied: new clauses
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.
Wed, 21 Feb 2007 13:51:12 +0100 Fixed print translations for quantifiers a la "ALL x>=t. P x". These used
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".
Wed, 21 Feb 2007 02:30:06 +0100 prevent quadratic time removal of duplicates if filter list is empty (likely to have too many results)
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)
Tue, 20 Feb 2007 00:53:18 +0100 added missing \
kleing [Tue, 20 Feb 2007 00:53:18 +0100] rev 22342
added missing \
Tue, 20 Feb 2007 00:23:58 +0100 updated docs with new with_dups syntax for find_theorems
kleing [Tue, 20 Feb 2007 00:23:58 +0100] rev 22341
updated docs with new with_dups syntax for find_theorems
Tue, 20 Feb 2007 00:14:33 +0100 Remove duplicates from printed theorems in 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.
Mon, 19 Feb 2007 16:44:08 +0100 more precise error message in parameter unification
schirmer [Mon, 19 Feb 2007 16:44:08 +0100] rev 22339
more precise error message in parameter unification
Sat, 17 Feb 2007 18:01:22 +0100 Updated
aspinall [Sat, 17 Feb 2007 18:01:22 +0100] rev 22338
Updated
Sat, 17 Feb 2007 18:00:59 +0100 Fix <pgipquit>. Remove unused pgmlatomsN. Make showid match askids. Use string functions for showid, avoiding printwrap kludge.
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.
Sat, 17 Feb 2007 17:22:53 +0100 <idvalue>: add name attribute to allow unsolicited updates.
aspinall [Sat, 17 Feb 2007 17:22:53 +0100] rev 22336
<idvalue>: add name attribute to allow unsolicited updates.
Sat, 17 Feb 2007 17:19:59 +0100 pretty_full_theory: expose in signature.
aspinall [Sat, 17 Feb 2007 17:19:59 +0100] rev 22335
pretty_full_theory: expose in signature.
Sat, 17 Feb 2007 17:18:47 +0100 Clarify comment
aspinall [Sat, 17 Feb 2007 17:18:47 +0100] rev 22334
Clarify comment
Fri, 16 Feb 2007 22:46:03 +0100 unified arity parser/arguments;
wenzelm [Fri, 16 Feb 2007 22:46:03 +0100] rev 22333
unified arity parser/arguments;
Fri, 16 Feb 2007 22:13:16 +0100 ML text: informative Output.debug only;
wenzelm [Fri, 16 Feb 2007 22:13:16 +0100] rev 22332
ML text: informative Output.debug only;
Fri, 16 Feb 2007 22:13:15 +0100 unified arity parser/arguments;
wenzelm [Fri, 16 Feb 2007 22:13:15 +0100] rev 22331
unified arity parser/arguments;
(0) -10000 -3000 -1000 -300 -100 -50 -32 +32 +50 +100 +300 +1000 +3000 +10000 +30000 tip