Sat, 26 Mar 2011 12:01:40 +0100 added Syntax.const_abs_tr' with proper eta_abs and Term.is_dependent;
wenzelm [Sat, 26 Mar 2011 12:01:40 +0100] rev 42086
added Syntax.const_abs_tr' with proper eta_abs and Term.is_dependent; recovered printing of Hoare assign statements from 45d090186bbe;
Sat, 26 Mar 2011 10:52:29 +0100 tuned;
wenzelm [Sat, 26 Mar 2011 10:52:29 +0100] rev 42085
tuned;
Sat, 26 Mar 2011 10:25:17 +0100 dependent_tr': formal treatment of bounds after stripping Abs, although it should only happen for malformed terms, since print_translations work top-down;
wenzelm [Sat, 26 Mar 2011 10:25:17 +0100] rev 42084
dependent_tr': formal treatment of bounds after stripping Abs, although it should only happen for malformed terms, since print_translations work top-down;
Thu, 24 Mar 2011 16:56:19 +0100 added Term.is_open and Term.is_dependent convenience, to cover common situations of loose bounds;
wenzelm [Thu, 24 Mar 2011 16:56:19 +0100] rev 42083
added Term.is_open and Term.is_dependent convenience, to cover common situations of loose bounds;
Thu, 24 Mar 2011 16:47:24 +0100 more direct loose_bvar1;
wenzelm [Thu, 24 Mar 2011 16:47:24 +0100] rev 42082
more direct loose_bvar1; tuned;
Thu, 24 Mar 2011 13:54:39 +0100 indentation;
wenzelm [Thu, 24 Mar 2011 13:54:39 +0100] rev 42081
indentation;
Thu, 24 Mar 2011 11:45:39 +0100 update_name: more uniform treatment of type constraints (NB: type equality is hard to establish in parse trees);
wenzelm [Thu, 24 Mar 2011 11:45:39 +0100] rev 42080
update_name: more uniform treatment of type constraints (NB: type equality is hard to establish in parse trees);
Wed, 23 Mar 2011 21:07:05 +0100 added editor mode line;
wenzelm [Wed, 23 Mar 2011 21:07:05 +0100] rev 42079
added editor mode line;
Wed, 23 Mar 2011 20:57:37 +0100 isolate change of Proofterm.proofs in TPTP.thy from rest of session;
wenzelm [Wed, 23 Mar 2011 20:57:37 +0100] rev 42078
isolate change of Proofterm.proofs in TPTP.thy from rest of session; qualified Proofterm.proofs to facilitate grepping;
Wed, 23 Mar 2011 20:51:36 +0100 list Isabelle tools via perl script, which is much faster that bash plumbing, especially on Cygwin;
wenzelm [Wed, 23 Mar 2011 20:51:36 +0100] rev 42077
list Isabelle tools via perl script, which is much faster that bash plumbing, especially on Cygwin; exclude backup files;
Wed, 23 Mar 2011 16:42:09 +0100 updated contributed components
boehmes [Wed, 23 Mar 2011 16:42:09 +0100] rev 42076
updated contributed components
Wed, 23 Mar 2011 15:33:17 +0100 Z3 non-commercial usage may explicitly be declined
boehmes [Wed, 23 Mar 2011 15:33:17 +0100] rev 42075
Z3 non-commercial usage may explicitly be declined
Wed, 23 Mar 2011 14:29:29 +0100 export status function to query whether Z3 has been activated for usage within Isabelle
boehmes [Wed, 23 Mar 2011 14:29:29 +0100] rev 42074
export status function to query whether Z3 has been activated for usage within Isabelle
Wed, 23 Mar 2011 10:38:50 +0100 merge
blanchet [Wed, 23 Mar 2011 10:38:50 +0100] rev 42073
merge
Wed, 23 Mar 2011 10:18:42 +0100 avoid illegal variable names, which then yield "Not an identifier" errors in "rename_tac"
blanchet [Wed, 23 Mar 2011 10:18:42 +0100] rev 42072
avoid illegal variable names, which then yield "Not an identifier" errors in "rename_tac"
Wed, 23 Mar 2011 10:06:27 +0100 move "TPTP" wrapper and "Sledgehammer as a tactic" to "HOL/ex"
blanchet [Wed, 23 Mar 2011 10:06:27 +0100] rev 42071
move "TPTP" wrapper and "Sledgehammer as a tactic" to "HOL/ex" default to "e" rather than "vampire" since E is part of the Isabelle bundle
Wed, 23 Mar 2011 10:21:29 +0100 really be quiet
boehmes [Wed, 23 Mar 2011 10:21:29 +0100] rev 42070
really be quiet
Wed, 23 Mar 2011 09:15:49 +0100 replace hardwired MIRABELLE_OUTPUT_PATH by temporary directory derived from ISABELLE_TMP_PREFIX and $$ -- old behaviour can be achieved by manually setting MIRABELLE_OUTPUT_PATH
krauss [Wed, 23 Mar 2011 09:15:49 +0100] rev 42069
replace hardwired MIRABELLE_OUTPUT_PATH by temporary directory derived from ISABELLE_TMP_PREFIX and $$ -- old behaviour can be achieved by manually setting MIRABELLE_OUTPUT_PATH
Tue, 22 Mar 2011 21:22:50 +0100 merged
wenzelm [Tue, 22 Mar 2011 21:22:50 +0100] rev 42068
merged
Tue, 22 Mar 2011 20:06:10 +0100 standardized headers
hoelzl [Tue, 22 Mar 2011 20:06:10 +0100] rev 42067
standardized headers
Tue, 22 Mar 2011 18:53:05 +0100 generalized Caratheodory from algebra to ring_of_sets
hoelzl [Tue, 22 Mar 2011 18:53:05 +0100] rev 42066
generalized Caratheodory from algebra to ring_of_sets
Tue, 22 Mar 2011 16:44:57 +0100 add ring_of_sets and subset_class as basis for algebra
hoelzl [Tue, 22 Mar 2011 16:44:57 +0100] rev 42065
add ring_of_sets and subset_class as basis for algebra
Tue, 22 Mar 2011 19:04:32 +0100 added first-order TPTP version of Nitpick to Isabelle, so that its sources stay in sync with Isabelle and it is easier to install new versions for SystemOnTPTP and CASC -- the tool is called "isabelle nitrox" but is deliberately omitted from the tool list unless the component is explicitly enabled, to avoid clutter
blanchet [Tue, 22 Mar 2011 19:04:32 +0100] rev 42064
added first-order TPTP version of Nitpick to Isabelle, so that its sources stay in sync with Isabelle and it is easier to install new versions for SystemOnTPTP and CASC -- the tool is called "isabelle nitrox" but is deliberately omitted from the tool list unless the component is explicitly enabled, to avoid clutter
Tue, 22 Mar 2011 18:38:29 +0100 added "TPTP" theory with IsabelleP tactic, so that it is maintained alongside with Isabelle and that the CASC version of Isabelle is provided by Isabelle itself instead of being stored on the TPTP servers
blanchet [Tue, 22 Mar 2011 18:38:29 +0100] rev 42063
added "TPTP" theory with IsabelleP tactic, so that it is maintained alongside with Isabelle and that the CASC version of Isabelle is provided by Isabelle itself instead of being stored on the TPTP servers
Tue, 22 Mar 2011 18:27:47 +0100 remove lie from documentation
blanchet [Tue, 22 Mar 2011 18:27:47 +0100] rev 42062
remove lie from documentation
Tue, 22 Mar 2011 17:20:54 +0100 let SMT errors through -- the main reason for keeping them quiet was that the SMT bridge used to suffer from internal bugs, but these have been fixed for some time now
blanchet [Tue, 22 Mar 2011 17:20:54 +0100] rev 42061
let SMT errors through -- the main reason for keeping them quiet was that the SMT bridge used to suffer from internal bugs, but these have been fixed for some time now
Tue, 22 Mar 2011 17:20:53 +0100 make Minimizer honor "verbose" and "debug" options better
blanchet [Tue, 22 Mar 2011 17:20:53 +0100] rev 42060
make Minimizer honor "verbose" and "debug" options better
Tue, 22 Mar 2011 12:49:07 +0100 fixed a printing problem for bounded quantifiers and bounded set operators in the case of tuples
nipkow [Tue, 22 Mar 2011 12:49:07 +0100] rev 42059
fixed a printing problem for bounded quantifiers and bounded set operators in the case of tuples
Mon, 21 Mar 2011 21:10:29 +0100 moved some configurations to AFP, and fixed others
krauss [Mon, 21 Mar 2011 21:10:29 +0100] rev 42058
moved some configurations to AFP, and fixed others
Tue, 22 Mar 2011 20:44:47 +0100 more selective strip_positions in case patterns -- reactivate translations based on "case _ of _" in HOL and special patterns in HOLCF;
wenzelm [Tue, 22 Mar 2011 20:44:47 +0100] rev 42057
more selective strip_positions in case patterns -- reactivate translations based on "case _ of _" in HOL and special patterns in HOLCF;
Tue, 22 Mar 2011 18:03:28 +0100 enable inner syntax source positions by default (controlled via configuration option);
wenzelm [Tue, 22 Mar 2011 18:03:28 +0100] rev 42056
enable inner syntax source positions by default (controlled via configuration option); disable source positions for HOLCF, due to special pattern translations;
Tue, 22 Mar 2011 17:51:15 +0100 binder_tr: more informative exception;
wenzelm [Tue, 22 Mar 2011 17:51:15 +0100] rev 42055
binder_tr: more informative exception;
Tue, 22 Mar 2011 16:39:34 +0100 Hoare syntax: strip positions where they crash translation functions;
wenzelm [Tue, 22 Mar 2011 16:39:34 +0100] rev 42054
Hoare syntax: strip positions where they crash translation functions; re-unified some clones (!);
Tue, 22 Mar 2011 16:15:50 +0100 update_name_tr: more precise handling of explicit constraints, including positions;
wenzelm [Tue, 22 Mar 2011 16:15:50 +0100] rev 42053
update_name_tr: more precise handling of explicit constraints, including positions;
Tue, 22 Mar 2011 15:32:47 +0100 statespace syntax: strip positions -- type constraints are unexpected here;
wenzelm [Tue, 22 Mar 2011 15:32:47 +0100] rev 42052
statespace syntax: strip positions -- type constraints are unexpected here;
Tue, 22 Mar 2011 14:45:48 +0100 let syntax: reverted to plain "id", since translations cannot cope with constraints (notably position information);
wenzelm [Tue, 22 Mar 2011 14:45:48 +0100] rev 42051
let syntax: reverted to plain "id", since translations cannot cope with constraints (notably position information);
Tue, 22 Mar 2011 14:22:40 +0100 datatype case_tr: strip positions -- type constraints are unexpected despite the "any" category in "case_syn";
wenzelm [Tue, 22 Mar 2011 14:22:40 +0100] rev 42050
datatype case_tr: strip positions -- type constraints are unexpected despite the "any" category in "case_syn";
Tue, 22 Mar 2011 13:55:39 +0100 tuned indendation and parentheses;
wenzelm [Tue, 22 Mar 2011 13:55:39 +0100] rev 42049
tuned indendation and parentheses;
Tue, 22 Mar 2011 13:32:20 +0100 support for encoded positions (for id_position, longid_position) as pseudo type-constraints -- still inactive;
wenzelm [Tue, 22 Mar 2011 13:32:20 +0100] rev 42048
support for encoded positions (for id_position, longid_position) as pseudo type-constraints -- still inactive; simplified/generalized abs_tr/binder_tr: allow iterated constraints, stemming from positions; Ast.pretty_ast: special treatment of encoded positions; eliminated Ast.str_of_ast in favour of uniform Ast.pretty_ast;
Tue, 22 Mar 2011 11:14:33 +0100 pretty_string: proper handling of negative max_len;
wenzelm [Tue, 22 Mar 2011 11:14:33 +0100] rev 42047
pretty_string: proper handling of negative max_len;
Mon, 21 Mar 2011 23:38:32 +0100 added Lexicon.encode_position, Lexicon.decode_position;
wenzelm [Mon, 21 Mar 2011 23:38:32 +0100] rev 42046
added Lexicon.encode_position, Lexicon.decode_position;
Mon, 21 Mar 2011 21:16:39 +0100 tuned;
wenzelm [Mon, 21 Mar 2011 21:16:39 +0100] rev 42045
tuned;
Mon, 21 Mar 2011 21:05:08 +0100 tuned;
wenzelm [Mon, 21 Mar 2011 21:05:08 +0100] rev 42044
tuned;
Mon, 21 Mar 2011 20:56:44 +0100 clarified Syn_Trans.parsetree_to_ast and Syn_Trans.ast_to_term;
wenzelm [Mon, 21 Mar 2011 20:56:44 +0100] rev 42043
clarified Syn_Trans.parsetree_to_ast and Syn_Trans.ast_to_term;
Mon, 21 Mar 2011 20:15:03 +0100 tuned;
wenzelm [Mon, 21 Mar 2011 20:15:03 +0100] rev 42042
tuned;
Mon, 21 Mar 2011 17:14:52 +0100 merged
wenzelm [Mon, 21 Mar 2011 17:14:52 +0100] rev 42041
merged
Mon, 21 Mar 2011 16:24:52 +0100 added judgement day configurations
krauss [Mon, 21 Mar 2011 16:24:52 +0100] rev 42040
added judgement day configurations
Mon, 21 Mar 2011 16:38:28 +0100 another attempt to exec ISABELLE_GHC robustly (cf. d8c3b26b3da4, 994d088fbfbc);
wenzelm [Mon, 21 Mar 2011 16:38:28 +0100] rev 42039
another attempt to exec ISABELLE_GHC robustly (cf. d8c3b26b3da4, 994d088fbfbc);
Mon, 21 Mar 2011 14:46:59 +0100 fixed perl error
krauss [Mon, 21 Mar 2011 14:46:59 +0100] rev 42038
fixed perl error
Mon, 21 Mar 2011 14:37:10 +0100 eliminated unnecessary generated ROOT.ML
krauss [Mon, 21 Mar 2011 14:37:10 +0100] rev 42037
eliminated unnecessary generated ROOT.ML
Mon, 21 Mar 2011 14:25:59 +0100 more precise dependencies
krauss [Mon, 21 Mar 2011 14:25:59 +0100] rev 42036
more precise dependencies
Mon, 21 Mar 2011 12:43:26 +0100 small test case for main mirabelle functionality, which easily breaks without noticing
krauss [Mon, 21 Mar 2011 12:43:26 +0100] rev 42035
small test case for main mirabelle functionality, which easily breaks without noticing
Mon, 21 Mar 2011 12:43:25 +0100 propagate mirabelle failures properly;
krauss [Mon, 21 Mar 2011 12:43:25 +0100] rev 42034
propagate mirabelle failures properly; flatten obscure return code semantics of Perl system command to 0/1
Mon, 21 Mar 2011 12:43:23 +0100 mirabelle: create modified theory file in original location, to ensure that its dependencies can be found (cf. aa8dce9ab8a9)
krauss [Mon, 21 Mar 2011 12:43:23 +0100] rev 42033
mirabelle: create modified theory file in original location, to ensure that its dependencies can be found (cf. aa8dce9ab8a9)
Mon, 21 Mar 2011 08:29:16 +0100 merged
bulwahn [Mon, 21 Mar 2011 08:29:16 +0100] rev 42032
merged
Fri, 18 Mar 2011 18:19:42 +0100 adapting predicate_compile_quickcheck; tuned
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42031
adapting predicate_compile_quickcheck; tuned
Fri, 18 Mar 2011 18:19:42 +0100 adapting mutabelle
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42030
adapting mutabelle
Fri, 18 Mar 2011 18:19:42 +0100 adapting SML_Quickcheck
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42029
adapting SML_Quickcheck
Fri, 18 Mar 2011 18:19:42 +0100 passing a term with free variables to the quickcheck tester functions instead of an lambda expression because this is more natural with passing further evaluation terms; added output of evaluation terms; added evaluation of terms in the exhaustive testing
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42028
passing a term with free variables to the quickcheck tester functions instead of an lambda expression because this is more natural with passing further evaluation terms; added output of evaluation terms; added evaluation of terms in the exhaustive testing
Fri, 18 Mar 2011 18:19:42 +0100 extending the test data generators to take the evaluation terms as arguments
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42027
extending the test data generators to take the evaluation terms as arguments
Fri, 18 Mar 2011 18:19:42 +0100 adding option of evaluating terms after invocation in quickcheck
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42026
adding option of evaluating terms after invocation in quickcheck
Fri, 18 Mar 2011 18:19:42 +0100 adding eval option to quickcheck
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42025
adding eval option to quickcheck
Fri, 18 Mar 2011 18:19:42 +0100 handling a quite restricted set of functions in Quickcheck_Narrowing by an easy transformation
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42024
handling a quite restricted set of functions in Quickcheck_Narrowing by an easy transformation
Fri, 18 Mar 2011 18:19:42 +0100 adding minimalistic setup and transformation to handle functions as data to enable naive function generation for Quickcheck_Narrowing
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42023
adding minimalistic setup and transformation to handle functions as data to enable naive function generation for Quickcheck_Narrowing
Fri, 18 Mar 2011 18:19:42 +0100 adding a simple datatype for representing functions in Quickcheck_Narrowing
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42022
adding a simple datatype for representing functions in Quickcheck_Narrowing
Fri, 18 Mar 2011 18:19:42 +0100 extending code_int type more; adding narrowing instance for type int; added test case for int instance
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42021
extending code_int type more; adding narrowing instance for type int; added test case for int instance
Fri, 18 Mar 2011 18:19:42 +0100 translating bash output in quickcheck_narrowing to handle special characters; adding simple test cases
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42020
translating bash output in quickcheck_narrowing to handle special characters; adding simple test cases
Fri, 18 Mar 2011 18:19:42 +0100 adding size as static argument in quickcheck_narrowing compilation
bulwahn [Fri, 18 Mar 2011 18:19:42 +0100] rev 42019
adding size as static argument in quickcheck_narrowing compilation
Sun, 20 Mar 2011 23:07:06 +0100 modernized specifications;
wenzelm [Sun, 20 Mar 2011 23:07:06 +0100] rev 42018
modernized specifications;
Sun, 20 Mar 2011 22:48:08 +0100 dropped unused structure aliases;
wenzelm [Sun, 20 Mar 2011 22:48:08 +0100] rev 42017
dropped unused structure aliases;
Sun, 20 Mar 2011 22:47:08 +0100 tuned;
wenzelm [Sun, 20 Mar 2011 22:47:08 +0100] rev 42016
tuned;
Sun, 20 Mar 2011 22:26:43 +0100 NEWS: structure Timing provides various operations for timing;
wenzelm [Sun, 20 Mar 2011 22:26:43 +0100] rev 42015
NEWS: structure Timing provides various operations for timing;
Sun, 20 Mar 2011 22:08:12 +0100 simplified various cpu_time clones (!): eliminated odd Exn.capture/Exn.release (no need to "stop" timing);
wenzelm [Sun, 20 Mar 2011 22:08:12 +0100] rev 42014
simplified various cpu_time clones (!): eliminated odd Exn.capture/Exn.release (no need to "stop" timing);
Sun, 20 Mar 2011 21:44:38 +0100 pure Timing.timing, without any exception handling;
wenzelm [Sun, 20 Mar 2011 21:44:38 +0100] rev 42013
pure Timing.timing, without any exception handling; clarified cond_timeit: propagate interrupt without side-effect;
Sun, 20 Mar 2011 21:28:11 +0100 structure Timing: covers former start_timing/end_timing and Output.timeit etc;
wenzelm [Sun, 20 Mar 2011 21:28:11 +0100] rev 42012
structure Timing: covers former start_timing/end_timing and Output.timeit etc; explicit Timing.message function; eliminated Output.timing flag, cf. Toplevel.timing; tuned;
Sun, 20 Mar 2011 21:20:07 +0100 pervasive cond_timeit;
wenzelm [Sun, 20 Mar 2011 21:20:07 +0100] rev 42011
pervasive cond_timeit;
Sun, 20 Mar 2011 20:20:41 +0100 eliminated dead code;
wenzelm [Sun, 20 Mar 2011 20:20:41 +0100] rev 42010
eliminated dead code;
Sun, 20 Mar 2011 20:05:43 +0100 parallel preparation of document variants, within separate directories;
wenzelm [Sun, 20 Mar 2011 20:05:43 +0100] rev 42009
parallel preparation of document variants, within separate directories;
Sun, 20 Mar 2011 19:47:26 +0100 Present.init/finish/no_document are not thread-safe -- eliminated futile CRITICAL sections;
wenzelm [Sun, 20 Mar 2011 19:47:26 +0100] rev 42008
Present.init/finish/no_document are not thread-safe -- eliminated futile CRITICAL sections; tuned;
Sun, 20 Mar 2011 19:34:18 +0100 eliminated redundant doc_prefix1;
wenzelm [Sun, 20 Mar 2011 19:34:18 +0100] rev 42007
eliminated redundant doc_prefix1; tuned;
Sun, 20 Mar 2011 19:10:09 +0100 renamed doc_prefix2 to dump_prefix;
wenzelm [Sun, 20 Mar 2011 19:10:09 +0100] rev 42006
renamed doc_prefix2 to dump_prefix;
Sun, 20 Mar 2011 18:56:36 +0100 tuned;
wenzelm [Sun, 20 Mar 2011 18:56:36 +0100] rev 42005
tuned;
Sun, 20 Mar 2011 18:09:32 +0100 tuned terminology for document variants;
wenzelm [Sun, 20 Mar 2011 18:09:32 +0100] rev 42004
tuned terminology for document variants;
Sun, 20 Mar 2011 17:40:45 +0100 replaced File.check by specific File.check_file, File.check_dir;
wenzelm [Sun, 20 Mar 2011 17:40:45 +0100] rev 42003
replaced File.check by specific File.check_file, File.check_dir; clarified File.full_path -- include parts of former Thy_Load.get_file; simplified Thy_Load.check_file -- do not read/digest yet; merged Thy_Load.check_thy/deps_thy -- always read text and parse header; clarified Thy_Header.read -- NB: partial Path.explode outside of args parser combinator; Thy_Info.check_deps etc.: File.read exactly once;
Sun, 20 Mar 2011 13:49:21 +0100 tuned;
wenzelm [Sun, 20 Mar 2011 13:49:21 +0100] rev 42002
tuned;
Sat, 19 Mar 2011 14:03:13 +0100 preencode value of "need" selectors in Kodkod bounds as an optimization
blanchet [Sat, 19 Mar 2011 14:03:13 +0100] rev 42001
preencode value of "need" selectors in Kodkod bounds as an optimization
Sat, 19 Mar 2011 11:22:23 +0100 ignore "need" axioms for "nat"-like types
blanchet [Sat, 19 Mar 2011 11:22:23 +0100] rev 42000
ignore "need" axioms for "nat"-like types
Fri, 18 Mar 2011 22:55:28 +0100 added "simp:", "intro:", and "elim:" to "try" command
blanchet [Fri, 18 Mar 2011 22:55:28 +0100] rev 41999
added "simp:", "intro:", and "elim:" to "try" command
Fri, 18 Mar 2011 17:27:28 +0100 optimize Kodkod axioms further w.r.t. "need" option
blanchet [Fri, 18 Mar 2011 17:27:28 +0100] rev 41998
optimize Kodkod axioms further w.r.t. "need" option
Fri, 18 Mar 2011 12:20:32 +0100 optimize Kodkod bounds of nat-like datatypes
blanchet [Fri, 18 Mar 2011 12:20:32 +0100] rev 41997
optimize Kodkod bounds of nat-like datatypes
Fri, 18 Mar 2011 12:05:23 +0100 more optimizations of bounds for "need"
blanchet [Fri, 18 Mar 2011 12:05:23 +0100] rev 41996
more optimizations of bounds for "need"
Fri, 18 Mar 2011 11:43:28 +0100 optimize Kodkod bounds when "need" is specified
blanchet [Fri, 18 Mar 2011 11:43:28 +0100] rev 41995
optimize Kodkod bounds when "need" is specified
Fri, 18 Mar 2011 10:17:37 +0100 always destroy constructor patterns, since this seems to be always useful
blanchet [Fri, 18 Mar 2011 10:17:37 +0100] rev 41994
always destroy constructor patterns, since this seems to be always useful
Thu, 17 Mar 2011 22:07:17 +0100 reintroduced "show_skolems" option -- useful when too many Skolems are displayed
blanchet [Thu, 17 Mar 2011 22:07:17 +0100] rev 41993
reintroduced "show_skolems" option -- useful when too many Skolems are displayed
Thu, 17 Mar 2011 14:43:53 +0100 reword Nitpick's wording concerning potential counterexamples
blanchet [Thu, 17 Mar 2011 14:43:53 +0100] rev 41992
reword Nitpick's wording concerning potential counterexamples
Thu, 17 Mar 2011 14:43:51 +0100 prevent an exception if "card" is empty (e.g., "nitpick [card]")
blanchet [Thu, 17 Mar 2011 14:43:51 +0100] rev 41991
prevent an exception if "card" is empty (e.g., "nitpick [card]")
Thu, 17 Mar 2011 11:18:31 +0100 add option to function to keep trivial ATP formulas, needed for some experiments
blanchet [Thu, 17 Mar 2011 11:18:31 +0100] rev 41990
add option to function to keep trivial ATP formulas, needed for some experiments
Thu, 17 Mar 2011 11:18:31 +0100 add option to relevance filter's "all_facts" function to really get all facts (needed for some experiments)
blanchet [Thu, 17 Mar 2011 11:18:31 +0100] rev 41989
add option to relevance filter's "all_facts" function to really get all facts (needed for some experiments)
Thu, 17 Mar 2011 09:58:13 +0100 tuned lemma
nipkow [Thu, 17 Mar 2011 09:58:13 +0100] rev 41988
tuned lemma
Wed, 16 Mar 2011 19:50:56 +0100 added lemmas
nipkow [Wed, 16 Mar 2011 19:50:56 +0100] rev 41987
added lemmas
Tue, 15 Mar 2011 22:04:02 +0100 added lemma
nipkow [Tue, 15 Mar 2011 22:04:02 +0100] rev 41986
added lemma
Tue, 15 Mar 2011 15:49:42 +0100 support non-ground "need" values
blanchet [Tue, 15 Mar 2011 15:49:42 +0100] rev 41985
support non-ground "need" values
Tue, 15 Mar 2011 13:03:54 +0100 recover Isabelle symlink for public distribution, notably website;
wenzelm [Tue, 15 Mar 2011 13:03:54 +0100] rev 41984
recover Isabelle symlink for public distribution, notably website;
Mon, 14 Mar 2011 16:59:37 +0100 standardized headers;
wenzelm [Mon, 14 Mar 2011 16:59:37 +0100] rev 41983
standardized headers;
Mon, 14 Mar 2011 15:29:10 +0100 merged
hoelzl [Mon, 14 Mar 2011 15:29:10 +0100] rev 41982
merged
Mon, 14 Mar 2011 14:37:49 +0100 reworked Probability theory: measures are not type restricted to positive extended reals
hoelzl [Mon, 14 Mar 2011 14:37:49 +0100] rev 41981
reworked Probability theory: measures are not type restricted to positive extended reals
Mon, 14 Mar 2011 14:37:47 +0100 split Extended_Reals into parts for Library and Multivariate_Analysis
hoelzl [Mon, 14 Mar 2011 14:37:47 +0100] rev 41980
split Extended_Reals into parts for Library and Multivariate_Analysis
Mon, 14 Mar 2011 14:37:46 +0100 lemmas about addition, SUP on countable sets and infinite sums for extreal
hoelzl [Mon, 14 Mar 2011 14:37:46 +0100] rev 41979
lemmas about addition, SUP on countable sets and infinite sums for extreal
Mon, 14 Mar 2011 14:37:45 +0100 add infinite sums and power on extreal
hoelzl [Mon, 14 Mar 2011 14:37:45 +0100] rev 41978
add infinite sums and power on extreal
Mon, 14 Mar 2011 14:37:44 +0100 introduce setsum on extreal
hoelzl [Mon, 14 Mar 2011 14:37:44 +0100] rev 41977
introduce setsum on extreal
Mon, 14 Mar 2011 14:37:42 +0100 use abs_extreal
hoelzl [Mon, 14 Mar 2011 14:37:42 +0100] rev 41976
use abs_extreal
Mon, 14 Mar 2011 14:37:41 +0100 simplified definition of open_extreal
hoelzl [Mon, 14 Mar 2011 14:37:41 +0100] rev 41975
simplified definition of open_extreal
Mon, 14 Mar 2011 14:37:40 +0100 use case_product for extrel[2,3]_cases
hoelzl [Mon, 14 Mar 2011 14:37:40 +0100] rev 41974
use case_product for extrel[2,3]_cases
Mon, 14 Mar 2011 14:37:39 +0100 add Extended_Reals from AFP/Lower_Semicontinuous
hoelzl [Mon, 14 Mar 2011 14:37:39 +0100] rev 41973
add Extended_Reals from AFP/Lower_Semicontinuous
Mon, 14 Mar 2011 14:37:37 +0100 add lemmas for monotone sequences
hoelzl [Mon, 14 Mar 2011 14:37:37 +0100] rev 41972
add lemmas for monotone sequences
Mon, 14 Mar 2011 14:37:36 +0100 add lemmas for SUP and INF
hoelzl [Mon, 14 Mar 2011 14:37:36 +0100] rev 41971
add lemmas for SUP and INF
Mon, 14 Mar 2011 14:37:35 +0100 generalize infinite sums
hoelzl [Mon, 14 Mar 2011 14:37:35 +0100] rev 41970
generalize infinite sums
Mon, 14 Mar 2011 14:37:33 +0100 moved t2_spaces to HOL image
hoelzl [Mon, 14 Mar 2011 14:37:33 +0100] rev 41969
moved t2_spaces to HOL image
Mon, 14 Mar 2011 15:17:10 +0100 example settings for ISABELLE_GHC, ISABELLE_OCAML, ISABELLE_SWIPL;
wenzelm [Mon, 14 Mar 2011 15:17:10 +0100] rev 41968
example settings for ISABELLE_GHC, ISABELLE_OCAML, ISABELLE_SWIPL;
Mon, 14 Mar 2011 15:13:00 +0100 isatest: fresh copy of settings avoids odd cumulative environment;
wenzelm [Mon, 14 Mar 2011 15:13:00 +0100] rev 41967
isatest: fresh copy of settings avoids odd cumulative environment;
Mon, 14 Mar 2011 12:34:12 +0100 tuned exhaustive_generators
bulwahn [Mon, 14 Mar 2011 12:34:12 +0100] rev 41966
tuned exhaustive_generators
Mon, 14 Mar 2011 12:34:11 +0100 removing definition of cons0; hiding constants in Quickcheck_Narrowing
bulwahn [Mon, 14 Mar 2011 12:34:11 +0100] rev 41965
removing definition of cons0; hiding constants in Quickcheck_Narrowing
Mon, 14 Mar 2011 12:34:10 +0100 tuned subsubsection names in Quickcheck_Narrowing
bulwahn [Mon, 14 Mar 2011 12:34:10 +0100] rev 41964
tuned subsubsection names in Quickcheck_Narrowing
Mon, 14 Mar 2011 12:34:10 +0100 tuned exhaustive generator compilation; added narrowing generator compilation; removed exec as does not work properly here (reverting changeset 994d088fbfbc)
bulwahn [Mon, 14 Mar 2011 12:34:10 +0100] rev 41963
tuned exhaustive generator compilation; added narrowing generator compilation; removed exec as does not work properly here (reverting changeset 994d088fbfbc)
Mon, 14 Mar 2011 12:34:09 +0100 correcting names in Narrowing_Engine and example theory for Quickcheck_Narrowing
bulwahn [Mon, 14 Mar 2011 12:34:09 +0100] rev 41962
correcting names in Narrowing_Engine and example theory for Quickcheck_Narrowing
Mon, 14 Mar 2011 12:34:08 +0100 renaming series and serial to narrowing in Quickcheck_Narrowing
bulwahn [Mon, 14 Mar 2011 12:34:08 +0100] rev 41961
renaming series and serial to narrowing in Quickcheck_Narrowing
Sun, 13 Mar 2011 23:12:38 +0100 eliminated Bali.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 9b19cbb0af28;
wenzelm [Sun, 13 Mar 2011 23:12:38 +0100] rev 41960
eliminated Bali.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 9b19cbb0af28;
Sun, 13 Mar 2011 22:55:50 +0100 tuned headers;
wenzelm [Sun, 13 Mar 2011 22:55:50 +0100] rev 41959
tuned headers;
Sun, 13 Mar 2011 22:24:10 +0100 eliminated hard tabs;
wenzelm [Sun, 13 Mar 2011 22:24:10 +0100] rev 41958
eliminated hard tabs;
Sun, 13 Mar 2011 21:41:44 +0100 less ambitious isatest;
wenzelm [Sun, 13 Mar 2011 21:41:44 +0100] rev 41957
less ambitious isatest;
Sun, 13 Mar 2011 21:21:48 +0100 modernized imports (untested!?);
wenzelm [Sun, 13 Mar 2011 21:21:48 +0100] rev 41956
modernized imports (untested!?);
Sun, 13 Mar 2011 20:56:00 +0100 files are identified via SHA1 digests -- discontinued ISABELLE_FILE_IDENT;
wenzelm [Sun, 13 Mar 2011 20:56:00 +0100] rev 41955
files are identified via SHA1 digests -- discontinued ISABELLE_FILE_IDENT;
Sun, 13 Mar 2011 20:21:24 +0100 explicit type SHA1.digest;
wenzelm [Sun, 13 Mar 2011 20:21:24 +0100] rev 41954
explicit type SHA1.digest;
Sun, 13 Mar 2011 19:27:39 +0100 slightly more robust bash exec, which fails on empty executable;
wenzelm [Sun, 13 Mar 2011 19:27:39 +0100] rev 41953
slightly more robust bash exec, which fails on empty executable;
Sun, 13 Mar 2011 19:16:19 +0100 cleanup of former settings GHC_PATH, EXEC_GHC, EXEC_OCAML, EXEC_SWIPL, EXEC_YAP -- discontinued implicit detection;
wenzelm [Sun, 13 Mar 2011 19:16:19 +0100] rev 41952
cleanup of former settings GHC_PATH, EXEC_GHC, EXEC_OCAML, EXEC_SWIPL, EXEC_YAP -- discontinued implicit detection; determine swipl_version at runtime;
Sun, 13 Mar 2011 17:35:35 +0100 some cleanup of old-style settings;
wenzelm [Sun, 13 Mar 2011 17:35:35 +0100] rev 41951
some cleanup of old-style settings;
Sun, 13 Mar 2011 17:28:14 +0100 clarified ISABELLE_CSDP setting (formerly CSDP_EXE);
wenzelm [Sun, 13 Mar 2011 17:28:14 +0100] rev 41950
clarified ISABELLE_CSDP setting (formerly CSDP_EXE);
Sun, 13 Mar 2011 16:52:59 +0100 more conventional Mutabelle settings -- similar to Mirabelle;
wenzelm [Sun, 13 Mar 2011 16:52:59 +0100] rev 41949
more conventional Mutabelle settings -- similar to Mirabelle;
Sun, 13 Mar 2011 16:38:54 +0100 more basic use of Path.position/File.read;
wenzelm [Sun, 13 Mar 2011 16:38:54 +0100] rev 41948
more basic use of Path.position/File.read;
Sun, 13 Mar 2011 16:38:14 +0100 prefer qualified ISABELLE_NEOS_SERVER;
wenzelm [Sun, 13 Mar 2011 16:38:14 +0100] rev 41947
prefer qualified ISABELLE_NEOS_SERVER;
Sun, 13 Mar 2011 16:30:02 +0100 proper File.shell_path;
wenzelm [Sun, 13 Mar 2011 16:30:02 +0100] rev 41946
proper File.shell_path;
Sun, 13 Mar 2011 16:14:14 +0100 more conventional variable name;
wenzelm [Sun, 13 Mar 2011 16:14:14 +0100] rev 41945
more conventional variable name;
Sun, 13 Mar 2011 16:01:00 +0100 Path.print is the official way to show file-system paths to users -- note that Path.implode often indicates violation of the abstract datatype;
wenzelm [Sun, 13 Mar 2011 16:01:00 +0100] rev 41944
Path.print is the official way to show file-system paths to users -- note that Path.implode often indicates violation of the abstract datatype;
Sun, 13 Mar 2011 15:16:37 +0100 fixed document;
wenzelm [Sun, 13 Mar 2011 15:16:37 +0100] rev 41943
fixed document;
Sun, 13 Mar 2011 15:13:53 +0100 isatest: test more external code;
wenzelm [Sun, 13 Mar 2011 15:13:53 +0100] rev 41942
isatest: test more external code;
Sun, 13 Mar 2011 15:10:00 +0100 tuned headers;
wenzelm [Sun, 13 Mar 2011 15:10:00 +0100] rev 41941
tuned headers;
Sun, 13 Mar 2011 14:51:38 +0100 allow spaces in executable names;
wenzelm [Sun, 13 Mar 2011 14:51:38 +0100] rev 41940
allow spaces in executable names; simplified generated bash scripts;
Sun, 13 Mar 2011 13:57:20 +0100 tuned;
wenzelm [Sun, 13 Mar 2011 13:57:20 +0100] rev 41939
tuned;
Sun, 13 Mar 2011 13:53:54 +0100 tuned headers;
wenzelm [Sun, 13 Mar 2011 13:53:54 +0100] rev 41938
tuned headers;
Fri, 11 Mar 2011 15:21:13 +0100 adapting example file to renaming of the quickcheck tester
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41937
adapting example file to renaming of the quickcheck tester
Fri, 11 Mar 2011 15:21:13 +0100 renaming tester from lazy_exhaustive to narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41936
renaming tester from lazy_exhaustive to narrowing
Fri, 11 Mar 2011 15:21:13 +0100 minor corrections for renaming; moved postprocessing of terms to Quickcheck_Common
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41935
minor corrections for renaming; moved postprocessing of terms to Quickcheck_Common
Fri, 11 Mar 2011 15:21:13 +0100 renaming example file correctly
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41934
renaming example file correctly
Fri, 11 Mar 2011 15:21:13 +0100 adapting Main file generation for Quickcheck_Narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41933
adapting Main file generation for Quickcheck_Narrowing
Fri, 11 Mar 2011 15:21:13 +0100 adapting Quickcheck_Narrowing and example file to new names
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41932
adapting Quickcheck_Narrowing and example file to new names
Fri, 11 Mar 2011 15:21:13 +0100 renaming LSC_Examples theory to Quickcheck_Narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41931
renaming LSC_Examples theory to Quickcheck_Narrowing
Fri, 11 Mar 2011 15:21:13 +0100 renaming lazysmallcheck ML file to Quickcheck_Narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41930
renaming lazysmallcheck ML file to Quickcheck_Narrowing
Fri, 11 Mar 2011 15:21:13 +0100 renaming LSC to Quickcheck_Narrowing
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41929
renaming LSC to Quickcheck_Narrowing
Fri, 11 Mar 2011 15:21:13 +0100 adaptions in generators using the common functions
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41928
adaptions in generators using the common functions
Fri, 11 Mar 2011 15:21:13 +0100 adding file quickcheck_common to carry common functions of all quickcheck generators
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41927
adding file quickcheck_common to carry common functions of all quickcheck generators
Fri, 11 Mar 2011 15:21:13 +0100 adapting record package to renaming of quickcheck's structures
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41926
adapting record package to renaming of quickcheck's structures
Fri, 11 Mar 2011 15:21:13 +0100 moving and renaming lazysmallcheck to narrowing which reflects the characteristical behaviour better
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41925
moving and renaming lazysmallcheck to narrowing which reflects the characteristical behaviour better
Fri, 11 Mar 2011 15:21:13 +0100 correcting dependencies in IsaMakefile
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41924
correcting dependencies in IsaMakefile
Fri, 11 Mar 2011 15:21:13 +0100 renaming signatures and structures; correcting header
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41923
renaming signatures and structures; correcting header
Fri, 11 Mar 2011 15:21:13 +0100 adapting Quickcheck theory after moving ML files
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41922
adapting Quickcheck theory after moving ML files
Fri, 11 Mar 2011 15:21:13 +0100 moving quickcheck_generators.ML to Quickcheck directory and renaming it random_generators.ML
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41921
moving quickcheck_generators.ML to Quickcheck directory and renaming it random_generators.ML
Fri, 11 Mar 2011 15:21:13 +0100 moving exhaustive_generators.ML to Quickcheck directory
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41920
moving exhaustive_generators.ML to Quickcheck directory
Fri, 11 Mar 2011 15:21:13 +0100 correcting dependencies after renaming
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41919
correcting dependencies after renaming
Fri, 11 Mar 2011 15:21:13 +0100 replacing naming of small by exhaustive
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41918
replacing naming of small by exhaustive
Fri, 11 Mar 2011 15:21:13 +0100 renaming smallvalue_generators.ML to exhaustive_generators.ML
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41917
renaming smallvalue_generators.ML to exhaustive_generators.ML
Fri, 11 Mar 2011 15:21:13 +0100 renaming constants in Quickcheck_Exhaustive theory
bulwahn [Fri, 11 Mar 2011 15:21:13 +0100] rev 41916
renaming constants in Quickcheck_Exhaustive theory
Fri, 11 Mar 2011 15:21:12 +0100 renaming Smallcheck to Quickcheck_Exhaustive
bulwahn [Fri, 11 Mar 2011 15:21:12 +0100] rev 41915
renaming Smallcheck to Quickcheck_Exhaustive
Fri, 11 Mar 2011 10:37:45 +0100 only testing theory LSC_Examples when GHC is installed on the machine
bulwahn [Fri, 11 Mar 2011 10:37:45 +0100] rev 41914
only testing theory LSC_Examples when GHC is installed on the machine
Fri, 11 Mar 2011 10:37:43 +0100 increasing timeout of example for counterexample generation
bulwahn [Fri, 11 Mar 2011 10:37:43 +0100] rev 41913
increasing timeout of example for counterexample generation
Fri, 11 Mar 2011 10:37:42 +0100 adding termination proofs to series functions in LSC; commenting out momentarily unused term refinement functions in LSC
bulwahn [Fri, 11 Mar 2011 10:37:42 +0100] rev 41912
adding termination proofs to series functions in LSC; commenting out momentarily unused term refinement functions in LSC
Fri, 11 Mar 2011 10:37:41 +0100 adding lazysmallcheck example theory to HOL-ex session
bulwahn [Fri, 11 Mar 2011 10:37:41 +0100] rev 41911
adding lazysmallcheck example theory to HOL-ex session
Fri, 11 Mar 2011 10:37:40 +0100 adding serial instance of finite_4 in lazysmallcheck; changing code equations for implies
bulwahn [Fri, 11 Mar 2011 10:37:40 +0100] rev 41910
adding serial instance of finite_4 in lazysmallcheck; changing code equations for implies
Fri, 11 Mar 2011 10:37:38 +0100 replacing strings in generated Code resolves the changing names of Typerep in lazysmallcheck prototype
bulwahn [Fri, 11 Mar 2011 10:37:38 +0100] rev 41909
replacing strings in generated Code resolves the changing names of Typerep in lazysmallcheck prototype
Fri, 11 Mar 2011 10:37:37 +0100 changing invocation of ghc from interactive mode to compilation increases the performance of lazysmallcheck by a factor of twenty; changing Integer type to Int reduces by another 50 percent
bulwahn [Fri, 11 Mar 2011 10:37:37 +0100] rev 41908
changing invocation of ghc from interactive mode to compilation increases the performance of lazysmallcheck by a factor of twenty; changing Integer type to Int reduces by another 50 percent
Fri, 11 Mar 2011 10:37:37 +0100 adding an example theory for Lazysmallcheck prototype
bulwahn [Fri, 11 Mar 2011 10:37:37 +0100] rev 41907
adding an example theory for Lazysmallcheck prototype
Fri, 11 Mar 2011 10:37:36 +0100 adding Lazysmallcheck prototype to HOL-Library
bulwahn [Fri, 11 Mar 2011 10:37:36 +0100] rev 41906
adding Lazysmallcheck prototype to HOL-Library
Fri, 11 Mar 2011 10:37:35 +0100 adding files for prototype of lazysmallcheck
bulwahn [Fri, 11 Mar 2011 10:37:35 +0100] rev 41905
adding files for prototype of lazysmallcheck
Fri, 11 Mar 2011 08:58:29 +0100 removing debug message in quickcheck's postprocessor
bulwahn [Fri, 11 Mar 2011 08:58:29 +0100] rev 41904
removing debug message in quickcheck's postprocessor
Fri, 11 Mar 2011 08:13:00 +0100 fixing postprocessing; adding a configuration to enable and disable pretty presentation of quickcheck's counterexample
bulwahn [Fri, 11 Mar 2011 08:13:00 +0100] rev 41903
fixing postprocessing; adding a configuration to enable and disable pretty presentation of quickcheck's counterexample
Fri, 11 Mar 2011 08:12:59 +0100 renaming dest_plain_fun to dest_fun_upds and adding handling of undefined for postprocessing of quickcheck
bulwahn [Fri, 11 Mar 2011 08:12:59 +0100] rev 41902
renaming dest_plain_fun to dest_fun_upds and adding handling of undefined for postprocessing of quickcheck
Fri, 11 Mar 2011 08:12:58 +0100 improving term postprocessing for counterexample presentation in quickcheck
bulwahn [Fri, 11 Mar 2011 08:12:58 +0100] rev 41901
improving term postprocessing for counterexample presentation in quickcheck
Fri, 11 Mar 2011 08:12:55 +0100 tuned
bulwahn [Fri, 11 Mar 2011 08:12:55 +0100] rev 41900
tuned
Wed, 09 Mar 2011 21:40:38 +0100 finished and tested Z3 proof reconstruction for injective functions;
boehmes [Wed, 09 Mar 2011 21:40:38 +0100] rev 41899
finished and tested Z3 proof reconstruction for injective functions; only treat variables as atomic, and especially abstract constants (Isabelle's interpretation of these constants is most likely not known to Z3 and thus irrelevant for the proof)
Wed, 09 Mar 2011 10:28:01 +0100 improved formula for specialization, to prevent needless specializations -- and removed dead code
blanchet [Wed, 09 Mar 2011 10:28:01 +0100] rev 41898
improved formula for specialization, to prevent needless specializations -- and removed dead code
Wed, 09 Mar 2011 10:25:29 +0100 perform no arity check in debug mode so that we get to see the Kodkod problem
blanchet [Wed, 09 Mar 2011 10:25:29 +0100] rev 41897
perform no arity check in debug mode so that we get to see the Kodkod problem
Fri, 04 Mar 2011 17:39:30 +0100 spark_end now joins proofs of VCs before writing *.prv file.
berghofe [Fri, 04 Mar 2011 17:39:30 +0100] rev 41896
spark_end now joins proofs of VCs before writing *.prv file.
Fri, 04 Mar 2011 11:43:20 +0100 clarified
krauss [Fri, 04 Mar 2011 11:43:20 +0100] rev 41895
clarified
Fri, 04 Mar 2011 11:52:54 +0100 produce helpful mira summary for more errors
krauss [Fri, 04 Mar 2011 11:52:54 +0100] rev 41894
produce helpful mira summary for more errors
Fri, 04 Mar 2011 00:09:47 +0100 eliminated prems;
wenzelm [Fri, 04 Mar 2011 00:09:47 +0100] rev 41893
eliminated prems;
Thu, 03 Mar 2011 22:06:15 +0100 eliminated UNITY_Examples.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 3dec57ec3473;
wenzelm [Thu, 03 Mar 2011 22:06:15 +0100] rev 41892
eliminated UNITY_Examples.thy which takes quite long to merge and does not parallelize so well -- essentially reverting 3dec57ec3473;
Thu, 03 Mar 2011 21:43:06 +0100 tuned proofs -- eliminated prems;
wenzelm [Thu, 03 Mar 2011 21:43:06 +0100] rev 41891
tuned proofs -- eliminated prems;
Thu, 03 Mar 2011 18:43:15 +0100 merged
wenzelm [Thu, 03 Mar 2011 18:43:15 +0100] rev 41890
merged
Thu, 03 Mar 2011 14:38:31 +0100 merged
blanchet [Thu, 03 Mar 2011 14:38:31 +0100] rev 41889
merged
Thu, 03 Mar 2011 14:25:15 +0100 don't forget to look for constants appearing only in "need" option -- otherwise we get exceptions in "the_name" later on
blanchet [Thu, 03 Mar 2011 14:25:15 +0100] rev 41888
don't forget to look for constants appearing only in "need" option -- otherwise we get exceptions in "the_name" later on
Thu, 03 Mar 2011 18:42:12 +0100 simplified Thy_Info.check_file -- discontinued load path;
wenzelm [Thu, 03 Mar 2011 18:42:12 +0100] rev 41887
simplified Thy_Info.check_file -- discontinued load path;
Thu, 03 Mar 2011 18:10:28 +0100 discontinued legacy load path;
wenzelm [Thu, 03 Mar 2011 18:10:28 +0100] rev 41886
discontinued legacy load path;
Thu, 03 Mar 2011 15:56:17 +0100 re-interpret ProofGeneralPgip.changecwd as Thy_Load.set_master_path, presuming that this is close to the intended semantics;
wenzelm [Thu, 03 Mar 2011 15:56:17 +0100] rev 41885
re-interpret ProofGeneralPgip.changecwd as Thy_Load.set_master_path, presuming that this is close to the intended semantics;
Thu, 03 Mar 2011 15:46:02 +0100 modernized imports;
wenzelm [Thu, 03 Mar 2011 15:46:02 +0100] rev 41884
modernized imports;
Thu, 03 Mar 2011 15:36:54 +0100 observe standard header format;
wenzelm [Thu, 03 Mar 2011 15:36:54 +0100] rev 41883
observe standard header format;
Thu, 03 Mar 2011 15:19:20 +0100 removed spurious 'unused_thms' (cf. 1a65b780bd56);
wenzelm [Thu, 03 Mar 2011 15:19:20 +0100] rev 41882
removed spurious 'unused_thms' (cf. 1a65b780bd56);
Thu, 03 Mar 2011 15:18:05 +0100 isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
wenzelm [Thu, 03 Mar 2011 15:18:05 +0100] rev 41881
isatest cygwin-poly-e: new memory management of polyml-svn could be more stable;
Thu, 03 Mar 2011 11:36:10 +0100 merged
berghofe [Thu, 03 Mar 2011 11:36:10 +0100] rev 41880
merged
Thu, 03 Mar 2011 11:15:50 +0100 merged
berghofe [Thu, 03 Mar 2011 11:15:50 +0100] rev 41879
merged
Thu, 03 Mar 2011 11:01:42 +0100 - Made sure that sort_defs is aware of constants introduced by add_type_def
berghofe [Thu, 03 Mar 2011 11:01:42 +0100] rev 41878
- Made sure that sort_defs is aware of constants introduced by add_type_def - add_def now compares Isabelle types rather than SPARK types to ensure that type abbreviations are taken into account
Thu, 03 Mar 2011 11:20:48 +0100 mention new Nitpick options
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41877
mention new Nitpick options
Thu, 03 Mar 2011 11:20:48 +0100 simplify "need" option's syntax
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41876
simplify "need" option's syntax
Thu, 03 Mar 2011 11:20:48 +0100 renamed "preconstr" option "need"
blanchet [Thu, 03 Mar 2011 11:20:48 +0100] rev 41875
renamed "preconstr" option "need"
Thu, 03 Mar 2011 10:55:41 +0100 finally remove upper_bound_finite_set
hoelzl [Thu, 03 Mar 2011 10:55:41 +0100] rev 41874
finally remove upper_bound_finite_set
Thu, 03 Mar 2011 15:59:44 +1100 separate settings for afp test
kleing [Thu, 03 Mar 2011 15:59:44 +1100] rev 41873
separate settings for afp test
Wed, 02 Mar 2011 15:51:22 +0100 added missing spaces in output
blanchet [Wed, 02 Mar 2011 15:51:22 +0100] rev 41872
added missing spaces in output
Wed, 02 Mar 2011 14:50:16 +0100 lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
blanchet [Wed, 02 Mar 2011 14:50:16 +0100] rev 41871
lower threshold for implicitly using "nitpick_simp" for predicate definitions when "total_consts" is on
Wed, 02 Mar 2011 13:09:57 +0100 unfold definitions in "preconstrs" option
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41870
unfold definitions in "preconstrs" option
Wed, 02 Mar 2011 13:09:57 +0100 robust handling of types occurring in "eval" and "preconstr" options but not in the goal
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41869
robust handling of types occurring in "eval" and "preconstr" options but not in the goal
Wed, 02 Mar 2011 13:09:57 +0100 make "preconstr" option more robust -- shouldn't throw exceptions
blanchet [Wed, 02 Mar 2011 13:09:57 +0100] rev 41868
make "preconstr" option more robust -- shouldn't throw exceptions
Tue, 01 Mar 2011 10:40:14 +0000 merged
paulson [Tue, 01 Mar 2011 10:40:14 +0000] rev 41867
merged
Mon, 28 Feb 2011 15:06:55 +0000 merged
paulson [Mon, 28 Feb 2011 15:06:55 +0000] rev 41866
merged
Mon, 28 Feb 2011 15:06:36 +0000 declare ext [intro]: Extensionality now available by default
paulson [Mon, 28 Feb 2011 15:06:36 +0000] rev 41865
declare ext [intro]: Extensionality now available by default
Mon, 28 Feb 2011 22:12:09 +0100 merged
boehmes [Mon, 28 Feb 2011 22:12:09 +0100] rev 41864
merged
Mon, 28 Feb 2011 22:10:57 +0100 removed dependency on Dense_Linear_Order
boehmes [Mon, 28 Feb 2011 22:10:57 +0100] rev 41863
removed dependency on Dense_Linear_Order
Mon, 28 Feb 2011 19:06:24 +0100 adding function Quickcheck.test_terms to provide checking a batch of terms
bulwahn [Mon, 28 Feb 2011 19:06:24 +0100] rev 41862
adding function Quickcheck.test_terms to provide checking a batch of terms
Mon, 28 Feb 2011 19:06:23 +0100 adding a function to compile a batch of terms for quickcheck with one code generation invocation
bulwahn [Mon, 28 Feb 2011 19:06:23 +0100] rev 41861
adding a function to compile a batch of terms for quickcheck with one code generation invocation
Mon, 28 Feb 2011 17:53:10 +0100 improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41860
improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
Mon, 28 Feb 2011 17:53:10 +0100 made "fixed_is_special_eligible_arg" smarter w.r.t. pairs, and fixed previous unintended behavior because "andalso" ties more tightly than "orelse"
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41859
made "fixed_is_special_eligible_arg" smarter w.r.t. pairs, and fixed previous unintended behavior because "andalso" ties more tightly than "orelse"
Mon, 28 Feb 2011 17:53:10 +0100 if "total_consts" is set, report cex's as quasi-genuine
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41858
if "total_consts" is set, report cex's as quasi-genuine
Mon, 28 Feb 2011 17:53:10 +0100 document new "total_consts" option
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41857
document new "total_consts" option
Mon, 28 Feb 2011 17:53:10 +0100 added "total_consts" option
blanchet [Mon, 28 Feb 2011 17:53:10 +0100] rev 41856
added "total_consts" option
Sat, 26 Feb 2011 20:40:45 +0100 added a few lemmas by Andreas Lochbihler
nipkow [Sat, 26 Feb 2011 20:40:45 +0100] rev 41855
added a few lemmas by Andreas Lochbihler
Sat, 26 Feb 2011 20:16:44 +0100 Corrected HOLCF/FOCUS dependency
nipkow [Sat, 26 Feb 2011 20:16:44 +0100] rev 41854
Corrected HOLCF/FOCUS dependency
Sat, 26 Feb 2011 17:44:42 +0100 Added material by David Trachtenherz
nipkow [Sat, 26 Feb 2011 17:44:42 +0100] rev 41853
Added material by David Trachtenherz
Sat, 26 Feb 2011 16:16:36 +0100 corrected HOLCF dependency on Nat_Infinity
nipkow [Sat, 26 Feb 2011 16:16:36 +0100] rev 41852
corrected HOLCF dependency on Nat_Infinity
Fri, 25 Feb 2011 22:07:56 +0100 got rid of lemma upper_bound_finite_set
nipkow [Fri, 25 Feb 2011 22:07:56 +0100] rev 41851
got rid of lemma upper_bound_finite_set
Fri, 25 Feb 2011 20:08:00 +0100 merged
nipkow [Fri, 25 Feb 2011 20:08:00 +0100] rev 41850
merged
Fri, 25 Feb 2011 20:07:48 +0100 Some cleaning up
nipkow [Fri, 25 Feb 2011 20:07:48 +0100] rev 41849
Some cleaning up
Fri, 25 Feb 2011 17:11:24 +0100 updated generated files
krauss [Fri, 25 Feb 2011 17:11:24 +0100] rev 41848
updated generated files
Fri, 25 Feb 2011 17:11:05 +0100 fixed manual (rule no longer exists)
krauss [Fri, 25 Feb 2011 17:11:05 +0100] rev 41847
fixed manual (rule no longer exists)
(0) -30000 -10000 -3000 -1000 -240 +240 +1000 +3000 +10000 +30000 tip