Wed, 10 Nov 2010 17:53:41 +0100 |
wenzelm |
use official/portable Multithreading.max_threads_value, which is also subject to user preferences (NB: Thread.numProcessors is apt to lead to surprises like very high numbers for systems with hyperthreading);
|
changeset |
files
|
Wed, 10 Nov 2010 16:05:15 +0100 |
wenzelm |
merged
|
changeset |
files
|
Wed, 10 Nov 2010 09:03:07 +0100 |
blanchet |
make SML/NJ happy
|
changeset |
files
|
Tue, 09 Nov 2010 16:18:40 +0100 |
haftmann |
merged
|
changeset |
files
|
Tue, 09 Nov 2010 14:02:14 +0100 |
haftmann |
slightly changed fun_map_def
|
changeset |
files
|
Tue, 09 Nov 2010 14:02:14 +0100 |
haftmann |
fun_rel_def is no simp rule by default
|
changeset |
files
|
Tue, 09 Nov 2010 14:02:13 +0100 |
haftmann |
more appropriate specification packages; fun_rel_def is no simp rule by default
|
changeset |
files
|
Tue, 09 Nov 2010 14:02:13 +0100 |
haftmann |
type annotations in specifications; fun_rel_def is no simp rule by default; slightly changed fun_map_def; more on predicates on relation functions; proper HOL equations in definitions
|
changeset |
files
|
Tue, 09 Nov 2010 14:02:13 +0100 |
haftmann |
more appropriate specification packages; fun_rel_def is no simp rule by default
|
changeset |
files
|
Tue, 09 Nov 2010 14:02:12 +0100 |
haftmann |
type annotations in specifications; fun_rel_def is no simp rule by default
|
changeset |
files
|
Tue, 09 Nov 2010 14:02:12 +0100 |
haftmann |
fun_rel_def is no simp rule by default
|
changeset |
files
|
Tue, 09 Nov 2010 14:00:10 +0000 |
paulson |
merged
|
changeset |
files
|
Tue, 09 Nov 2010 13:59:37 +0000 |
paulson |
tidied using metis
|
changeset |
files
|
Wed, 10 Nov 2010 15:59:23 +0100 |
wenzelm |
manage folding via sidekick by default;
|
changeset |
files
|
Wed, 10 Nov 2010 15:47:56 +0100 |
wenzelm |
eliminated obsolete heading category -- superseded by heading_level;
|
changeset |
files
|
Wed, 10 Nov 2010 15:43:06 +0100 |
wenzelm |
treat main theory commands like headings, and nest anything else inside;
|
changeset |
files
|
Wed, 10 Nov 2010 15:42:20 +0100 |
wenzelm |
proper treatment of equal heading level;
|
changeset |
files
|
Wed, 10 Nov 2010 15:41:29 +0100 |
wenzelm |
added missing Keyword.THY_SCHEMATIC_GOAL;
|
changeset |
files
|
Wed, 10 Nov 2010 15:17:25 +0100 |
wenzelm |
default Sidekick parser based on section headings;
|
changeset |
files
|
Wed, 10 Nov 2010 15:00:40 +0100 |
wenzelm |
some support for nested source structure, based on section headings;
|
changeset |
files
|
Wed, 10 Nov 2010 11:44:35 +0100 |
wenzelm |
tuned;
|
changeset |
files
|
Tue, 09 Nov 2010 23:24:46 +0100 |
wenzelm |
misc tuning and simplification, using Isabelle_Sidekick.Asset (not sidekick.Asset, which is dynamically dispatched to slightly different semantics);
|
changeset |
files
|
Tue, 09 Nov 2010 22:37:10 +0100 |
wenzelm |
updated version;
|
changeset |
files
|
Tue, 09 Nov 2010 21:52:05 +0100 |
wenzelm |
private counter, to keep externalized ids a bit smaller;
|
changeset |
files
|
Tue, 09 Nov 2010 21:44:19 +0100 |
wenzelm |
added general Synchronized.counter convenience;
|
changeset |
files
|
Tue, 09 Nov 2010 21:13:06 +0100 |
wenzelm |
explicitly identify forked/joined tasks;
|
changeset |
files
|
Tue, 09 Nov 2010 11:27:58 +0100 |
wenzelm |
accomodate old manuals that include pdfsetup.sty without isabelle.sty;
|
changeset |
files
|
Tue, 09 Nov 2010 11:17:15 +0100 |
wenzelm |
merged
|
changeset |
files
|
Mon, 08 Nov 2010 23:02:20 +0100 |
krauss |
removed type-inference-like behaviour from relation_tac completely; tuned
|
changeset |
files
|
Mon, 08 Nov 2010 20:55:27 +0100 |
wenzelm |
avoid clash of \<upharpoonright> vs. \<restriction> (cf. 666ea7e62384 and 3c49dbece0a8);
|
changeset |
files
|
Mon, 08 Nov 2010 20:50:56 +0100 |
wenzelm |
explicitly check uniqueness of symbol recoding;
|
changeset |
files
|
Mon, 08 Nov 2010 17:44:47 +0100 |
wenzelm |
more hints on building and running Isabelle/jEdit from command line;
|
changeset |
files
|
Mon, 08 Nov 2010 14:41:11 +0100 |
wenzelm |
merged
|
changeset |
files
|
Mon, 08 Nov 2010 14:33:54 +0100 |
blanchet |
merge
|
changeset |
files
|
Mon, 08 Nov 2010 14:33:30 +0100 |
blanchet |
reduce the number of monomorphization iterations from 10 (the default) to 4, in the interest of faster SMT solving
|
changeset |
files
|
Mon, 08 Nov 2010 05:07:18 -0800 |
huffman |
merged
|
changeset |
files
|
Sat, 06 Nov 2010 10:01:00 -0700 |
huffman |
merged
|
changeset |
files
|
Fri, 05 Nov 2010 15:15:28 -0700 |
huffman |
(infixl "<<" 55) -> (infix "<<" 50)
|
changeset |
files
|
Wed, 03 Nov 2010 17:22:25 -0700 |
huffman |
simplify some proofs
|
changeset |
files
|
Wed, 03 Nov 2010 17:06:21 -0700 |
huffman |
remove unnecessary stuff from Discrete.thy
|
changeset |
files
|
Wed, 03 Nov 2010 16:39:23 -0700 |
huffman |
remove some unnecessary lemmas; move monofun_LAM to Cfun.thy
|
changeset |
files
|
Wed, 03 Nov 2010 15:57:39 -0700 |
huffman |
add lemma eq_imp_below
|
changeset |
files
|
Wed, 03 Nov 2010 15:47:46 -0700 |
huffman |
discontinue a bunch of legacy theorem names
|
changeset |
files
|
Wed, 03 Nov 2010 15:31:24 -0700 |
huffman |
move a few admissibility lemmas into FOCUS/Stream_adm.thy
|
changeset |
files
|
Wed, 03 Nov 2010 15:03:16 -0700 |
huffman |
simplify some proofs
|
changeset |
files
|
Mon, 08 Nov 2010 13:53:18 +0100 |
blanchet |
compile -- 7550b2cba1cb broke the build
|
changeset |
files
|
Mon, 08 Nov 2010 13:25:00 +0100 |
blanchet |
merge
|
changeset |
files
|
Mon, 08 Nov 2010 09:10:44 +0100 |
blanchet |
recognize Vampire error
|
changeset |
files
|
Mon, 08 Nov 2010 12:13:51 +0100 |
boehmes |
return the process return code along with the process outputs
|
changeset |
files
|
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)
|
changeset |
files
|
Mon, 08 Nov 2010 11:49:28 +0100 |
haftmann |
merged
|
changeset |
files
|
Mon, 08 Nov 2010 10:56:48 +0100 |
haftmann |
corrected slip: must keep constant map, not type map; tuned code
|
changeset |
files
|
Mon, 08 Nov 2010 10:43:24 +0100 |
haftmann |
constructors to datatypes in code_reflect can be globbed; dropped unused code
|
changeset |
files
|
Mon, 08 Nov 2010 09:25:43 +0100 |
bulwahn |
adding code and theory for smallvalue generators, but do not setup the interpretation yet
|
changeset |
files
|
Mon, 08 Nov 2010 02:33:48 +0100 |
blanchet |
make sure the SMT solver runs several iterations by lowering the timeout at each iteration -- yields better results in practice
|
changeset |
files
|
Mon, 08 Nov 2010 02:32:27 +0100 |
blanchet |
better detection of completely irrelevant facts
|
changeset |
files
|
Sun, 07 Nov 2010 18:19:04 +0100 |
blanchet |
always use a hard timeout in Mirabelle
|
changeset |
files
|
Sun, 07 Nov 2010 18:15:13 +0100 |
blanchet |
use "smt" (rather than "metis") to reconstruct SMT proofs
|
changeset |
files
|
Sun, 07 Nov 2010 18:03:24 +0100 |
blanchet |
don't pass too many facts on the first iteration of the SMT solver
|
changeset |
files
|
Sun, 07 Nov 2010 18:02:02 +0100 |
blanchet |
catch TimeOut exception
|
changeset |
files
|