Sun, 20 Mar 2011 22:26:43 +0100 |
wenzelm |
NEWS: structure Timing provides various operations for timing;
|
file |
diff |
annotate
|
Fri, 18 Mar 2011 22:55:28 +0100 |
blanchet |
added "simp:", "intro:", and "elim:" to "try" command
|
file |
diff |
annotate
|
Thu, 17 Mar 2011 22:07:17 +0100 |
blanchet |
reintroduced "show_skolems" option -- useful when too many Skolems are displayed
|
file |
diff |
annotate
|
Sun, 13 Mar 2011 20:56:00 +0100 |
wenzelm |
files are identified via SHA1 digests -- discontinued ISABELLE_FILE_IDENT;
|
file |
diff |
annotate
|
Sun, 13 Mar 2011 19:16:19 +0100 |
wenzelm |
cleanup of former settings GHC_PATH, EXEC_GHC, EXEC_OCAML, EXEC_SWIPL, EXEC_YAP -- discontinued implicit detection;
|
file |
diff |
annotate
|
Sun, 13 Mar 2011 17:28:14 +0100 |
wenzelm |
clarified ISABELLE_CSDP setting (formerly CSDP_EXE);
|
file |
diff |
annotate
|
Sun, 13 Mar 2011 16:01:00 +0100 |
wenzelm |
Path.print is the official way to show file-system paths to users -- note that Path.implode often indicates violation of the abstract datatype;
|
file |
diff |
annotate
|
Thu, 03 Mar 2011 18:10:28 +0100 |
wenzelm |
discontinued legacy load path;
|
file |
diff |
annotate
|
Thu, 03 Mar 2011 11:20:48 +0100 |
blanchet |
mention new Nitpick options
|
file |
diff |
annotate
|
Fri, 25 Feb 2011 16:59:48 +0100 |
krauss |
removed support for tail-recursion from function package (now implemented by partial_function)
|
file |
diff |
annotate
|
Mon, 21 Feb 2011 10:44:19 +0100 |
blanchet |
renamed "nitpick\_def" to "nitpick_unfold" to reflect its new semantics
|
file |
diff |
annotate
|
Tue, 08 Feb 2011 21:12:27 +0100 |
wenzelm |
discontinued obsolete lib/scripts/polyml-platform;
|
file |
diff |
annotate
|
Tue, 08 Feb 2011 17:38:43 +0100 |
wenzelm |
merged
|
file |
diff |
annotate
|
Tue, 08 Feb 2011 16:10:10 +0100 |
blanchet |
available_provers ~> supported_provers (for clarity)
|
file |
diff |
annotate
|
Tue, 08 Feb 2011 17:36:21 +0100 |
wenzelm |
discontinued support for Poly/ML 5.2, which was the last version without proper multithreading and TimeLimit implementation;
|
file |
diff |
annotate
|
Fri, 04 Feb 2011 17:11:00 +0100 |
wenzelm |
parallelization of nested Isar proofs is subject to Goal.parallel_proofs_threshold;
|
file |
diff |
annotate
|
Tue, 01 Feb 2011 21:09:52 +0100 |
krauss |
term style 'isub': ad-hoc subscripting of variables that end with digits (x1, x23, ...)
|
file |
diff |
annotate
|
Mon, 31 Jan 2011 11:18:29 +0100 |
wenzelm |
merged
|
file |
diff |
annotate
|
Mon, 17 Jan 2011 20:20:51 +0100 |
wenzelm |
back to post-release mode;
|
file |
diff |
annotate
|
Wed, 19 Jan 2011 11:27:56 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Mon, 17 Jan 2011 18:32:16 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Mon, 17 Jan 2011 17:45:52 +0100 |
boehmes |
made Z3 the default SMT solver again
|
file |
diff |
annotate
|
Sun, 16 Jan 2011 21:10:30 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Sun, 16 Jan 2011 20:55:48 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Sun, 16 Jan 2011 20:54:30 +0100 |
wenzelm |
misc tuning for release;
|
file |
diff |
annotate
|
Sat, 15 Jan 2011 14:56:57 +0100 |
wenzelm |
global "prems" is legacy feature;
|
file |
diff |
annotate
|
Sat, 15 Jan 2011 14:19:37 +0100 |
wenzelm |
misc updates for release;
|
file |
diff |
annotate
|
Sat, 15 Jan 2011 14:02:24 +0100 |
wenzelm |
merged;
|
file |
diff |
annotate
|
Sat, 15 Jan 2011 13:34:10 +0100 |
wenzelm |
misc tuning for release;
|
file |
diff |
annotate
|
Sat, 15 Jan 2011 12:49:10 +0100 |
berghofe |
Added entry for HOL-SPARK
|
file |
diff |
annotate
|
Tue, 11 Jan 2011 20:01:57 +0100 |
wenzelm |
updated to Isabelle2011;
|
file |
diff |
annotate
|
Tue, 11 Jan 2011 18:23:29 +0100 |
haftmann |
NEWS
|
file |
diff |
annotate
|
Tue, 11 Jan 2011 17:59:35 +0100 |
bulwahn |
NEWS
|
file |
diff |
annotate
|
Fri, 07 Jan 2011 10:28:45 +0100 |
krauss |
tuned NEWS
|
file |
diff |
annotate
|
Thu, 06 Jan 2011 21:06:18 +0100 |
ballarin |
Diagnostic command to show locale dependencies.
|
file |
diff |
annotate
|
Thu, 06 Jan 2011 21:06:17 +0100 |
ballarin |
Documentation for 'interpret' and 'sublocale' with mixins.
|
file |
diff |
annotate
|
Thu, 06 Jan 2011 21:06:17 +0100 |
ballarin |
Abelian group facts obtained from group facts via interpretation (sublocale).
|
file |
diff |
annotate
|
Thu, 06 Jan 2011 17:51:56 +0100 |
boehmes |
differentiate between local and remote SMT solvers (e.g., "z3" vs. "remote_z3");
|
file |
diff |
annotate
|
Tue, 04 Jan 2011 15:32:56 -0800 |
huffman |
change some lemma names containing 'UU' to 'bottom'
|
file |
diff |
annotate
|
Tue, 04 Jan 2011 15:03:27 -0800 |
huffman |
renamed constant 'UU' to 'bottom', keeping 'UU' as alternative input syntax;
|
file |
diff |
annotate
|
Wed, 29 Dec 2010 18:18:42 +0100 |
wenzelm |
theory loader: implicit load path is considered legacy;
|
file |
diff |
annotate
|
Thu, 23 Dec 2010 13:11:40 -0800 |
huffman |
NEWS updates for HOLCF
|
file |
diff |
annotate
|
Thu, 23 Dec 2010 12:20:09 +0100 |
haftmann |
tuned order of NEWS
|
file |
diff |
annotate
|
Thu, 23 Dec 2010 12:04:29 +0100 |
haftmann |
NEWS
|
file |
diff |
annotate
|
Tue, 21 Dec 2010 21:54:51 +0100 |
wenzelm |
configuration option "rule_trace";
|
file |
diff |
annotate
|
Tue, 21 Dec 2010 21:21:21 +0100 |
wenzelm |
configuration option "syntax_ast_trace" and "syntax_ast_stat";
|
file |
diff |
annotate
|
Mon, 20 Dec 2010 16:44:33 +0100 |
wenzelm |
proper identifiers for consts and types;
|
file |
diff |
annotate
|
Sun, 19 Dec 2010 18:38:50 -0800 |
huffman |
rename function cprod_map to prod_map
|
file |
diff |
annotate
|
Sun, 19 Dec 2010 18:10:54 -0800 |
huffman |
fix typo
|
file |
diff |
annotate
|
Sun, 19 Dec 2010 06:34:41 -0800 |
huffman |
type 'defl' takes a type parameter again (cf. b525988432e9)
|
file |
diff |
annotate
|
Sun, 19 Dec 2010 05:15:31 -0800 |
huffman |
reintroduce 'bifinite' class, now with existentially-quantified approx function (cf. b525988432e9)
|
file |
diff |
annotate
|
Fri, 17 Dec 2010 18:10:37 +0100 |
wenzelm |
Command 'type_synonym' (with single argument) supersedes 'types' (legacy feature);
|
file |
diff |
annotate
|
Fri, 17 Dec 2010 17:43:54 +0100 |
wenzelm |
replaced command 'nonterminals' by slightly modernized version 'nonterminal';
|
file |
diff |
annotate
|
Fri, 17 Dec 2010 17:08:56 +0100 |
wenzelm |
renamed structure MetaSimplifier to raw_Simplifer, to emphasize its meaning;
|
file |
diff |
annotate
|
Wed, 08 Dec 2010 14:52:23 +0100 |
haftmann |
NEWS
|
file |
diff |
annotate
|
Mon, 06 Dec 2010 13:43:05 -0800 |
huffman |
merged
|
file |
diff |
annotate
|
Mon, 06 Dec 2010 11:22:42 -0800 |
huffman |
remove lemma cont_cfun;
|
file |
diff |
annotate
|
Mon, 06 Dec 2010 10:08:33 -0800 |
huffman |
rename lub_fun -> is_lub_fun, thelub_fun -> lub_fun
|
file |
diff |
annotate
|
Fri, 03 Dec 2010 15:25:14 +0100 |
hoelzl |
it is known as the extended reals, not the infinite reals
|
file |
diff |
annotate
|
Mon, 06 Dec 2010 16:37:15 +0100 |
wenzelm |
more correct NEWS;
|
file |
diff |
annotate
|
Sun, 05 Dec 2010 15:23:33 +0100 |
wenzelm |
IsabelleText font: include Cyrillic, Hebrew, Arabic from DejaVu Sans 2.32;
|
file |
diff |
annotate
|
Sun, 05 Dec 2010 14:02:16 +0100 |
wenzelm |
command 'notepad' replaces former 'example_proof';
|
file |
diff |
annotate
|
Sat, 04 Dec 2010 18:41:12 +0100 |
wenzelm |
added Syntax.default_root;
|
file |
diff |
annotate
|
Sat, 04 Dec 2010 14:57:04 +0100 |
wenzelm |
added Syntax.pretty_priority;
|
file |
diff |
annotate
|
Fri, 03 Dec 2010 22:08:14 +0100 |
wenzelm |
minor tuning for release;
|
file |
diff |
annotate
|
Fri, 03 Dec 2010 21:34:54 +0100 |
wenzelm |
source files are always encoded as UTF-8;
|
file |
diff |
annotate
|
Fri, 03 Dec 2010 17:59:13 +0100 |
wenzelm |
setup subtyping/coercions once in HOL.thy, but enable it only later via configuration option;
|
file |
diff |
annotate
|
Fri, 03 Dec 2010 09:58:32 +0100 |
bulwahn |
NEWS
|
file |
diff |
annotate
|
Thu, 02 Dec 2010 16:52:52 +0100 |
wenzelm |
configuration option "show_abbrevs" supersedes print mode "no_abbrevs", with inverted meaning;
|
file |
diff |
annotate
|
Thu, 02 Dec 2010 16:04:22 +0100 |
wenzelm |
renamed trace_simp to simp_trace, and debug_simp to simp_debug;
|
file |
diff |
annotate
|
Thu, 02 Dec 2010 08:34:23 +0100 |
nipkow |
coercions
|
file |
diff |
annotate
|
Wed, 01 Dec 2010 19:33:49 +0100 |
hoelzl |
Updated NEWS
|
file |
diff |
annotate
|
Wed, 01 Dec 2010 11:45:37 +0100 |
haftmann |
NEWS
|
file |
diff |
annotate
|
Tue, 30 Nov 2010 15:58:21 +0100 |
haftmann |
merged
|
file |
diff |
annotate
|
Mon, 29 Nov 2010 13:44:54 +0100 |
haftmann |
equivI has replaced equiv.intro
|
file |
diff |
annotate
|
Mon, 29 Nov 2010 11:22:40 +0100 |
wenzelm |
added document antiquotation @{file};
|
file |
diff |
annotate
|
Sun, 28 Nov 2010 13:58:29 +0100 |
wenzelm |
recovered Isabelle2009-2 NEWS -- published part is read-only;
|
file |
diff |
annotate
|
Sat, 27 Nov 2010 13:12:10 -0800 |
huffman |
renamed several HOLCF theorems (listed in NEWS)
|
file |
diff |
annotate
|
Fri, 26 Nov 2010 23:41:23 +0100 |
wenzelm |
merged
|
file |
diff |
annotate
|
Fri, 26 Nov 2010 22:36:55 +0100 |
blanchet |
document changes in Nitpick and MESON/Metis
|
file |
diff |
annotate
|
Fri, 26 Nov 2010 22:29:41 +0100 |
wenzelm |
make two copies (!) of Library.UnequalLengths coincide with ListPair.UnequalLengths;
|
file |
diff |
annotate
|
Fri, 26 Nov 2010 14:19:16 +0100 |
wenzelm |
more correct spelling;
|
file |
diff |
annotate
|
Fri, 26 Nov 2010 12:03:17 +0100 |
haftmann |
globbing constant expressions use more idiomatic underscore rather than star;
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 10:34:33 +0100 |
hoelzl |
Replace surj by abbreviation; remove surj_on.
|
file |
diff |
annotate
|
Wed, 24 Nov 2010 10:23:52 +0100 |
bulwahn |
announcing some latest change (d40b347d5b0b)
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 17:49:12 +0100 |
haftmann |
merged
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 17:46:51 +0100 |
haftmann |
replaced misleading Fset/fset name -- these do not stand for finite sets
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 10:41:56 +0100 |
bulwahn |
renaming quickcheck generator code to random
|
file |
diff |
annotate
|
Sat, 20 Nov 2010 00:53:26 +0100 |
wenzelm |
renamed raw "explode" function to "raw_explode" to emphasize its meaning;
|
file |
diff |
annotate
|
Fri, 19 Nov 2010 09:07:23 -0800 |
huffman |
merged
|
file |
diff |
annotate
|
Wed, 17 Nov 2010 12:19:19 -0800 |
huffman |
accumulated NEWS updates for HOLCF
|
file |
diff |
annotate
|
Thu, 18 Nov 2010 18:12:03 +0100 |
blanchet |
mention Sledgehammer with SMT
|
file |
diff |
annotate
|
Wed, 17 Nov 2010 09:22:23 +0100 |
boehmes |
require the b2i file ending in the boogie_open command (for consistency with the theory header)
|
file |
diff |
annotate
|
Mon, 08 Nov 2010 12:13:44 +0100 |
boehmes |
better modularization: moved SMT configuration options and diagnostics as well as SMT failure and exception into separate structures (both of which are loaded first and consequently are available to other SMT structures)
|
file |
diff |
annotate
|
Sat, 06 Nov 2010 00:10:32 +0100 |
krauss |
abolished obscure goal variant of [split_format] -- unused (cf. d1c14898fd04), unrelated to '(complete)' variant, and not at all canonical
|
file |
diff |
annotate
|
Fri, 05 Nov 2010 23:19:20 +0100 |
wenzelm |
moved ISABELLE_IDENTIFIER from ISABELLE_OUTPUT further up to ISABELLE_HOME_USER;
|
file |
diff |
annotate
|
Thu, 04 Nov 2010 09:54:16 +0100 |
haftmann |
merged
|
file |
diff |
annotate
|
Wed, 03 Nov 2010 12:20:33 +0100 |
haftmann |
Theory Multiset provides stable quicksort implementation of sort_key.
|
file |
diff |
annotate
|
Wed, 03 Nov 2010 22:26:53 +0100 |
blanchet |
standardize on seconds for Nitpick and Sledgehammer timeouts
|
file |
diff |
annotate
|
Wed, 03 Nov 2010 11:33:51 +0100 |
wenzelm |
discontinued obsolete function sys_error and exception SYS_ERROR;
|
file |
diff |
annotate
|
Sun, 31 Oct 2010 11:45:45 +0100 |
nipkow |
merged
|
file |
diff |
annotate
|
Fri, 29 Oct 2010 17:57:36 +0200 |
nipkow |
Plus -> Sum_Type.Plus
|
file |
diff |
annotate
|
Sat, 30 Oct 2010 21:08:20 +0200 |
wenzelm |
support for real valued preferences;
|
file |
diff |
annotate
|
Sat, 30 Oct 2010 16:33:58 +0200 |
wenzelm |
support for real valued configuration options;
|
file |
diff |
annotate
|
Fri, 29 Oct 2010 11:07:21 +0200 |
wenzelm |
merged
|
file |
diff |
annotate
|
Fri, 29 Oct 2010 08:44:46 +0200 |
bulwahn |
NEWS
|
file |
diff |
annotate
|
Thu, 28 Oct 2010 23:19:52 +0200 |
wenzelm |
discontinued obsolete ML antiquotation @{theory_ref};
|
file |
diff |
annotate
|
Tue, 26 Oct 2010 15:06:36 +0200 |
krauss |
fixed typo
|
file |
diff |
annotate
|
Tue, 26 Oct 2010 13:50:18 +0200 |
krauss |
NEWS
|
file |
diff |
annotate
|
Tue, 26 Oct 2010 11:45:12 +0200 |
boehmes |
joined setup of SMT solvers in one place; turned Z3-specific options into SMT options (renamed configuration options from z3_* to smt_*); more detailed SMT exception; improved SMT filter interface
|
file |
diff |
annotate
|
Mon, 25 Oct 2010 16:18:00 +0200 |
wenzelm |
merged
|
file |
diff |
annotate
|
Mon, 25 Oct 2010 16:17:16 +0200 |
wenzelm |
significantly improved Isabelle/Isar implementation manual;
|
file |
diff |
annotate
|
Mon, 25 Oct 2010 11:42:05 +0200 |
blanchet |
merged
|
file |
diff |
annotate
|
Mon, 25 Oct 2010 10:30:46 +0200 |
blanchet |
introduced manual version of "Auto Solve" as "solve_direct"
|
file |
diff |
annotate
|
Mon, 25 Oct 2010 11:16:23 +0200 |
wenzelm |
added ML antiquotation @{assert};
|
file |
diff |
annotate
|
Sun, 24 Oct 2010 20:37:30 +0200 |
nipkow |
renamed nat_number
|
file |
diff |
annotate
|
Fri, 22 Oct 2010 11:11:34 +0200 |
blanchet |
make Sledgehammer minimizer fully work with SMT
|
file |
diff |
annotate
|
Thu, 21 Oct 2010 14:55:09 +0200 |
blanchet |
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
|
file |
diff |
annotate
|
Thu, 14 Oct 2010 12:40:14 +0200 |
krauss |
NEWS
|
file |
diff |
annotate
|
Wed, 06 Oct 2010 17:44:21 +0200 |
blanchet |
merged
|
file |
diff |
annotate
|