Thu, 04 Nov 2010 16:15:13 +0100 |
wenzelm |
added property "tooltip-margin";
|
changeset |
files
|
Thu, 04 Nov 2010 10:58:03 +0100 |
wenzelm |
clarified tooltips: message output by default, extra info via control/command;
|
changeset |
files
|
Thu, 04 Nov 2010 10:33:37 +0100 |
wenzelm |
warn in correlation with report -- avoid spurious message duplicates;
|
changeset |
files
|
Thu, 04 Nov 2010 10:22:59 +0100 |
wenzelm |
tuned;
|
changeset |
files
|
Wed, 03 Nov 2010 21:53:56 +0100 |
wenzelm |
feeder: treat header as escaped utf8 to allow initial ML text to refer to non-ASCII file/directory names (e.g. "Documents/" on Chinese Ubuntu);
|
changeset |
files
|
Wed, 03 Nov 2010 17:11:40 +0100 |
boehmes |
merged
|
changeset |
files
|
Wed, 03 Nov 2010 17:02:53 +0100 |
boehmes |
updated SMT certificates
|
changeset |
files
|
Wed, 03 Nov 2010 16:44:38 +0100 |
boehmes |
standardize timeout value based on reals
|
changeset |
files
|
Wed, 03 Nov 2010 15:56:15 +0100 |
wenzelm |
merged
|
changeset |
files
|
Wed, 03 Nov 2010 07:02:09 -0700 |
huffman |
merged
|
changeset |
files
|
Sat, 30 Oct 2010 15:13:11 -0700 |
huffman |
change default_sort of HOLCF from pcpo to bifinite; rename command 'new_domain' to 'domain'; rename 'domain' to 'domain (unsafe)'
|
changeset |
files
|
Sat, 30 Oct 2010 12:25:18 -0700 |
huffman |
merged
|
changeset |
files
|
Fri, 29 Oct 2010 17:15:28 -0700 |
huffman |
renamed {Rep,Abs}_CFun to {Rep,Abs}_cfun
|
changeset |
files
|
Fri, 29 Oct 2010 16:51:40 -0700 |
huffman |
renamed lemma cont2cont_Rep_CFun to cont2cont_APP
|
changeset |
files
|
Fri, 29 Oct 2010 16:24:07 -0700 |
huffman |
simplify proof of typedef_cont_Abs
|
changeset |
files
|
Wed, 27 Oct 2010 15:50:01 -0700 |
huffman |
rename constant trifte to tr_case
|
changeset |
files
|
Wed, 27 Oct 2010 14:31:39 -0700 |
huffman |
add 'LAM (Def x). t' as alternative syntax for 'FLIFT x. t'
|
changeset |
files
|
Wed, 27 Oct 2010 14:15:54 -0700 |
huffman |
make syntax of continuous if-then-else consistent with HOL if-then-else
|
changeset |
files
|
Wed, 27 Oct 2010 13:54:18 -0700 |
huffman |
rename lemmas *_defined_iff and *_strict_iff to *_bottom_iff
|
changeset |
files
|
Wed, 03 Nov 2010 10:44:53 +0100 |
haftmann |
polyml_as_definition does not require explicit dependencies on external ML files
|
changeset |
files
|
Wed, 03 Nov 2010 13:54:23 +0100 |
wenzelm |
explicit warning about opaque signature matching -- saves extra paragraph in implementation manual;
|
changeset |
files
|
Wed, 03 Nov 2010 11:33:51 +0100 |
wenzelm |
discontinued obsolete function sys_error and exception SYS_ERROR;
|
changeset |
files
|
Wed, 03 Nov 2010 11:11:49 +0100 |
wenzelm |
replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
|
changeset |
files
|
Wed, 03 Nov 2010 11:06:22 +0100 |
wenzelm |
replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
|
changeset |
files
|
Wed, 03 Nov 2010 10:51:40 +0100 |
wenzelm |
try_param_tac: plain user error appears more appropriate;
|
changeset |
files
|
Wed, 03 Nov 2010 10:48:55 +0100 |
wenzelm |
replaced ancient sys_error by raise Fail, assuming that the latter is not handled specifically by the environment;
|
changeset |
files
|
Wed, 03 Nov 2010 10:20:37 +0100 |
wenzelm |
eliminated dead code;
|
changeset |
files
|
Wed, 03 Nov 2010 10:18:05 +0100 |
wenzelm |
more conventional exceptions for abstract syntax operations -- eliminated ancient SYS_ERROR;
|
changeset |
files
|
Wed, 03 Nov 2010 08:29:32 +0100 |
nipkow |
removed assumption
|
changeset |
files
|
Tue, 02 Nov 2010 21:59:21 +0100 |
wenzelm |
more on naming tactics;
|
changeset |
files
|
Tue, 02 Nov 2010 21:24:07 +0100 |
wenzelm |
merged
|
changeset |
files
|
Tue, 02 Nov 2010 20:32:33 +0100 |
haftmann |
merged
|
changeset |
files
|
Tue, 02 Nov 2010 16:59:40 +0100 |
haftmann |
tuned proof
|
changeset |
files
|
Tue, 02 Nov 2010 16:48:19 +0100 |
haftmann |
tuned proof
|
changeset |
files
|
Tue, 02 Nov 2010 16:36:33 +0100 |
haftmann |
tuned lemma proposition of properties_for_sort_key
|
changeset |
files
|
Tue, 02 Nov 2010 16:31:57 +0100 |
haftmann |
lemmas sorted_map_same, sorted_same
|
changeset |
files
|
Tue, 02 Nov 2010 16:31:56 +0100 |
haftmann |
lemmas multiset_of_filter, sort_key_by_quicksort
|
changeset |
files
|
Tue, 02 Nov 2010 21:21:07 +0100 |
wenzelm |
more on "Time" in Isabelle/ML;
|
changeset |
files
|
Tue, 02 Nov 2010 20:55:12 +0100 |
wenzelm |
simplified some time constants;
|
changeset |
files
|
Tue, 02 Nov 2010 20:31:46 +0100 |
wenzelm |
added convenience operation seconds: real -> time;
|
changeset |
files
|
Tue, 02 Nov 2010 20:16:56 +0100 |
wenzelm |
avoid catch-all exception handling;
|
changeset |
files
|
Tue, 02 Nov 2010 20:15:57 +0100 |
wenzelm |
eliminated fragile catch-all pattern, based on educated guess about the intended exception;
|
changeset |
files
|
Tue, 02 Nov 2010 12:37:12 +0100 |
traytel |
Attribute map_function -> coercion_map;
|
changeset |
files
|
Sun, 31 Oct 2010 13:26:37 +0100 |
wenzelm |
syntax category "real" subsumes plain "int";
|
changeset |
files
|
Sun, 31 Oct 2010 11:45:45 +0100 |
nipkow |
merged
|
changeset |
files
|
Fri, 29 Oct 2010 17:57:36 +0200 |
nipkow |
Plus -> Sum_Type.Plus
|
changeset |
files
|
Sun, 31 Oct 2010 11:38:09 +0100 |
ballarin |
Minor reformat.
|
changeset |
files
|
Sat, 30 Oct 2010 21:08:20 +0200 |
wenzelm |
support for real valued preferences;
|
changeset |
files
|
Sat, 30 Oct 2010 16:33:58 +0200 |
wenzelm |
support for real valued configuration options;
|
changeset |
files
|
Sat, 30 Oct 2010 15:26:40 +0200 |
wenzelm |
support for floating-point tokens in outer syntax (coinciding with inner syntax version);
|
changeset |
files
|
Fri, 29 Oct 2010 23:15:01 +0200 |
wenzelm |
merged
|
changeset |
files
|
Fri, 29 Oct 2010 21:41:14 +0200 |
krauss |
added rule let_mono
|
changeset |
files
|
Fri, 29 Oct 2010 22:59:40 +0200 |
wenzelm |
CONTRIBUTORS;
|
changeset |
files
|
Fri, 29 Oct 2010 22:54:54 +0200 |
wenzelm |
more sharing of operations, without aliases;
|
changeset |
files
|
Fri, 29 Oct 2010 22:22:36 +0200 |
wenzelm |
simplified data lookup;
|
changeset |
files
|
Fri, 29 Oct 2010 22:19:27 +0200 |
wenzelm |
export declarations by default, to allow other ML packages by-pass concrete syntax;
|
changeset |
files
|
Fri, 29 Oct 2010 22:07:48 +0200 |
wenzelm |
proper signature constraint for ML structure;
|
changeset |
files
|
Fri, 29 Oct 2010 21:49:33 +0200 |
wenzelm |
proper header;
|
changeset |
files
|
Fri, 29 Oct 2010 21:34:07 +0200 |
wenzelm |
Coercive subtyping via subtype constraints, by Dmitriy Traytel (21-Oct-2010).
|
changeset |
files
|
Fri, 29 Oct 2010 18:17:11 +0200 |
boehmes |
updated SMT certificates
|
changeset |
files
|
Fri, 29 Oct 2010 18:17:10 +0200 |
boehmes |
eta-expand built-in constants; also rewrite partially applied natural number terms
|
changeset |
files
|
Fri, 29 Oct 2010 18:17:09 +0200 |
boehmes |
optionally drop assumptions which cannot be preprocessed
|
changeset |
files
|
Fri, 29 Oct 2010 18:17:08 +0200 |
boehmes |
added crafted list of SMT built-in constants
|
changeset |
files
|
Fri, 29 Oct 2010 18:17:06 +0200 |
boehmes |
clarified error message
|
changeset |
files
|
Fri, 29 Oct 2010 18:17:05 +0200 |
boehmes |
tuned
|
changeset |
files
|
Fri, 29 Oct 2010 18:17:04 +0200 |
boehmes |
introduced SMT.distinct as a representation of the solvers' built-in predicate; check that SMT.distinct is always applied to an explicit list
|
changeset |
files
|
Fri, 29 Oct 2010 17:38:57 +0200 |
wenzelm |
merged
|
changeset |
files
|
Fri, 29 Oct 2010 17:28:27 +0200 |
nipkow |
added listrel1
|
changeset |
files
|
Fri, 29 Oct 2010 17:25:22 +0200 |
nipkow |
hide Sum_Type.Plus
|
changeset |
files
|
Fri, 29 Oct 2010 16:51:20 +0200 |
wenzelm |
merged
|
changeset |
files
|
Fri, 29 Oct 2010 16:04:35 +0200 |
haftmann |
added user aliasses (still unclear how to specify names with whitespace contained)
|
changeset |
files
|
Fri, 29 Oct 2010 14:06:10 +0200 |
haftmann |
merged
|
changeset |
files
|
Fri, 29 Oct 2010 14:03:02 +0200 |
haftmann |
tuned structure of theory
|
changeset |
files
|
Fri, 29 Oct 2010 13:49:49 +0200 |
haftmann |
remove term_of equations for Heap type explicitly
|
changeset |
files
|
Fri, 29 Oct 2010 12:49:05 +0200 |
blanchet |
no need for setting up the kodkodi environment since Kodkodi 1.2.9
|
changeset |
files
|
Fri, 29 Oct 2010 12:49:05 +0200 |
blanchet |
fixed order of quantifier instantiation in new Skolemizer
|
changeset |
files
|
Fri, 29 Oct 2010 12:49:05 +0200 |
blanchet |
restructure Skolemization code slightly
|
changeset |
files
|
Fri, 29 Oct 2010 12:49:05 +0200 |
blanchet |
ensure that MESON correctly preserves the name of variables (needed by the new Skolemizer)
|
changeset |
files
|
Fri, 29 Oct 2010 12:49:05 +0200 |
blanchet |
more work on new Skolemizer without Hilbert_Choice
|
changeset |
files
|
Fri, 29 Oct 2010 12:49:05 +0200 |
blanchet |
fix cluster numbering in the absense of Hilbert_Choice (reverts acde1b606b0e, effectively reintroducing most of 0bfaaa81fc62)
|
changeset |
files
|
Fri, 29 Oct 2010 12:49:05 +0200 |
blanchet |
prevent type errors because of inconsistent skolem Var types by giving fresh indices to Skolems
|
changeset |
files
|
Fri, 29 Oct 2010 12:49:05 +0200 |
blanchet |
make handling of parameters more robust, by querying the goal
|
changeset |
files
|
Fri, 29 Oct 2010 11:35:28 +0200 |
haftmann |
actually pass "verbose" argument
|
changeset |
files
|
Fri, 29 Oct 2010 16:16:10 +0200 |
wenzelm |
eliminated obsolete \_ escape;
|
changeset |
files
|
Fri, 29 Oct 2010 11:49:56 +0200 |
wenzelm |
eliminated obsolete \_ escapes in rail environments;
|
changeset |
files
|
Fri, 29 Oct 2010 11:35:47 +0200 |
wenzelm |
proper markup of formal text;
|
changeset |
files
|
Fri, 29 Oct 2010 11:07:21 +0200 |
wenzelm |
merged
|
changeset |
files
|
Fri, 29 Oct 2010 11:04:41 +0200 |
krauss |
hide_const various constants, in particular to avoid ugly qualifiers in HOLCF
|
changeset |
files
|
Fri, 29 Oct 2010 10:40:36 +0200 |
blanchet |
reverted e31e3f0071d4 because "foo.bar(5)" (with quotes) is wrong
|
changeset |
files
|
Fri, 29 Oct 2010 10:14:49 +0200 |
Lars Noschinski |
merged
|
changeset |
files
|
Wed, 22 Sep 2010 09:56:39 +0200 |
Lars Noschinski |
Remove unnecessary premise of mult1_union
|
changeset |
files
|
Fri, 29 Oct 2010 08:44:49 +0200 |
bulwahn |
adapting HOL-Mutabelle to changes in quickcheck
|
changeset |
files
|
Fri, 29 Oct 2010 08:44:46 +0200 |
bulwahn |
NEWS
|
changeset |
files
|
Fri, 29 Oct 2010 08:44:44 +0200 |
bulwahn |
changed global fixed timeout to a configurable timeout for quickcheck; test parameters in quickcheck are now fully passed around with the context
|
changeset |
files
|
Fri, 29 Oct 2010 08:44:43 +0200 |
bulwahn |
updating documentation on quickcheck in the Isar reference
|
changeset |
files
|
Thu, 28 Oct 2010 18:36:34 +0200 |
bulwahn |
merged
|
changeset |
files
|
Thu, 28 Oct 2010 17:28:45 +0200 |
bulwahn |
adding a simple check to only run with a SWI-Prolog version known to work
|
changeset |
files
|
Thu, 28 Oct 2010 23:54:39 +0200 |
wenzelm |
tuned messages;
|
changeset |
files
|
Thu, 28 Oct 2010 23:19:52 +0200 |
wenzelm |
discontinued obsolete ML antiquotation @{theory_ref};
|
changeset |
files
|
Thu, 28 Oct 2010 22:59:33 +0200 |
wenzelm |
tuned;
|
changeset |
files
|
Thu, 28 Oct 2010 22:39:59 +0200 |
wenzelm |
moved FOL/ex/Iff_Oracle.thy to HOL/ex where it is more accessible to most readers of isar-ref;
|
changeset |
files
|
Thu, 28 Oct 2010 22:23:11 +0200 |
wenzelm |
type attribute is derived concept outside the kernel;
|
changeset |
files
|
Thu, 28 Oct 2010 22:12:08 +0200 |
wenzelm |
preserve original source position of exn;
|
changeset |
files
|
Thu, 28 Oct 2010 22:11:06 +0200 |
wenzelm |
handle Type.TYPE_MATCH, not arbitrary exceptions via MATCH_TYPE variable;
|
changeset |
files
|
Thu, 28 Oct 2010 22:04:00 +0200 |
wenzelm |
use Exn.interruptible_capture to keep user-code interruptible (Exn.capture not immediately followed by Exn.release here);
|
changeset |
files
|
Thu, 28 Oct 2010 21:59:01 +0200 |
wenzelm |
added Exn.interruptible_capture, which reraises interrupts as required by user-code (when Exn.capture is not immediately followed by Exn.release);
|
changeset |
files
|
Thu, 28 Oct 2010 21:52:33 +0200 |
wenzelm |
eliminated dead code;
|
changeset |
files
|
Thu, 28 Oct 2010 21:51:34 +0200 |
wenzelm |
tuned white-space;
|
changeset |
files
|
Thu, 28 Oct 2010 17:54:25 +0200 |
nipkow |
merged
|
changeset |
files
|
Thu, 28 Oct 2010 17:54:09 +0200 |
nipkow |
added lemmas about listrel(1)
|
changeset |
files
|
Thu, 28 Oct 2010 17:25:46 +0200 |
wenzelm |
tuned;
|
changeset |
files
|
Thu, 28 Oct 2010 15:10:34 +0200 |
wenzelm |
merged
|
changeset |
files
|
Thu, 28 Oct 2010 12:33:24 +0200 |
blanchet |
support non-identifier-like fact names in Sledgehammer (e.g., "my lemma") by quoting them
|
changeset |
files
|
Thu, 28 Oct 2010 10:38:29 +0200 |
blanchet |
merged
|
changeset |
files
|
Thu, 28 Oct 2010 09:40:57 +0200 |
blanchet |
clear identification
|
changeset |
files
|
Thu, 28 Oct 2010 09:36:51 +0200 |
blanchet |
clear identification;
|
changeset |
files
|
Thu, 28 Oct 2010 09:29:57 +0200 |
blanchet |
clear identification
|
changeset |
files
|
Wed, 27 Oct 2010 19:14:33 +0200 |
blanchet |
reintroduced Auto Try, but this time really off by default -- and leave some classical+simp reasoners out for Auto Try (but keep them for Try)
|
changeset |
files
|
Wed, 27 Oct 2010 16:32:13 +0200 |
blanchet |
do not let Metis be confused by higher-order reasoning leading to literals of the form "~ ~ p", which are really the same as "p"
|
changeset |
files
|
Wed, 27 Oct 2010 09:22:40 +0200 |
blanchet |
generalize to handle any prover (not just E)
|
changeset |
files
|
Wed, 27 Oct 2010 11:11:35 -0700 |
huffman |
merged
|
changeset |
files
|
Wed, 27 Oct 2010 11:10:36 -0700 |
huffman |
make domain package work with non-cpo argument types
|
changeset |
files
|
Wed, 27 Oct 2010 11:06:53 -0700 |
huffman |
make op -->> infixr, to match op --->
|
changeset |
files
|
Tue, 26 Oct 2010 14:19:59 -0700 |
huffman |
use Named_Thms instead of Theory_Data for some domain package theorems
|
changeset |
files
|
Tue, 26 Oct 2010 09:00:07 -0700 |
huffman |
change types of ML commands add_domain, add_new_domain to take 'sort' instead of 'string option'
|
changeset |
files
|
Tue, 26 Oct 2010 08:36:52 -0700 |
huffman |
use Term.add_tfreesT
|
changeset |
files
|
Sun, 24 Oct 2010 15:42:57 -0700 |
huffman |
rename case combinators generated by domain package to 'foo_case' instead of 'foo_when'
|
changeset |
files
|
Sun, 24 Oct 2010 15:19:17 -0700 |
huffman |
rename constant 'one_when' to 'one_case'
|
changeset |
files
|
Wed, 27 Oct 2010 16:40:34 +0200 |
haftmann |
merged
|
changeset |
files
|
Wed, 27 Oct 2010 16:40:31 +0200 |
haftmann |
sorting: avoid _key suffix if lemma applies both to simple and generalized variant; generalized insort_insert to insort_insert_key; additional lemmas
|
changeset |
files
|
Wed, 27 Oct 2010 13:46:30 +0200 |
krauss |
regenerated keyword file
|
changeset |
files
|
Wed, 27 Oct 2010 08:58:03 +0200 |
boehmes |
made SML/NJ happy
|
changeset |
files
|
Tue, 26 Oct 2010 21:51:04 +0200 |
blanchet |
adapted SMT solver error handling to reflect latest changes in "SMT_Solver"
|
changeset |
files
|
Tue, 26 Oct 2010 21:43:50 +0200 |
blanchet |
better list of irrelevant SMT constants
|
changeset |
files
|
Tue, 26 Oct 2010 21:34:01 +0200 |
blanchet |
if "debug" is on, print list of relevant facts (poweruser request);
|
changeset |
files
|
Tue, 26 Oct 2010 21:01:28 +0200 |
blanchet |
standardize on "fact" terminology (vs. "axiom" or "theorem") in Sledgehammer -- but keep "Axiom" in the lower-level "ATP_Problem" module
|
changeset |
files
|
Tue, 26 Oct 2010 20:12:33 +0200 |
blanchet |
"Nitpick" -> "Sledgehammer";
|
changeset |
files
|
Tue, 26 Oct 2010 20:09:38 +0200 |
blanchet |
merge
|
changeset |
files
|
Tue, 26 Oct 2010 16:59:19 +0200 |
blanchet |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 16:56:54 +0200 |
blanchet |
remove needless context argument;
|
changeset |
files
|
Tue, 26 Oct 2010 17:35:54 +0200 |
boehmes |
use proper context
|
changeset |
files
|
Tue, 26 Oct 2010 17:35:52 +0200 |
boehmes |
trace assumptions before giving them to the SMT solver
|
changeset |
files
|
Tue, 26 Oct 2010 17:35:51 +0200 |
boehmes |
capture out-of-memory warnings of Z3 and turn them into proper exceptions; be more precise about SMT solver run-time: return NONE instead of ~1
|
changeset |
files
|
Tue, 26 Oct 2010 17:35:49 +0200 |
boehmes |
honor choice of either local or remote SMT solver only for smt_filter and keep default behaviour for the SMT tactic; omit messages when running smt_filter
|
changeset |
files
|
Tue, 26 Oct 2010 16:39:21 +0200 |
haftmann |
include ATP in theory List -- avoid theory edge by-passing the prominent list theory
|
changeset |
files
|
Tue, 26 Oct 2010 15:06:36 +0200 |
krauss |
fixed typo
|
changeset |
files
|
Tue, 26 Oct 2010 15:01:39 +0200 |
blanchet |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 15:01:02 +0200 |
blanchet |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 14:49:48 +0200 |
blanchet |
put theorems added using "add:" at the beginning of the list returned by the relevance filter, so that they don't get truncated away
|
changeset |
files
|
Tue, 26 Oct 2010 14:48:55 +0200 |
blanchet |
tuning
|
changeset |
files
|
Tue, 26 Oct 2010 15:00:57 +0200 |
haftmann |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 14:06:22 +0200 |
haftmann |
consider base sorts of superclasses simultaneously during processing of class specification -- avoids clash of different base sorts
|
changeset |
files
|
Tue, 26 Oct 2010 15:00:42 +0200 |
haftmann |
more general treatment of type argument in code certificates for operations on abstract types
|
changeset |
files
|
Tue, 26 Oct 2010 14:11:34 +0200 |
haftmann |
partial_function is a declaration command
|
changeset |
files
|
Tue, 26 Oct 2010 14:06:21 +0200 |
blanchet |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 13:50:57 +0200 |
blanchet |
proper error handling for SMT solvers in Sledgehammer
|
changeset |
files
|
Tue, 26 Oct 2010 13:50:18 +0200 |
krauss |
NEWS
|
changeset |
files
|
Tue, 26 Oct 2010 13:17:37 +0200 |
blanchet |
merge
|
changeset |
files
|
Tue, 26 Oct 2010 13:16:43 +0200 |
blanchet |
integrated "smt" proof method with Sledgehammer
|
changeset |
files
|
Tue, 26 Oct 2010 13:19:31 +0200 |
krauss |
fixed confusion introduced in 008dc2d2c395
|
changeset |
files
|
Tue, 26 Oct 2010 12:23:39 +0200 |
blanchet |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 12:17:19 +0200 |
blanchet |
reverted e7a80c6752c9 -- there's not much point in putting a diagnosis tool (as opposed to a proof method) in Plain, but more importantly Sledgehammer must be in Main to use SMT solvers
|
changeset |
files
|
Tue, 26 Oct 2010 12:19:31 +0200 |
haftmann |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 12:19:22 +0200 |
haftmann |
tuned
|
changeset |
files
|
Tue, 26 Oct 2010 12:21:45 +0200 |
krauss |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 12:19:02 +0200 |
krauss |
use partial_function instead of MREC combinator; curried rev'
|
changeset |
files
|
Tue, 26 Oct 2010 12:19:02 +0200 |
krauss |
added Heap monad instance of partial_function package
|
changeset |
files
|
Tue, 26 Oct 2010 12:19:02 +0200 |
krauss |
added Spec_Rule declaration to partial_function
|
changeset |
files
|
Tue, 26 Oct 2010 12:19:01 +0200 |
krauss |
basic documentation for command partial_function
|
changeset |
files
|
Tue, 26 Oct 2010 12:19:01 +0200 |
krauss |
remove outdated "(otherwise)" syntax from manual
|
changeset |
files
|
Tue, 26 Oct 2010 12:19:01 +0200 |
krauss |
declare recursive equation as ".simps", in accordance with other packages
|
changeset |
files
|
Tue, 26 Oct 2010 12:16:08 +0200 |
haftmann |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 12:15:55 +0200 |
haftmann |
dropped accidental doubled computation
|
changeset |
files
|
Tue, 26 Oct 2010 11:51:09 +0200 |
boehmes |
optionally force the remote version of an SMT solver to be executed
|
changeset |
files
|
Tue, 26 Oct 2010 11:49:36 +0200 |
boehmes |
tuned
|
changeset |
files
|
Tue, 26 Oct 2010 11:49:23 +0200 |
boehmes |
added a mode to only filter assumptions used in a Z3 proof (in which no proof reconstruction is performed)
|
changeset |
files
|
Tue, 26 Oct 2010 11:46:19 +0200 |
boehmes |
changed SMT configuration options; updated SMT certificates
|
changeset |
files
|
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
|
changeset |
files
|
Tue, 26 Oct 2010 11:39:26 +0200 |
boehmes |
keep track of theorems initially given to SMT (even if they are rewritten); provide interface to filter theorems necessary for SMT proofs
|
changeset |
files
|
Tue, 26 Oct 2010 11:31:03 +0200 |
blanchet |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 11:21:08 +0200 |
blanchet |
merge
|
changeset |
files
|
Tue, 26 Oct 2010 11:11:23 +0200 |
blanchet |
clearer error messages
|
changeset |
files
|
Tue, 26 Oct 2010 11:10:00 +0200 |
blanchet |
renaming
|
changeset |
files
|
Thu, 28 Oct 2010 15:06:47 +0200 |
wenzelm |
back again to non-Apple font rendering (cf. 4977324373f2);
|
changeset |
files
|
Thu, 28 Oct 2010 14:56:14 +0200 |
wenzelm |
dock isabelle-session at bottom (again, cf. 37bdc2220cf8) to ensure that controls are fully visible;
|
changeset |
files
|
Tue, 26 Oct 2010 16:56:07 +0200 |
wenzelm |
disable broken popups for now;
|
changeset |
files
|
Tue, 26 Oct 2010 15:57:16 +0200 |
wenzelm |
tuned;
|
changeset |
files
|
Tue, 26 Oct 2010 11:31:22 +0200 |
wenzelm |
do not handle arbitrary exceptions;
|
changeset |
files
|
Tue, 26 Oct 2010 11:23:27 +0200 |
wenzelm |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 11:20:14 +0200 |
haftmann |
Code_Runtime.trace
|
changeset |
files
|
Tue, 26 Oct 2010 11:22:18 +0200 |
wenzelm |
proper markup of uninterpreted ML text as @{ML_text}, not @{verbatim};
|
changeset |
files
|
Tue, 26 Oct 2010 11:06:12 +0200 |
wenzelm |
merged
|
changeset |
files
|
Tue, 26 Oct 2010 11:00:17 +0200 |
blanchet |
improved English
|
changeset |
files
|
Tue, 26 Oct 2010 10:59:28 +0200 |
blanchet |
whitespace tuning
|
changeset |
files
|
Tue, 26 Oct 2010 10:57:04 +0200 |
blanchet |
no need to encode theorem number twice in skolem names
|
changeset |
files
|
Tue, 26 Oct 2010 10:39:52 +0200 |
blanchet |
tuning
|
changeset |
files
|
Tue, 26 Oct 2010 09:40:20 +0200 |
blanchet |
make SML/NJ happy
|
changeset |
files
|
Mon, 25 Oct 2010 21:17:16 +0200 |
bulwahn |
relaxing the filtering condition for getting specifications from Spec_Rules
|
changeset |
files
|
Mon, 25 Oct 2010 21:17:16 +0200 |
bulwahn |
adding new predicate compiler files to the IsaMakefile
|
changeset |
files
|
Mon, 25 Oct 2010 21:17:15 +0200 |
bulwahn |
using mode_eq instead of op = for lookup in the predicate compiler
|
changeset |
files
|
Mon, 25 Oct 2010 21:17:14 +0200 |
bulwahn |
renaming split_modeT' to split_modeT
|
changeset |
files
|
Mon, 25 Oct 2010 21:17:13 +0200 |
bulwahn |
options as first argument to check functions
|
changeset |
files
|
Mon, 25 Oct 2010 21:17:12 +0200 |
bulwahn |
changing test parameters in examples to get to a result within the global timelimit
|
changeset |
files
|
Mon, 25 Oct 2010 21:17:11 +0200 |
bulwahn |
adding a global fixed timeout to quickcheck
|
changeset |
files
|
Mon, 25 Oct 2010 21:17:10 +0200 |
bulwahn |
adding a global time limit to the values command
|
changeset |
files
|
Mon, 25 Oct 2010 22:47:02 +0200 |
wenzelm |
explicit message_output thread, with flushing after timeout, ensure atomic user-operations without the danger of IO Interrupt;
|
changeset |
files
|
Mon, 25 Oct 2010 21:23:09 +0200 |
wenzelm |
more explicit indication of Output.Private_Hooks (still public to accomodate clones of Proof General for now);
|
changeset |
files
|
Mon, 25 Oct 2010 21:06:56 +0200 |
wenzelm |
renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
|
changeset |
files
|
Mon, 25 Oct 2010 20:24:13 +0200 |
wenzelm |
explicitly qualify type Output.output, which is a slightly odd internal feature;
|
changeset |
files
|
Mon, 25 Oct 2010 16:52:20 +0200 |
wenzelm |
export main ML entry by default;
|
changeset |
files
|
Mon, 25 Oct 2010 16:41:23 +0200 |
wenzelm |
observe Isabelle/ML coding standards;
|
changeset |
files
|
Mon, 25 Oct 2010 16:18:00 +0200 |
wenzelm |
merged
|
changeset |
files
|
Mon, 25 Oct 2010 16:17:16 +0200 |
wenzelm |
significantly improved Isabelle/Isar implementation manual;
|
changeset |
files
|
Mon, 25 Oct 2010 16:14:40 +0200 |
wenzelm |
misc tuning;
|
changeset |
files
|
Mon, 25 Oct 2010 11:39:52 +0200 |
wenzelm |
removed some remains of Output.debug (follow-up to fce2202892c4);
|
changeset |
files
|
Mon, 25 Oct 2010 11:22:30 +0200 |
wenzelm |
recovered some odd two-dimensional layout;
|
changeset |
files
|
Mon, 25 Oct 2010 13:36:20 +0200 |
haftmann |
merged
|
changeset |
files
|
Mon, 25 Oct 2010 13:34:58 +0200 |
haftmann |
dropped (almost) redundant distinct.induct rule; distinct_simps again named distinct.simps
|
changeset |
files
|
Mon, 25 Oct 2010 13:34:57 +0200 |
haftmann |
moved sledgehammer to Plain; tuned dependencies
|
changeset |
files
|
Mon, 25 Oct 2010 13:34:57 +0200 |
haftmann |
CONTRIBUTORS
|
changeset |
files
|
Mon, 25 Oct 2010 12:24:38 +0200 |
blanchet |
merge
|
changeset |
files
|
Mon, 25 Oct 2010 11:42:05 +0200 |
blanchet |
merged
|
changeset |
files
|
Mon, 25 Oct 2010 10:38:41 +0200 |
blanchet |
updated keywords
|
changeset |
files
|
Mon, 25 Oct 2010 10:30:46 +0200 |
blanchet |
introduced manual version of "Auto Solve" as "solve_direct"
|
changeset |
files
|
Mon, 25 Oct 2010 09:29:43 +0200 |
blanchet |
make "sledgehammer_params" work on single-threaded platforms
|
changeset |
files
|
Fri, 22 Oct 2010 18:31:45 +0200 |
blanchet |
tuning
|
changeset |
files
|
Fri, 22 Oct 2010 18:24:10 +0200 |
blanchet |
handle timeouts (to prevent failure from other threads);
|
changeset |
files
|
Mon, 25 Oct 2010 12:11:12 +0200 |
haftmann |
update keywords
|
changeset |
files
|
Mon, 25 Oct 2010 10:45:22 +0200 |
krauss |
some partial_function examples
|
changeset |
files
|
Mon, 25 Oct 2010 11:16:23 +0200 |
wenzelm |
added ML antiquotation @{assert};
|
changeset |
files
|
Mon, 25 Oct 2010 11:01:00 +0200 |
wenzelm |
updated keywords;
|
changeset |
files
|
Sat, 23 Oct 2010 23:42:04 +0200 |
krauss |
integrated partial_function into HOL-Plain
|
changeset |
files
|
Sat, 23 Oct 2010 23:41:19 +0200 |
krauss |
first version of partial_function package
|
changeset |
files
|
Sat, 23 Oct 2010 23:39:37 +0200 |
krauss |
Complete_Partial_Order.thy: complete partial orders over arbitrary chains, with fixpoint theorem
|
changeset |
files
|
Mon, 25 Oct 2010 08:08:08 +0200 |
bulwahn |
merged
|
changeset |
files
|
Fri, 22 Oct 2010 18:38:59 +0200 |
bulwahn |
splitting Hotel Key card example into specification and the two tests for counter example generation
|
changeset |
files
|
Fri, 22 Oct 2010 18:38:59 +0200 |
bulwahn |
adding generator quickcheck
|
changeset |
files
|
Fri, 22 Oct 2010 18:38:59 +0200 |
bulwahn |
restructuring values command and adding generator compilation
|
changeset |
files
|
Fri, 22 Oct 2010 18:38:59 +0200 |
bulwahn |
moving general functions from core_data to predicate_compile_aux
|
changeset |
files
|
Fri, 22 Oct 2010 18:38:59 +0200 |
bulwahn |
updating to new notation in commented examples
|
changeset |
files
|