2009-11-05 |
wenzelm |
misc tuning and clarification;
|
changeset |
files
|
2009-11-05 |
wenzelm |
scalable version of Named_Thms, using Item_Net;
|
changeset |
files
|
2009-11-05 |
wenzelm |
merged
|
changeset |
files
|
2009-11-05 |
wenzelm |
merged
|
changeset |
files
|
2009-11-05 |
wenzelm |
more accurate cleanup;
|
changeset |
files
|
2009-11-05 |
wenzelm |
merged
|
changeset |
files
|
2009-11-05 |
wenzelm |
more accurate dependencies;
|
changeset |
files
|
2009-11-05 |
boehmes |
merged
|
changeset |
files
|
2009-11-05 |
boehmes |
handle let expressions inside terms by unfolding (instead of raising an exception),
|
changeset |
files
|
2009-11-05 |
boehmes |
shorter names for variables and verification conditions,
|
changeset |
files
|
2009-11-05 |
boehmes |
added references to HOL-Boogie papers
|
changeset |
files
|
2009-11-05 |
wenzelm |
tuned header;
|
changeset |
files
|
2009-11-05 |
wenzelm |
made SML/NJ happy;
|
changeset |
files
|
2009-11-05 |
wenzelm |
eliminated funny record patterns and made SML/NJ happy;
|
changeset |
files
|
2009-11-05 |
wenzelm |
proper header;
|
changeset |
files
|
2009-11-05 |
wenzelm |
more accurate dependencies;
|
changeset |
files
|
2009-11-05 |
wenzelm |
merged
|
changeset |
files
|
2009-11-04 |
krauss |
added Tree23 to IsaMakefile
|
changeset |
files
|
2009-11-04 |
nipkow |
New
|
changeset |
files
|
2009-11-04 |
nipkow |
merged
|
changeset |
files
|
2009-11-04 |
nipkow |
fixed order of parameters in induction rules
|
changeset |
files
|
2009-11-04 |
krauss |
added bulwahn to isatest mailings
|
changeset |
files
|
2009-11-04 |
nipkow |
merged
|
changeset |
files
|
2009-11-04 |
nipkow |
Completely overhauled
|
changeset |
files
|
2009-11-04 |
huffman |
better error handling for fixrec_simp
|
changeset |
files
|
2009-11-04 |
huffman |
add more fixrec_simp rules
|
changeset |
files
|
2009-11-04 |
huffman |
fixrec examples use fixrec_simp instead of fixpat
|
changeset |
files
|
2009-11-04 |
huffman |
domain package registers fixrec_simp lemmas
|
changeset |
files
|
2009-11-04 |
huffman |
merged
|
changeset |
files
|
2009-11-04 |
huffman |
add fixrec_simp attribute and method (eventually to replace fixpat)
|
changeset |
files
|
2009-11-03 |
boehmes |
proper and unique case names for the split_vc method,
|
changeset |
files
|
2009-11-03 |
haftmann |
merged
|
changeset |
files
|
2009-11-03 |
haftmann |
merged
|
changeset |
files
|
2009-11-03 |
haftmann |
always be qualified -- suspected smartness in fact never worked as expected
|
changeset |
files
|
2009-11-03 |
haftmann |
pretty name for ==>
|
changeset |
files
|
2009-11-03 |
boehmes |
added HOL-Boogie
|
changeset |
files
|
2009-11-03 |
boehmes |
added a specific SMT exception captured by smt_tac (prevents the SMT method from failing with an exception),
|
changeset |
files
|
2009-11-03 |
boehmes |
ignore parsing errors, return empty assignment instead
|
changeset |
files
|
2009-11-05 |
wenzelm |
scheduler: clarified interrupt attributes and handling;
|
changeset |
files
|
2009-11-05 |
wenzelm |
worker_next: plain signalling via work_available only, not scheduler_event;
|
changeset |
files
|
2009-11-04 |
wenzelm |
revert fulfill_proof_future tuning (actually a bit slower due to granularity issues?);
|
changeset |
files
|
2009-11-04 |
wenzelm |
avoid broadcast work_available, use daisy-chained signal instead;
|
changeset |
files
|
2009-11-04 |
wenzelm |
fulfill_proof_future: tuned important special case of singleton promise;
|
changeset |
files
|
2009-11-04 |
wenzelm |
worker_next: treat wait for work_available as Sleeping, not Waiting;
|
changeset |
files
|
2009-11-04 |
wenzelm |
worker activity: distinguish between waiting (formerly active) and sleeping;
|
changeset |
files
|
2009-11-04 |
wenzelm |
tuned;
|
changeset |
files
|
2009-11-04 |
wenzelm |
tuned thread data;
|
changeset |
files
|
2009-11-03 |
wenzelm |
worker_next: ensure that work_available is passed on before sleeping (was occasionally lost when worker configuration changed, causing scheduler deadlock);
|
changeset |
files
|
2009-11-03 |
wenzelm |
slightly leaner and more direct control of worker activity etc.;
|
changeset |
files
|
2009-11-03 |
bulwahn |
adding testcases for code inlining, sets and numerals to the example files of the predicate compiler and its quickcheck prototype; disabling length example
|
changeset |
files
|
2009-11-03 |
bulwahn |
adapted the inlining in the predicate compiler
|
changeset |
files
|
2009-11-03 |
bulwahn |
recursively replacing abstractions by new definitions in the predicate compiler
|
changeset |
files
|
2009-11-03 |
huffman |
merge
|
changeset |
files
|
2009-11-03 |
huffman |
add fixrec support for HOL pair constructor patterns
|
changeset |
files
|
2009-11-03 |
huffman |
define cprod_fun using Pair instead of cpair
|
changeset |
files
|
2009-11-03 |
huffman |
add (LAM (x, y). t) syntax and lemma csplit_Pair
|
changeset |
files
|
2009-11-02 |
krauss |
lexicographic order: run local descent proofs in parallel
|
changeset |
files
|
2009-11-02 |
huffman |
merged
|
changeset |
files
|
2009-11-02 |
huffman |
domain package no longer uses cfst/csnd/cpair
|
changeset |
files
|
2009-11-02 |
krauss |
conceal partial rules depending on config flag (i.e. when called via "fun")
|
changeset |
files
|