wenzelm [Wed, 14 Apr 2010 22:13:28 +0200] rev 36145
merged
blanchet [Wed, 14 Apr 2010 21:22:48 +0200] rev 36144
merged
blanchet [Wed, 14 Apr 2010 21:22:13 +0200] rev 36143
added "overlord" option (to get easy access to output files for debugging) + systematically use "raw_goal" rather than an inconsistent mixture
blanchet [Wed, 14 Apr 2010 18:23:51 +0200] rev 36142
make Sledgehammer "minimize" output less confusing + round up (not down) time limits to nearest second
blanchet [Wed, 14 Apr 2010 17:10:16 +0200] rev 36141
make Sledgehammer's "timeout" option work for "minimize"
blanchet [Wed, 14 Apr 2010 16:50:25 +0200] rev 36140
fixed handling of "sledgehammer_params" that get a default value from Isabelle menu;
and added "atp" as alias for "atps"
hoelzl [Wed, 14 Apr 2010 19:46:36 +0200] rev 36139
Spelling error: theroems -> theorems
krauss [Wed, 14 Apr 2010 17:50:22 +0200] rev 36138
advertise [rename_abs] attribute in LaTeXsugar -- wish I had known about this earier.
krauss [Wed, 14 Apr 2010 16:15:19 +0200] rev 36137
record package: corrected sort handling in type translations to avoid crashes when default sort is changed.
Test case:
record 'a T = elem :: 'a
defaultsort order
term elem (* low-level exception *)
wenzelm [Wed, 14 Apr 2010 22:08:47 +0200] rev 36136
more precise treatment of UNC server prefix, e.g. //foo;
wenzelm [Wed, 14 Apr 2010 22:07:01 +0200] rev 36135
support named_root, which approximates UNC server prefix (for Cygwin);
tuned representation: reversed elements;
misc simplification and cleanup;
wenzelm [Wed, 14 Apr 2010 11:24:31 +0200] rev 36134
updated Thm.add_axiom/add_def;
wenzelm [Wed, 14 Apr 2010 11:11:23 +0200] rev 36133
adapted PUBLISH_TEST for atbroy102, which only mounts /home/isatest;
huffman [Tue, 13 Apr 2010 11:04:27 -0700] rev 36132
bring HOLCF/ex/Domain_Proofs.thy up to date
blanchet [Tue, 13 Apr 2010 15:30:15 +0200] rev 36131
adapt Refute example to reflect latest soundness fix to Refute
blanchet [Tue, 13 Apr 2010 15:16:54 +0200] rev 36130
commented out unsound "lfp"/"gfp" handling + fixed set output syntax;
the "lfp"/"gfp" bug can be reproduced by looking for a counterexample to
lemma "(A \<union> B)^+ = A^+ \<union> B^+"
Refute incorrectly finds a countermodel for cardinality 1 (the smallest
counterexample requires cardinality 2).
blanchet [Tue, 13 Apr 2010 14:08:58 +0200] rev 36129
merged
blanchet [Tue, 13 Apr 2010 13:26:06 +0200] rev 36128
make Nitpick output everything to tracing in debug mode;
so that when an exception occurs, I can switch to the tracing window to see what was in the response window before the exception blew everything away
blanchet [Tue, 13 Apr 2010 13:24:03 +0200] rev 36127
fix bug in Nitpick's handling of "<" (exposed by "GCD.setprod_coprime_int")
blanchet [Tue, 13 Apr 2010 11:43:11 +0200] rev 36126
cosmetics
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 13 Apr 2010 11:54:05 +0200] rev 36125
merge
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 13 Apr 2010 11:40:55 +0200] rev 36124
merge
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 13 Apr 2010 11:40:03 +0200] rev 36123
add If respectfullness and preservation to Quotient package database
haftmann [Tue, 13 Apr 2010 11:30:12 +0200] rev 36122
more accurate pattern match
haftmann [Tue, 13 Apr 2010 11:13:52 +0200] rev 36121
dropped dead code
huffman [Mon, 12 Apr 2010 19:29:16 -0700] rev 36120
update domain package examples
huffman [Mon, 12 Apr 2010 16:21:27 -0700] rev 36119
remove dead code
huffman [Mon, 12 Apr 2010 16:04:32 -0700] rev 36118
share more code between definitional and axiomatic domain packages
huffman [Mon, 12 Apr 2010 15:05:42 -0700] rev 36117
for axiomatic domain package, declare types and arities in domain_axioms.ML instead of domain_extender.ML
Cezary Kaliszyk <kaliszyk@in.tum.de> [Mon, 12 Apr 2010 13:19:28 +0200] rev 36116
Changed the type of Quot_True, so that it is an HOL constant.