blanchet [Wed, 21 Apr 2010 12:22:04 +0200] rev 36265
distinguish between the different ATP errors in the user interface;
in particular, tell users to upgrade their SPASS if they try to run "spass_tptp" with an old SPASS version with no TPTP support
blanchet [Wed, 21 Apr 2010 11:03:35 +0200] rev 36264
added "spass_tptp" prover, which requires SPASS x.y > 3.0;
once users have upgraded their SPASS and we have determined that "spass_tptp" works well, we can make "spass_tptp" the one and only "spass"
blanchet [Tue, 20 Apr 2010 17:41:00 +0200] rev 36263
use "Proof.goal" in Sledgehammer's minimizer (just like everywhere else in Sledgehammer), not "Proof.raw_goal"
bulwahn [Wed, 21 Apr 2010 12:11:48 +0200] rev 36262
merged
bulwahn [Wed, 21 Apr 2010 12:10:53 +0200] rev 36261
make profiling depend on reference Quickcheck.timing
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36260
added examples for detecting switches
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36259
adopting documentation of the predicate compiler
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36258
removing dead code; clarifying function names; removing clone
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36257
adopting examples to changes in the predicate compiler
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36256
adopting quickcheck
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36255
tuning mutabelle; adding output of mutant theoryfile for interactive evaluation
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36254
added switch detection to the predicate compiler
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36253
added further inlining of boolean constants to the predicate compiler
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36252
adding more profiling to the predicate compiler
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36251
only add relevant predicates to the list of extra modes
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36250
switched off no_topmost_reordering
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36249
replaced call to inductive package by axiomatization in the function flattening of the predicate compiler
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36248
added option for specialisation to the predicate compiler
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36247
prefer functional modes of functions in the mode analysis
bulwahn [Wed, 21 Apr 2010 12:10:52 +0200] rev 36246
added peephole optimisations to the predicate compiler; added structure Predicate_Compile_Simps for peephole optimisations
hoelzl [Wed, 21 Apr 2010 11:23:04 +0200] rev 36245
merged
hoelzl [Wed, 21 Apr 2010 10:44:44 +0200] rev 36244
Only use provided SMT-certificates in HOL-Multivariate_Analysis.
himmelma [Tue, 20 Apr 2010 14:07:52 +0200] rev 36243
Translated remaining theorems about integration from HOL light.
wenzelm [Wed, 21 Apr 2010 11:11:42 +0200] rev 36242
marked cygwin-poly as "e" test, which means further stages do not depend on it (website etc.);
huffman [Tue, 20 Apr 2010 13:44:28 -0700] rev 36241
replace many uses of Drule.export_without_context with Drule.zero_var_indexes
ballarin [Tue, 20 Apr 2010 22:34:17 +0200] rev 36240
Remove garbage.
ballarin [Tue, 20 Apr 2010 22:31:08 +0200] rev 36239
Remove garbage.
wenzelm [Tue, 20 Apr 2010 17:07:53 +0200] rev 36238
recovered isabelle java, which was broken in ebfa4bb0d50f;
blanchet [Tue, 20 Apr 2010 16:14:45 +0200] rev 36237
fix bug in SPASS's DFG output files, where "tc_bool" wasn't declared;
this bug occurs when the explicit "hAPP" or "hBOOL" functions are introduced and full types is activated
blanchet [Tue, 20 Apr 2010 16:04:49 +0200] rev 36236
merged
blanchet [Tue, 20 Apr 2010 16:04:36 +0200] rev 36235
added "explicit_apply" option to Sledgehammer, to control whether an explicit apply function should be used as much or as little as possible (replaces a previous global variable)
blanchet [Tue, 20 Apr 2010 14:39:42 +0200] rev 36234
merge
blanchet [Mon, 19 Apr 2010 19:41:30 +0200] rev 36233
cosmetics
blanchet [Mon, 19 Apr 2010 19:41:15 +0200] rev 36232
don't redo an axiom selection in the first round of Sledgehammer "minimize"!;
this is needlessly slow and messes up the declared functions/predicates in SPASS DFG files
blanchet [Mon, 19 Apr 2010 18:44:12 +0200] rev 36231
get rid of "conjecture_pos", which is no longer necessary now that it's Metis's job, not Sledgehammer's, to report inconsistent contexts
blanchet [Mon, 19 Apr 2010 18:14:45 +0200] rev 36230
added warning about inconsistent context to Metis;
it makes more sense here than in Sledgehammer, because Sledgehammer is unsound and there's no point in having people panicking about the consistency of their context when their context is in fact consistent
blanchet [Mon, 19 Apr 2010 17:18:21 +0200] rev 36229
workaround for Proof General's off-by-a-few sendback display bug, whereby "pr" in "proof" is not highlighted
blanchet [Mon, 19 Apr 2010 16:33:48 +0200] rev 36228
got rid of somewhat pointless "pairname" function in Sledgehammer
blanchet [Mon, 19 Apr 2010 16:33:20 +0200] rev 36227
make Sledgehammer's "add:" and "del:" syntax really work (I hope), by comparing CNF theorems with CNF theorems
blanchet [Mon, 19 Apr 2010 16:29:52 +0200] rev 36226
cosmetics
blanchet [Mon, 19 Apr 2010 15:24:57 +0200] rev 36225
cosmetics
blanchet [Mon, 19 Apr 2010 15:21:35 +0200] rev 36224
cosmetics
blanchet [Mon, 19 Apr 2010 15:15:21 +0200] rev 36223
make Sledgehammer's minimizer also minimize Isar proofs
blanchet [Mon, 19 Apr 2010 11:54:07 +0200] rev 36222
don't use readable names if proof reconstruction is needed, because it uses the structure of names
blanchet [Mon, 19 Apr 2010 11:02:00 +0200] rev 36221
allow "_" in TPTP names in debug mode
blanchet [Mon, 19 Apr 2010 10:45:08 +0200] rev 36220
rename Sledgehammer "theory_const" option to "theory_relevant", now that I understand better what it does
blanchet [Mon, 19 Apr 2010 10:15:02 +0200] rev 36219
set SPASS option on the command-line, so that it doesn't vanish when moving to TPTP format
blanchet [Mon, 19 Apr 2010 09:53:31 +0200] rev 36218
get rid of "List.foldl" + add timestamp to SPASS
wenzelm [Tue, 20 Apr 2010 15:17:18 +0200] rev 36217
less ambitious settings for cygwin-poly;
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 20 Apr 2010 14:56:58 +0200] rev 36216
respectfullness and preservation of map for identity quotients
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 20 Apr 2010 14:56:20 +0200] rev 36215
respectfullness and preservation of function composition
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 20 Apr 2010 14:55:53 +0200] rev 36214
eta-normalize the goal since the original theorem is atomized
wenzelm [Tue, 20 Apr 2010 11:31:14 +0200] rev 36213
accept x86_64 results gracefully -- NB: Mac OS does report that if booted in 64 bit mode;
wenzelm [Tue, 20 Apr 2010 11:26:25 +0200] rev 36212
refer to THIS_JAVA dynamically, and treat ISABELLE_JAVA as static default -- relevant for nested JVM invocation within an existing Isabelle enviroment;
haftmann [Tue, 20 Apr 2010 06:53:50 +0200] rev 36211
merged
haftmann [Mon, 19 Apr 2010 15:31:58 +0200] rev 36210
more appropriate representation of valid positions for abstractors
haftmann [Mon, 19 Apr 2010 15:31:56 +0200] rev 36209
more appropriate representation of valid positions for abstractors; more accurate checking of abstype certificates
wenzelm [Mon, 19 Apr 2010 23:11:39 +0200] rev 36208
update_syntax: add new productions only once, to allow repeated local notation, for example;
wenzelm [Mon, 19 Apr 2010 17:57:07 +0200] rev 36207
tuned;
wenzelm [Mon, 19 Apr 2010 17:31:48 +0200] rev 36206
more platform information;
wenzelm [Mon, 19 Apr 2010 17:27:41 +0200] rev 36205
check JVM platform at most once -- still non-strict to prevent potential failure during initialization of object Platform;
wenzelm [Mon, 19 Apr 2010 16:04:42 +0200] rev 36204
some updates on multi-platform support;
haftmann [Mon, 19 Apr 2010 12:15:06 +0200] rev 36203
merged
haftmann [Mon, 19 Apr 2010 11:30:08 +0200] rev 36202
explicit check sorts in abstract certificates; abstractor is part of dependencies
wenzelm [Mon, 19 Apr 2010 10:56:26 +0200] rev 36201
polyml-platform script is superseded by ISABELLE_PLATFORM;
wenzelm [Mon, 19 Apr 2010 10:19:37 +0200] rev 36200
less ambitious settings for cygwin-poly;
haftmann [Mon, 19 Apr 2010 07:38:35 +0200] rev 36199
merged
haftmann [Mon, 19 Apr 2010 07:38:08 +0200] rev 36198
more convenient equations for zip
wenzelm [Sat, 17 Apr 2010 23:05:52 +0200] rev 36197
more platform info;
wenzelm [Sat, 17 Apr 2010 22:58:29 +0200] rev 36196
added ISABELLE_PLATFORM and ISABELLE_PLATFORM64 -- NB: ML and JVM may have a different idea;
wenzelm [Sat, 17 Apr 2010 21:40:29 +0200] rev 36195
system properties determine the JVM platform, not the Isabelle one;
wenzelm [Sat, 17 Apr 2010 21:01:55 +0200] rev 36194
THIS_CYGWIN;
wenzelm [Sat, 17 Apr 2010 20:42:26 +0200] rev 36193
improved ISABELLE_JAVA, based on THIS_JAVA of the actually running JVM;
wenzelm [Sat, 17 Apr 2010 19:35:35 +0200] rev 36192
isatest: more robust treatment of remote files, less reliance on mounted file system;
blanchet [Sat, 17 Apr 2010 11:05:22 +0200] rev 36191
merged
blanchet [Sat, 17 Apr 2010 10:42:09 +0200] rev 36190
added missing \n in output
blanchet [Fri, 16 Apr 2010 21:18:05 +0200] rev 36189
by default, don't try to start ATPs that aren't installed
blanchet [Fri, 16 Apr 2010 20:51:15 +0200] rev 36188
fiddle with Sledgehammer option syntax
blanchet [Fri, 16 Apr 2010 20:50:50 +0200] rev 36187
added timestamp to proof
blanchet [Fri, 16 Apr 2010 16:54:05 +0200] rev 36186
restore order of clauses in TPTP output;
there's a rather subtle invariant w.r.t. "extract_lemmas"
blanchet [Fri, 16 Apr 2010 16:53:00 +0200] rev 36185
optimize relevance filter by doing a Table.fold directly rather than destroying the datastructure each time;
saves 2 sec per Sledgehammer invocation on my laptop!
blanchet [Fri, 16 Apr 2010 16:51:54 +0200] rev 36184
output total time taken by Sledgehammer if "verbose" is set
blanchet [Fri, 16 Apr 2010 16:13:49 +0200] rev 36183
Sledgehammer: the empty set of fact () should mean nothing, not unchanged
blanchet [Fri, 16 Apr 2010 16:08:43 +0200] rev 36182
reorganize Sledgehammer's relevance filter slightly
blanchet [Fri, 16 Apr 2010 15:59:53 +0200] rev 36181
tell the user that Sledgehammer kills its siblings
wenzelm [Fri, 16 Apr 2010 22:52:49 +0200] rev 36180
updated keywords;
wenzelm [Fri, 16 Apr 2010 22:45:07 +0200] rev 36179
replaced old Sign.add_tyabbrs(_i) by Sign.add_type_abbrev (without mixfix);
misc tuning and simplification;
wenzelm [Fri, 16 Apr 2010 22:18:59 +0200] rev 36178
keep localized 'types' as regular non-old-style version -- 'type_abbrev' as 'type' just causes too many problems, e.g. clash with "type" in translations or "type:" argument syntax;
wenzelm [Fri, 16 Apr 2010 22:15:09 +0200] rev 36177
separate commands 'hide_class', 'hide_type', 'hide_const', 'hide_fact';
wenzelm [Fri, 16 Apr 2010 21:28:09 +0200] rev 36176
replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
wenzelm [Fri, 16 Apr 2010 20:56:40 +0200] rev 36175
allow syntax types within abbreviations;
wenzelm [Fri, 16 Apr 2010 20:17:38 +0200] rev 36174
modernized old-style type abbreviations;
wenzelm [Fri, 16 Apr 2010 19:58:04 +0200] rev 36173
modernized type abbreviations;
wenzelm [Fri, 16 Apr 2010 19:43:06 +0200] rev 36172
local type abbreviations;
blanchet [Fri, 16 Apr 2010 15:49:46 +0200] rev 36171
merged
blanchet [Fri, 16 Apr 2010 15:49:13 +0200] rev 36170
added original constant names to Sledgehammer internal terms + output short names if "debug" is set (for increased readability)
blanchet [Fri, 16 Apr 2010 14:48:34 +0200] rev 36169
store nonmangled names along with mangled type names in Sledgehammer for debugging purposes
blanchet [Thu, 15 Apr 2010 13:57:17 +0200] rev 36168
give more sensible names to "fol_type" constructors, as requested by a FIXME comment
blanchet [Thu, 15 Apr 2010 13:49:46 +0200] rev 36167
make Sledgehammer's output more debugging friendly
wenzelm [Fri, 16 Apr 2010 12:51:57 +0200] rev 36166
made SML/NJ happy;
wenzelm [Fri, 16 Apr 2010 12:51:37 +0200] rev 36165
proper masking of dummy name_space;
wenzelm [Fri, 16 Apr 2010 11:40:01 +0200] rev 36164
salvaged some ML functors from decay, which is the natural consequence of lack of formal checking;
wenzelm [Fri, 16 Apr 2010 11:39:08 +0200] rev 36163
proper checking of ML functors (in Poly/ML 5.2 or later);
eliminated pathetic comments;
wenzelm [Fri, 16 Apr 2010 10:52:10 +0200] rev 36162
added ML antiquotation @{make_string}, which produces proper pretty printed version in Poly/ML 5.3.0 or later;
wenzelm [Fri, 16 Apr 2010 10:15:00 +0200] rev 36161
isatest: improved treatment of local files on atbroy102;
huffman [Thu, 15 Apr 2010 18:21:05 -0700] rev 36160
add rule deflation_ID to proof script for take + constructor rules
wenzelm [Thu, 15 Apr 2010 21:24:00 +0200] rev 36159
more robust record syntax: use Type.raw_match to ignore sort constraints as in regular abbreviations (also note that constraints only affect operations, not types);
wenzelm [Thu, 15 Apr 2010 20:56:04 +0200] rev 36158
HOL record: explicitly allow sort constraints;
wenzelm [Thu, 15 Apr 2010 20:37:27 +0200] rev 36157
misc tuning and simplification;
wenzelm [Thu, 15 Apr 2010 20:31:21 +0200] rev 36156
explicit ProofContext.check_tfree;
wenzelm [Thu, 15 Apr 2010 18:13:25 +0200] rev 36155
merged
Cezary Kaliszyk <kaliszyk@in.tum.de> [Thu, 15 Apr 2010 16:55:12 +0200] rev 36154
Respectfullness and preservation of list_rel
wenzelm [Thu, 15 Apr 2010 18:09:22 +0200] rev 36153
replaced slightly odd Typedecl.predeclare_constraints by plain declaration of type arguments -- also avoid "recursive" declaration of type constructor, which can cause problems with sequential definitions B.foo = A.foo;
simplified via ProofContext.check_tfree;
wenzelm [Thu, 15 Apr 2010 18:00:21 +0200] rev 36152
get_sort: suppress dummyS from input;
added check_tvar, check_tfree convenience;
tuned;
wenzelm [Thu, 15 Apr 2010 16:58:12 +0200] rev 36151
modernized treatment of sort constraints in specification;
pass-through type variables as usual as (string * sort) internally -- recovers proper sort handling;
wenzelm [Thu, 15 Apr 2010 16:55:49 +0200] rev 36150
typecopy: observe given sort constraints more precisely;
wenzelm [Thu, 15 Apr 2010 15:39:50 +0200] rev 36149
inline old Record.read_typ/cert_typ;
spelling;
wenzelm [Thu, 15 Apr 2010 15:38:58 +0200] rev 36148
spelling;
haftmann [Thu, 15 Apr 2010 12:27:14 +0200] rev 36147
theory RBT with abstract type of red-black trees backed by implementation RBT_Impl
wenzelm [Wed, 14 Apr 2010 22:18:10 +0200] rev 36146
tuned whitespace;
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.
haftmann [Sun, 11 Apr 2010 17:46:42 +0200] rev 36115
removed rather toyish tree
haftmann [Sun, 11 Apr 2010 17:40:43 +0200] rev 36114
updated keywords
haftmann [Sun, 11 Apr 2010 16:51:36 +0200] rev 36113
merged
haftmann [Sun, 11 Apr 2010 16:51:07 +0200] rev 36112
user interface for abstract datatypes is an attribute, not a command
haftmann [Sun, 11 Apr 2010 16:51:06 +0200] rev 36111
implementation of mappings by rbts
haftmann [Sun, 11 Apr 2010 16:51:06 +0200] rev 36110
lemma is_empty_empty
haftmann [Sun, 11 Apr 2010 16:51:05 +0200] rev 36109
constructor Mapping replaces AList
wenzelm [Sun, 11 Apr 2010 15:42:05 +0200] rev 36108
stay within Local_Defs layer;
wenzelm [Sun, 11 Apr 2010 15:22:15 +0200] rev 36107
expose foundational typedef axiom name;
wenzelm [Sun, 11 Apr 2010 14:30:34 +0200] rev 36106
Thm.add_axiom/add_def: return internal name of foundational axiom;
wenzelm [Sun, 11 Apr 2010 14:06:35 +0200] rev 36105
modernized datatype constructors;
wenzelm [Sun, 11 Apr 2010 14:04:10 +0200] rev 36104
of_sort_derivation: weaken bypasses derivation for identical sort -- accomodate proof terms by krauss/schropp, for example;
wenzelm [Sun, 11 Apr 2010 13:13:23 +0200] rev 36103
tuned;
wenzelm [Sun, 11 Apr 2010 13:08:14 +0200] rev 36102
of_sort_derivation: pass-through full type information -- following the version by krauss/schropp;
wenzelm [Fri, 09 Apr 2010 13:35:54 +0200] rev 36101
include JEDIT_APPLE_PROPERTIES by default;
wenzelm [Fri, 09 Apr 2010 11:35:50 +0200] rev 36100
isatest: more uniform setup for Unix vs. Cygwin;
boehmes [Thu, 08 Apr 2010 22:39:06 +0200] rev 36099
added missing case: meta universal quantifier
bulwahn [Thu, 08 Apr 2010 08:17:27 +0200] rev 36098
added imperative SAT checker; improved headers of example files; adopted IsaMakefile
ballarin [Wed, 07 Apr 2010 22:22:49 +0200] rev 36097
Merged.
ballarin [Wed, 07 Apr 2010 19:17:10 +0200] rev 36096
Merged resolving conflicts NEWS and locale.ML.
ballarin [Fri, 02 Apr 2010 13:33:48 +0200] rev 36095
Proper inheritance of mixins for activated facts and locale dependencies.
ballarin [Mon, 15 Feb 2010 19:54:54 +0100] rev 36094
Removed obsolete function.
ballarin [Mon, 15 Feb 2010 01:34:08 +0100] rev 36093
Graceful treatment of non-locale subgoals by methods unfold_locales and intro_locales.
ballarin [Mon, 15 Feb 2010 01:27:06 +0100] rev 36092
Tuned interpretation proofs.
ballarin [Thu, 11 Feb 2010 21:00:36 +0100] rev 36091
A rough implementation of full mixin inheritance; additional unit tests.
ballarin [Tue, 02 Feb 2010 21:23:20 +0100] rev 36090
Clarified invariant; tuned.
ballarin [Mon, 01 Feb 2010 21:59:27 +0100] rev 36089
More mixin tests.
ballarin [Mon, 01 Feb 2010 21:55:00 +0100] rev 36088
Use serial to be more debug friendly.
boehmes [Wed, 07 Apr 2010 20:40:42 +0200] rev 36087
buffered output (faster than direct output)
boehmes [Wed, 07 Apr 2010 20:40:42 +0200] rev 36086
simplified Cache_IO interface (input is just a string and not already stored in a file)
boehmes [Wed, 07 Apr 2010 20:40:42 +0200] rev 36085
shortened interface (do not export unused options and functions)
boehmes [Wed, 07 Apr 2010 20:40:42 +0200] rev 36084
always unfold definitions of specific constants (including special binders)
boehmes [Wed, 07 Apr 2010 20:40:42 +0200] rev 36083
shorten the code by conditional function application
boehmes [Wed, 07 Apr 2010 20:38:11 +0200] rev 36082
fail for problems containg the universal sort (as those problems cannot be atomized)
boehmes [Wed, 07 Apr 2010 19:48:58 +0200] rev 36081
renamed "smt_record" to "smt_fixed" (somewhat more expressive) and inverted its semantics
hoelzl [Wed, 07 Apr 2010 17:24:44 +0200] rev 36080
Added Information theory and Example: dining cryptographers
Christian Urban <urbanc@in.tum.de> [Wed, 07 Apr 2010 11:05:11 +0200] rev 36079
simplified induction case in finite_psubset_induct; tuned the proof that uses this induction principle
krauss [Tue, 06 Apr 2010 11:00:57 +0200] rev 36078
removed (latex output) notation which is sometimes very ugly
boehmes [Tue, 06 Apr 2010 10:48:16 +0200] rev 36077
merged
boehmes [Tue, 06 Apr 2010 10:46:28 +0200] rev 36076
added missing mult_1_left to linarith simp rules
krauss [Tue, 06 Apr 2010 09:27:03 +0200] rev 36075
tuned proof (no induction needed); removed unused lemma and fuzzy comment
wenzelm [Fri, 02 Apr 2010 17:20:43 +0200] rev 36074
isatest: basic setup for cygwin-poly on atbroy102;