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.
simplified Session.Phase;
2010-09-23, by wenzelm
tuned messages -- cf. Admin/MacOS/App1;
2010-09-23, by wenzelm
tuned dialog;
2010-09-23, by wenzelm
explicit Session.Phase indication with associated event bus;
2010-09-23, by wenzelm
tuned signature;
2010-09-23, by wenzelm
Plugin.stop: refrain from invalidating Isabelle.session -- some actors/dockables out there might still refer to it;
2010-09-23, by wenzelm
tuned;
2010-09-23, by wenzelm
manage persistent syslog via Session, not Isabelle_Process;
2010-09-23, by wenzelm
tuned prover message categorization;
2010-09-23, by wenzelm
tuned Isabelle_Sidekick.complete: lock buffer, depend on document model;
2010-09-23, by wenzelm
tuned message;
2010-09-23, by wenzelm
Command.accumulate: refrain from adding tracing messages to markup tree -- potential scalability problem;
2010-09-22, by wenzelm
Snapshot.convert/revert: explicit error report to isolate sporadic crash;
2010-09-22, by wenzelm
make compiler doubly sure;
2010-09-22, by wenzelm
isabelle-process: less verbose no-commit mode;
2010-09-22, by wenzelm
tuned message;
2010-09-22, by wenzelm
tuned panel names and actions;
2010-09-22, by wenzelm
renamed setmp_noncritical to Unsynchronized.setmp to emphasize its meaning;
2010-09-22, by wenzelm
reactivated polyml-5.4.0 -- SVN 1214 fixes a problem with arbitrary precision arithmetic that was triggered by method "approximation" in HOL/Decision_Procs/Approximation_Ex.thy;
2010-09-22, by wenzelm
merged
2010-09-22, by nipkow
more lists lemmas
2010-09-22, by nipkow
merged
2010-09-22, by wenzelm
merged
2010-09-22, by haftmann
tuned text
2010-09-22, by haftmann
sections on @{code} and code_reflect
2010-09-22, by haftmann
formal syntax diagram for code_reflect
2010-09-22, by haftmann
distinguish SML and Eval explicitly
2010-09-22, by haftmann
no_frees_* is subsumed by new framework mechanisms in Code_Preproc
2010-09-21, by haftmann
reject term variables explicitly
2010-09-21, by haftmann
avoid frees and vars in terms to be evaluated by abstracting and applying
2010-09-21, by haftmann
tuned whitespace
2010-09-21, by haftmann
make SML/NJ happier
2010-09-22, by blanchet
more conventional conversion signature
2010-09-21, by haftmann
added nbe paper
2010-09-21, by haftmann
continued section abut evaluation
2010-09-21, by haftmann
make SML/NJ happier
2010-09-21, by blanchet
new lemma
2010-09-21, by nipkow
merged
2010-09-20, by nipkow
new lemmas
2010-09-20, by nipkow
revert b96941dddd04 and c13b4589fddf, which dramatically inflate proof terms
2010-09-20, by blanchet
basic setup for Session_Dockable controls;
2010-09-22, by wenzelm
tuned signature;
2010-09-22, by wenzelm
more content for Session_Dockable;
2010-09-22, by wenzelm
basic support for full document rendering;
2010-09-22, by wenzelm
Session_Dockable: basic syslog output;
2010-09-22, by wenzelm
just one Session.raw_messages event bus;
2010-09-22, by wenzelm
more reactive handling of Isabelle_Process startup errors;
2010-09-22, by wenzelm
eliminated Simple_Thread shorthands that can overlap with full version;
2010-09-22, by wenzelm
main Isabelle_Process via Isabelle_System.Managed_Process;
2010-09-22, by wenzelm
more robust Managed_Process.kill: check after sending signal;
2010-09-22, by wenzelm
more robust lib/scripts/process, with explicit script/no_script mode;
2010-09-22, by wenzelm
Standard_System.with_tmp_file: deleteOnExit to make double sure;
2010-09-22, by wenzelm
refined Isabelle_System.bash_output: pass pid via stdout, separate stdout/stderr;
2010-09-21, by wenzelm
tuned whitespace;
2010-09-21, by wenzelm
tuned;
2010-09-21, by wenzelm
added Standard_System.slurp convenience;
2010-09-21, by wenzelm
added Simple_Thread.future convenience;
2010-09-21, by wenzelm
refined ML/Scala bash wrapper, based on more general lib/scripts/process;
2010-09-20, by wenzelm
tuned;
2010-09-20, by wenzelm
more robust Isabelle_System.rm_fifo: avoid external bash invocation, which might not work in JVM shutdown phase (due to Runtime.addShutdownHook);
2010-09-20, by wenzelm
tuned;
2010-09-20, by wenzelm
added Isabelle_Process.syslog;
2010-09-20, by wenzelm
updated keywords;
2010-09-20, by wenzelm
merged
2010-09-20, by wenzelm
merged
2010-09-20, by haftmann
corrected long-overlooked slip: the Pure equality of a code equation is no part of the code equation itself
2010-09-20, by haftmann
dynamic_eval_conv static_eval_conv: certification of previously unreliably reconstructed evaluated term
2010-09-20, by haftmann
Pure equality is a regular cpde operation
2010-09-20, by haftmann
full palette of dynamic/static value(_strict/exn)
2010-09-20, by haftmann
Factored out ML into separate file
2010-09-20, by haftmann
merged
2010-09-20, by wenzelm
merged
2010-09-20, by blanchet
remove needless exception
2010-09-20, by blanchet
preprocess "Ex" before doing clausification in Metis;
2010-09-20, by blanchet
expand_fun_eq -> fun_eq_iff
2010-09-20, by haftmann
use buffers instead of string concatenation
2010-09-20, by haftmann
renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
2010-09-20, by wenzelm
more antiquotations;
2010-09-20, by wenzelm
added XML.content_of convenience -- cover XML.body, which is the general situation;
2010-09-20, by wenzelm
merged
2010-09-20, by wenzelm
merged
2010-09-20, by haftmann
more accurate exception handling
2010-09-20, by haftmann
merged
2010-09-20, by blanchet
merge tracing of two related modules
2010-09-20, by blanchet
merged
2010-09-20, by blanchet
preprocess "All" before doing clausification in Metis;
2010-09-18, by blanchet
reorder proof methods and take out "best";
2010-09-17, by blanchet
renaming variable name to decrease likelyhood of nameclash
2010-09-20, by bulwahn
code_pred_intro can be used to name facts for the code_pred command
2010-09-20, by bulwahn
replacing temporary hack by checking for environment settings of the component
2010-09-20, by bulwahn
removing unnessary options for code_pred
2010-09-20, by bulwahn
moving renaming_vars to post_processing; removing clone in values and quickcheck of code_prolog
2010-09-20, by bulwahn
removing clone in code_prolog and predicate_compile_quickcheck
2010-09-20, by bulwahn
adjusted
2010-09-20, by haftmann
updated file duplicate
2010-09-20, by haftmann
\\isatypewrite now part of isabelle latex style
2010-09-20, by haftmann
made smlnj happy
2010-09-20, by haftmann
properly parse Z3 error models, including datatypes, and represent function valuations as lambda terms; also normalize Z3 error models
2010-09-19, by boehmes
do not treat natural numbers as a datatype (natural numbers are considered an abstract type with a coercion to integers)
2010-09-19, by boehmes
generalized lemma insort_remove1 to insort_key_remove1
2010-09-17, by haftmann
generalized lemmas multiset_of_insort, multiset_of_sort, properties_for_sort for *_key variants
2010-09-17, by haftmann
merged
2010-09-17, by haftmann
less intermediate data structures
2010-09-17, by haftmann
Isabelle_Process: more robust rendezvous, even without proper blocking on open (Cygwin);
2010-09-20, by wenzelm
simplified Isabelle_System.mk_fifo: inlined script, append PPID and PID uniformly;
2010-09-19, by wenzelm
refined Isabelle_Process startup: emit \002 before rendezvous on fifos, more robust treatment of startup failure with timeout, do not quit() after main loop;
2010-09-19, by wenzelm
back to default fold painter -- Circle looks slightly odd in conjunction with bracket matching;
2010-09-19, by wenzelm
message_actor: more robust treatment of EOF;
2010-09-19, by wenzelm
simplified Isabelle_Process message kinds;
2010-09-19, by wenzelm
recovered basic session stop/restart;
2010-09-18, by wenzelm
simplified fifo handling -- rm_fifo always succeeds without ever blocking;
2010-09-18, by wenzelm
raw_execute: let IOException pass-through unhindered (again);
2010-09-18, by wenzelm
mkfifo: some workaround to ensure reasonably unique id, even on Cygwin where $PPID might fall back on odd default;
2010-09-18, by wenzelm
Isabelle_System.mk_fifo: more robust enumeration of unique names, based on persisting JVM pid (parent of shell process);
2010-09-18, by wenzelm
slightly more robust Isabelle_Process startup -- NB: openening fifo streams synchronizes with other end, which may fail to reach that point;
2010-09-18, by wenzelm
tuned;
2010-09-18, by wenzelm
separate Isabelle.logic_selector;
2010-09-18, by wenzelm
non-editable text area;
2010-09-18, by wenzelm
basic setup for prover session panel;
2010-09-18, by wenzelm
ML_Syntax.print_char: more readable output of some well-known ASCII controls -- this is relevant for ML toplevel pp;
2010-09-17, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip