Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
removed debug messages; exported to_pred in InductiveSet; added further display function; adjusted mode analysis
2009-08-04, by bulwahn
basic support for components (which imitate the usual Isabelle directory layout);
2009-08-04, by wenzelm
Tuned.
2009-08-02, by berghofe
the derived induction principles can be given an explicit name
2009-08-02, by Christian Urban
updated Variable.import;
2009-08-01, by wenzelm
merged
2009-08-01, by wenzelm
merged
2009-08-01, by wenzelm
modernized generated example session;
2009-07-31, by wenzelm
added Mirabelle
2009-07-31, by boehmes
Quickcheck callable from ML
2009-07-31, by boehmes
future scheduler: uninterruptible cancelation;
2009-08-01, by wenzelm
renamed Multithreading.regular_interrupts to Multithreading.public_interrupts;
2009-08-01, by wenzelm
recovered polyml-5.2 -- need to reload ML-Systems/multithreading.ML after overriding Thread structures;
2009-07-30, by wenzelm
tuned tracing;
2009-07-30, by wenzelm
ISABELLE_USEDIR_OPTIONS: -q 2 by default;
2009-07-30, by wenzelm
merged
2009-07-30, by wenzelm
merged
2009-07-30, by wenzelm
merged
2009-07-30, by haftmann
cleaned up abstract tuple operations and named them consistently
2009-07-29, by haftmann
cleaned up abstract tuple operations and named them consistently
2009-07-29, by haftmann
added Multithreading.sync_wait, which turns enabled interrupts to sync ones, to ensure that wait will reaquire its lock when interrupted;
2009-07-30, by wenzelm
trancl_tac etc.: back to static context -- problem was caused by bad solver in AFP/JiveDataStoreModel;
2009-07-30, by wenzelm
retrofit: more precise handling of locally introduced schematic variables (avoid zero_var_indexes);
2009-07-30, by wenzelm
qualified Subgoal.FOCUS;
2009-07-30, by wenzelm
FOCUS_PREMS as full replacement for METAHYPS, where the conclusion may still contain schematic variables;
2009-07-30, by wenzelm
focus: more precise treatment of schematic variables, only the "visible" part of the text is fixed;
2009-07-30, by wenzelm
Variable.importT/import: return full instantiations, tuned;
2009-07-30, by wenzelm
added certify_inst, certify_instantiate;
2009-07-30, by wenzelm
merged
2009-07-29, by wenzelm
trans_tac: use theory from goal state, not the static context, which seems to be outdated under certain circumstances (why?);
2009-07-29, by wenzelm
proper Jinja-Slicing;
2009-07-29, by wenzelm
merged
2009-07-29, by wenzelm
merged
2009-07-29, by haftmann
abstractions: desymbolize name hint
2009-07-29, by haftmann
added numeral code postprocessor rules on type int
2009-07-29, by haftmann
sos comments modified
2009-07-29, by nipkow
sos documentation
2009-07-29, by nipkow
Added remote-SOS changes by Philipp Meyer
2009-07-29, by nipkow
Functionality for sum of squares to call a remote csdp prover
2009-07-24, by Philipp Meyer
merged
2009-07-28, by wenzelm
updated generated document
2009-07-28, by haftmann
reinserted legacy ML function
2009-07-28, by haftmann
Set.UNIV and Set.empty are mere abbreviations for top and bot
2009-07-28, by haftmann
explicit is better than implicit
2009-07-28, by haftmann
Meson.first_order_resolve: avoid handle _;
2009-07-29, by wenzelm
removed old global get_claset/map_claset;
2009-07-29, by wenzelm
eliminated METAHYPS;
2009-07-28, by wenzelm
Future.shutdown before loading sequentially -- workaround scheduler deadlock;
2009-07-28, by wenzelm
ResAxioms.neg_conjecture_clauses: proper context;
2009-07-28, by wenzelm
neg_conjecture_clauses, neg_clausify_tac: proper context, eliminated METAHYPS;
2009-07-28, by wenzelm
Hilbert_Classical: sequential loading due to @{prf}, which joins within a critical section (via options);
2009-07-28, by wenzelm
eliminated separate Future.enabled -- let Future.join fail explicitly in critical section, instead of entering sequential mode silently;
2009-07-28, by wenzelm
non-critical use_thy;
2009-07-28, by wenzelm
future result: Synchronized.var;
2009-07-28, by wenzelm
added unsynchronized Synchronized.peek;
2009-07-28, by wenzelm
group status: Synchronized.var;
2009-07-28, by wenzelm
tuned;
2009-07-28, by wenzelm
Task_Queue.dequeue: explicit thread;
2009-07-28, by wenzelm
more precise treatment of scheduler_event: continous pulse (50ms) instead of flooding, which was burning many CPU cycles in spare threads;
2009-07-28, by wenzelm
interruptible_task: unified treatment of Multithreading.with_attributes (cf. 9f6461b1c9cc);
2009-07-28, by wenzelm
misc tuning;
2009-07-28, by wenzelm
tuned
2009-07-28, by krauss
moved obsolete same_fst to Recdef.thy
2009-07-28, by krauss
adapted doc to type of "op O"
2009-07-28, by krauss
merged
2009-07-28, by wenzelm
merged
2009-07-27, by wenzelm
merged
2009-07-27, by wenzelm
merged
2009-07-27, by wenzelm
added proof of Kleene_Algebra.star_decomp
2009-07-27, by krauss
added missing proof of RBT.map_of_alist_of (contributed by Peter Lammich)
2009-07-27, by krauss
some lemmas about maps (contributed by Peter Lammich)
2009-07-27, by krauss
"more standard" argument order of relation composition (op O)
2009-07-27, by krauss
added rail antiquotation environment, which coexists with old-style content markup;
2009-07-28, by wenzelm
proper header;
2009-07-28, by wenzelm
proper context for SAT tactics;
2009-07-27, by wenzelm
moved METAHYPS to old_goals.ML (cf. SUBPROOF and FOCUS in subgoal.ML for properly localized versions of the same idea);
2009-07-27, by wenzelm
interruptible: Thread.testInterrupt before changing thread attributes;
2009-07-27, by wenzelm
wait: absorb spurious interrupts;
2009-07-27, by wenzelm
scheduler: shutdown spontaneously (after some delay) if queue is empty;
2009-07-27, by wenzelm
join_next: do not yield, even if overloaded, to minimize "running" tasks;
2009-07-27, by wenzelm
tuned tracing;
2009-07-27, by wenzelm
cancel: improved reactivity due to more careful broadcasting;
2009-07-27, by wenzelm
dequeue_towards: always return active tasks;
2009-07-27, by wenzelm
merged
2009-07-27, by wenzelm
removed unused low-level interrupts;
2009-07-27, by wenzelm
tuned signature;
2009-07-27, by wenzelm
tuned;
2009-07-27, by wenzelm
more specific conditions: scheduler_event, work_available, work_finished -- considereably reduces overhead with many threads;
2009-07-27, by wenzelm
enqueue/finish: return minimal/maximal state of this task;
2009-07-27, by wenzelm
NEWS
2009-07-27, by haftmann
tacticals FOCUS and FOCUS_PARAMS;
2009-07-26, by wenzelm
replaced old METAHYPS by FOCUS;
2009-07-26, by wenzelm
replaced old METAHYPS by FOCUS;
2009-07-26, by wenzelm
added focus_params/FOCUS_PARAMS, which focus on the parameter prefix only;
2009-07-26, by wenzelm
replaced old METAHYPS by FOCUS;
2009-07-26, by wenzelm
tuned eval_tac: eliminated unused METAHYPS (FOCUS fails due to schematic goals);
2009-07-26, by wenzelm
retrofit: actually handle schematic variables -- need to export into original context;
2009-07-26, by wenzelm
merged
2009-07-26, by wenzelm
adapted to changed prefixes
2009-07-26, by haftmann
merged
2009-07-26, by haftmann
improved handling of parameter import; tuned
2009-07-25, by haftmann
explicit is better than implicit
2009-07-25, by haftmann
localized interpretation of min/max-lattice
2009-07-25, by haftmann
adapted to localized interpretation of min/max-lattice
2009-07-25, by haftmann
SUBPROOF/Obtain.result: named params;
2009-07-26, by wenzelm
updated Variable.focus, SUBPROOF, Obtain.result, Goal.finish;
2009-07-26, by wenzelm
advanced retrofit, which allows new subgoals and variables;
2009-07-26, by wenzelm
Variable.focus: named parameters;
2009-07-26, by wenzelm
lambda/cabs/all: named variants;
2009-07-26, by wenzelm
Goal.finish: explicit context for printing;
2009-07-26, by wenzelm
fixed Method.Basic;
2009-07-25, by wenzelm
eliminated obsolete/obscure Seq.wrap, Position.setmp_thread_data_seq;
2009-07-25, by wenzelm
Method.Basic: no position;
2009-07-25, by wenzelm
basic method application: avoid Position.setmp_thread_data_seq, which destroys transaction context;
2009-07-25, by wenzelm
dequeue_towards: need to try imm_preds as well;
2009-07-25, by wenzelm
internal session timing;
2009-07-25, by wenzelm
enqueue: maintain transitive closure, which simplifies dequeue_towards;
2009-07-25, by wenzelm
ML_Context.the_generic_context;
2009-07-25, by wenzelm
eliminated redundant Library.multiply;
2009-07-25, by wenzelm
renamed structure Display_Goal to Goal_Display;
2009-07-25, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip