paulson [Tue, 09 Sep 2008 16:16:20 +0200] rev 28174
more careful exception handling in order to prevent backtracking; miscellaneous tidying up.
paulson [Tue, 09 Sep 2008 16:15:25 +0200] rev 28173
Increasing the default limits in order to prevent unnecessary failures.
wenzelm [Mon, 08 Sep 2008 22:14:39 +0200] rev 28172
send: broadcast condition while locked!
wenzelm [Mon, 08 Sep 2008 21:08:30 +0200] rev 28171
proper signature constraint;
wenzelm [Mon, 08 Sep 2008 20:35:38 +0200] rev 28170
tuned Mailbox.send;
wenzelm [Mon, 08 Sep 2008 20:33:29 +0200] rev 28169
removed unused sync_interrupts;
wenzelm [Mon, 08 Sep 2008 20:33:27 +0200] rev 28168
moved thread data to future.ML (again);
dequeue: include group;
more interrupt operations;
misc tuning;
wenzelm [Mon, 08 Sep 2008 20:33:24 +0200] rev 28167
more interrupt operations;
maintain thread data (formerly in task_queue.ML);
wait: added tracing;
added requests mailbox;
handle excessive workers
fork: inherit group;
added rudimentary shutdown;
misc tuning;
wenzelm [Mon, 08 Sep 2008 16:08:23 +0200] rev 28166
moved task, thread_data, group, queue to task_queue.ML;
tuned signature;
SYNCHRONIZED notify_all!
misc tuning;
wenzelm [Mon, 08 Sep 2008 16:08:18 +0200] rev 28165
Ordered queue of grouped tasks.
formerly in future.ML;
added thread data;
added group;
more robust dequeue: change into running here;
misc tuning;
wenzelm [Mon, 08 Sep 2008 16:08:13 +0200] rev 28164
added Concurrent/task_queue.ML;
wenzelm [Mon, 08 Sep 2008 00:25:34 +0200] rev 28163
await: SYNCHRONIZED wait!
wenzelm [Mon, 08 Sep 2008 00:10:41 +0200] rev 28162
tuned check_cache;
removed broken self_synchronized, which cannot be used in conjunction with condition variables;
more precise use of SYNCHRONIZED vs. wait;
tuned worker_loop;
wenzelm [Sun, 07 Sep 2008 22:20:15 +0200] rev 28161
added sync_interrupts, regular_interrupts;
max_thread_value: enforce >= 1;
wenzelm [Sun, 07 Sep 2008 22:20:11 +0200] rev 28160
added sync_interrupts, regular_interrupts;
wenzelm [Sun, 07 Sep 2008 22:20:08 +0200] rev 28159
opaque signature constraint abstracts local type abbrev;
wenzelm [Sun, 07 Sep 2008 22:19:58 +0200] rev 28158
tuned;
wenzelm [Sun, 07 Sep 2008 22:19:46 +0200] rev 28157
added change_result;
wenzelm [Sun, 07 Sep 2008 22:19:42 +0200] rev 28156
Functional threads as future values.
wenzelm [Sun, 07 Sep 2008 22:19:31 +0200] rev 28155
added Concurrent/future.ML;
wenzelm [Sun, 07 Sep 2008 17:48:50 +0200] rev 28154
Default (mostly dummy) implementation of thread structures.
formerly in multithreading.ML;
create mutexes / condition variables without failure;
wenzelm [Sun, 07 Sep 2008 17:48:49 +0200] rev 28153
*** MESSAGE REFERS TO PREVIOUS VERSION ***
removed dummy thread structures from multithreading.ML;
wenzelm [Sun, 07 Sep 2008 17:46:44 +0200] rev 28152
*** empty log message ***
wenzelm [Sun, 07 Sep 2008 17:46:43 +0200] rev 28151
explicit use of universal.ML and dummy_thread.ML;
wenzelm [Sun, 07 Sep 2008 17:46:41 +0200] rev 28150
added no_interrupts;
tuned;
wenzelm [Sun, 07 Sep 2008 17:46:40 +0200] rev 28149
added no_interrupts;
moved dummy thread structures to dummy_thread.ML;
wenzelm [Sun, 07 Sep 2008 17:46:39 +0200] rev 28148
tuned;
wenzelm [Sun, 07 Sep 2008 17:46:38 +0200] rev 28147
send: broadcast to all waiting threads;
wenzelm [Sun, 07 Sep 2008 17:46:37 +0200] rev 28146
added ML-Systems/thread_dummy.ML;
haftmann [Sat, 06 Sep 2008 14:02:36 +0200] rev 28145
dropped "run" marker in monad syntax
wenzelm [Fri, 05 Sep 2008 11:50:35 +0200] rev 28144
multithreading.ML provides dummy thread structures;
haftmann [Fri, 05 Sep 2008 06:50:22 +0200] rev 28143
different bookkeeping for code equations
haftmann [Fri, 05 Sep 2008 06:50:20 +0200] rev 28142
renamed structure CodeTarget to Code_Target
huffman [Fri, 05 Sep 2008 00:19:50 +0200] rev 28141
instances comm_semiring_0_cancel < comm_semiring_0, comm_ring < comm_semiring_0_cancel
wenzelm [Thu, 04 Sep 2008 21:12:06 +0200] rev 28140
proper header;
wenzelm [Thu, 04 Sep 2008 21:02:42 +0200] rev 28139
added receive_timeout;
tuned comments;
wenzelm [Thu, 04 Sep 2008 20:06:23 +0200] rev 28138
check WRAPPER_OUTPUT node type;
wenzelm [Thu, 04 Sep 2008 20:05:48 +0200] rev 28137
init: disallow "" as out stream;
wenzelm [Thu, 04 Sep 2008 19:47:13 +0200] rev 28136
fixed deps: no Concurrent/receiver.ML yet;
wenzelm [Thu, 04 Sep 2008 19:45:13 +0200] rev 28135
Concurrent message exchange via mailbox -- with unbounded queueing.
wenzelm [Thu, 04 Sep 2008 19:45:12 +0200] rev 28134
added Concurrent/mailbox.ML;
huffman [Thu, 04 Sep 2008 17:24:18 +0200] rev 28133
reorganize subsections
huffman [Thu, 04 Sep 2008 17:21:49 +0200] rev 28132
rename INF_drop_prefix to INFM_drop_prefix
huffman [Thu, 04 Sep 2008 17:19:57 +0200] rev 28131
add lemma power_Suc2; generalize power_minus from class comm_ring_1 to ring_1
huffman [Thu, 04 Sep 2008 17:18:44 +0200] rev 28130
move diff_add_cancel, add_diff_cancel from class ab_group_add to group_add
wenzelm [Thu, 04 Sep 2008 16:43:51 +0200] rev 28129
tuned signature;
wenzelm [Thu, 04 Sep 2008 16:43:50 +0200] rev 28128
added General/queue.ML;
wenzelm [Thu, 04 Sep 2008 16:43:48 +0200] rev 28127
Efficient queues.
wenzelm [Thu, 04 Sep 2008 16:03:49 +0200] rev 28126
moved Multithreading.task/schedule to Concurrent/schedule.ML
wenzelm [Thu, 04 Sep 2008 16:03:48 +0200] rev 28125
multithreading.ML provides dummy thread structures;
wenzelm [Thu, 04 Sep 2008 16:03:47 +0200] rev 28124
moved Multithreading.task/schedule to Concurrent/schedule.ML;
wenzelm [Thu, 04 Sep 2008 16:03:46 +0200] rev 28123
provide dummy thread structures, including proper Thread.getLocal/setLocal;
moved task/schedule to Concurrent/schedule.ML;
wenzelm [Thu, 04 Sep 2008 16:03:44 +0200] rev 28122
Thread.getLocal/setLocal;
wenzelm [Thu, 04 Sep 2008 16:03:43 +0200] rev 28121
Scheduling -- multiple threads working on a queue of tasks.
formerly in ML-Systems/multithreading_polyml.ML;
simplified -- less tracing;
use regular Isabelle/ML functions instead of NJ stuff;
wenzelm [Thu, 04 Sep 2008 16:03:41 +0200] rev 28120
added Concurrent/schedule.ML;
convert-repo [Wed, 03 Sep 2008 20:32:33 +0000] rev 28119
update tags
wenzelm [Wed, 03 Sep 2008 20:04:54 +0200] rev 28118
use /home/isabelle/mercurial/bin/hg wrapper;
wenzelm [Wed, 03 Sep 2008 19:52:45 +0200] rev 28117
exclude large .mov files;
wenzelm [Wed, 03 Sep 2008 17:50:37 +0200] rev 28116
simplified add_axiom: no hyps;
wenzelm [Wed, 03 Sep 2008 17:47:40 +0200] rev 28115
discontinued local axioms -- too difficult to implement, too easy to produce nonsense;
wenzelm [Wed, 03 Sep 2008 17:47:38 +0200] rev 28114
axiomatization is now global-only;
wenzelm [Wed, 03 Sep 2008 17:47:37 +0200] rev 28113
added const_decl;
wenzelm [Wed, 03 Sep 2008 17:47:35 +0200] rev 28112
simplified specify_const: canonical args, global deps;
wenzelm [Wed, 03 Sep 2008 17:47:34 +0200] rev 28111
declare_const: Name.binding, store/report position;
wenzelm [Wed, 03 Sep 2008 17:47:30 +0200] rev 28110
Sign.declare_const: Name.binding;
nipkow [Wed, 03 Sep 2008 12:11:28 +0200] rev 28109
removed ex/Puzzle
wenzelm [Wed, 03 Sep 2008 11:44:52 +0200] rev 28108
added qualified: string -> binding -> binding;
wenzelm [Wed, 03 Sep 2008 11:44:48 +0200] rev 28107
Name.qualified;
wenzelm [Wed, 03 Sep 2008 11:27:15 +0200] rev 28106
theorem dependency hook: check previous state;
wenzelm [Wed, 03 Sep 2008 11:26:59 +0200] rev 28105
added pos_of;
nipkow [Wed, 03 Sep 2008 11:18:55 +0200] rev 28104
-> AFP
wenzelm [Wed, 03 Sep 2008 11:09:08 +0200] rev 28103
simplified Toplevel.add_hook: cover successful transactions only;
kleing [Wed, 03 Sep 2008 00:11:27 +0200] rev 28102
retired Ben Porter's DenumRat in favour of the shorter proof in
Real/Rational.thy
wenzelm [Tue, 02 Sep 2008 23:52:51 +0200] rev 28101
made SML/NJ happy;
wenzelm [Tue, 02 Sep 2008 23:27:44 +0200] rev 28100
refined theorem dependency output: previous state needs to contain a theory (not empty toplevel);
new_thms_deps: explicity theory values;
wenzelm [Tue, 02 Sep 2008 22:41:36 +0200] rev 28099
* Generic Toplevel.add_hook interface allows to analyze the result of
transactions (including failed ones). For example, see
src/Pure/ProofGeneral/proof_general_pgip.ML for theorem dependency
output of transactions resulting in a new theory state.
nipkow [Tue, 02 Sep 2008 22:37:20 +0200] rev 28098
Replaced Library/NatPair by Nat_Int_Bij.
wenzelm [Tue, 02 Sep 2008 22:20:27 +0200] rev 28097
added new_thms_deps (operates on global facts, some name_hint approximation);
theorem dependency output: Toplevel.add_hook, ProofGeneralPgip.new_thms_deps;
wenzelm [Tue, 02 Sep 2008 22:20:25 +0200] rev 28096
theorem dependency output: Toplevel.add_hook, ProofGeneralPgip.new_thms_deps;
wenzelm [Tue, 02 Sep 2008 22:20:24 +0200] rev 28095
added add_hook interface for post-transition hooks;
wenzelm [Tue, 02 Sep 2008 22:20:21 +0200] rev 28094
tuned;
wenzelm [Tue, 02 Sep 2008 22:20:20 +0200] rev 28093
ProofDisplay.print_results;
wenzelm [Tue, 02 Sep 2008 22:20:16 +0200] rev 28092
no pervasive bindings;
removed theory_results and related hook;
print_results: ignore empty/internal kind -- like former theory_results;
nipkow [Tue, 02 Sep 2008 21:31:28 +0200] rev 28091
Streamlined parts of Complex/ex/DenumRat and AFP/Integration/Rats and
distributed them over Real/ (to do with bijections and density).
Library/NatPair became Nat_Int_Bij and made that part of Main.
haftmann [Tue, 02 Sep 2008 20:38:17 +0200] rev 28090
distributed literal code generation out of central infrastructure
wenzelm [Tue, 02 Sep 2008 20:07:51 +0200] rev 28089
* Result facts now refer to the *full* internal name;
wenzelm [Tue, 02 Sep 2008 20:04:26 +0200] rev 28088
* Name bindings in higher specification mechanisms;
wenzelm [Tue, 02 Sep 2008 18:01:24 +0200] rev 28087
pretty_fact/results: display base only, since results now come with full names (note that Facts.extern is not really well-defined unless we present the real target context);
wenzelm [Tue, 02 Sep 2008 18:01:23 +0200] rev 28086
updated generated file;
ballarin [Tue, 02 Sep 2008 17:31:20 +0200] rev 28085
Interpretation commands no longer accept interpretation attributes.
wenzelm [Tue, 02 Sep 2008 16:55:33 +0200] rev 28084
type Attrib.binding abbreviates Name.binding without attributes;
Attrib.no_binding refers to Name.no_binding;
wenzelm [Tue, 02 Sep 2008 14:10:45 +0200] rev 28083
explicit type Name.binding for higher-specification elements;
wenzelm [Tue, 02 Sep 2008 14:10:32 +0200] rev 28082
explicit type Name.binding for higher-specification elements;
report local_fact_decl, fixed_decl;
simplified ProofContext.inferred_param;
wenzelm [Tue, 02 Sep 2008 14:10:31 +0200] rev 28081
explicit type Name.binding for higher-specification elements;
added binding, parbinding;
wenzelm [Tue, 02 Sep 2008 14:10:30 +0200] rev 28080
explicit type Name.binding for higher-specification elements;
simplified ProofContext.inferred_param;
wenzelm [Tue, 02 Sep 2008 14:10:29 +0200] rev 28079
explicit type Name.binding for higher-specification elements;
name/var morphism operates on Name.binding;
wenzelm [Tue, 02 Sep 2008 14:10:28 +0200] rev 28078
added binding;
thm_name/opt_thm_name: Name.binding;
wenzelm [Tue, 02 Sep 2008 14:10:27 +0200] rev 28077
added fixed_decl, fact_decl, local_fact_decl;
wenzelm [Tue, 02 Sep 2008 14:10:25 +0200] rev 28076
name_thm etc.: pass position;
note_thms etc.: Name.binding, report fact_decl;
wenzelm [Tue, 02 Sep 2008 14:10:24 +0200] rev 28075
added type binding -- generic name bindings;
wenzelm [Tue, 02 Sep 2008 14:10:19 +0200] rev 28074
name/var morphism operates on Name.binding;
haftmann [Tue, 02 Sep 2008 12:07:34 +0200] rev 28073
adapted to class instantiation compliance
nipkow [Mon, 01 Sep 2008 22:10:42 +0200] rev 28072
It appears that the code generator (Stefan's) needs some laws that appear superfluous: {..n} = set ...
nipkow [Mon, 01 Sep 2008 19:17:47 +0200] rev 28071
renamed lemma
nipkow [Mon, 01 Sep 2008 19:17:37 +0200] rev 28070
moved more lemmas here from AFP/Integration/Rats
nipkow [Mon, 01 Sep 2008 19:17:04 +0200] rev 28069
moved lemma into SetInterval where it belongs
nipkow [Mon, 01 Sep 2008 19:16:40 +0200] rev 28068
cleaned up code generation for {.._} and {..<_}
moved lemmas into SetInterval where they belong
nipkow [Mon, 01 Sep 2008 10:28:04 +0200] rev 28067
*** empty log message ***
nipkow [Mon, 01 Sep 2008 10:20:14 +0200] rev 28066
extended interface to preferences to allow adding new ones
nipkow [Mon, 01 Sep 2008 10:19:38 +0200] rev 28065
Prover is set via menu now
haftmann [Mon, 01 Sep 2008 10:18:37 +0200] rev 28064
restructured code generation of literals
wenzelm [Fri, 29 Aug 2008 20:36:08 +0200] rev 28063
IsabelleSystem.mk_fifo, IsabelleSystem.rm_fifo;
IsabelleSystem.exec: varargs convenience;
more robust message thread management: no interrupt, but proper rendezvous via fifo (rm_fifo removes unused fifo, if isabelle-process fails);
wenzelm [Fri, 29 Aug 2008 20:36:07 +0200] rev 28062
init: more explicit protocol of open/remove rendezvous;
wenzelm [Fri, 29 Aug 2008 20:36:05 +0200] rev 28061
use hardwired /tmp -- fifo only work on local file-system;
haftmann [Fri, 29 Aug 2008 08:14:59 +0200] rev 28060
separate module for code output
haftmann [Fri, 29 Aug 2008 08:14:58 +0200] rev 28059
fixed names of class assumptions
haftmann [Fri, 29 Aug 2008 07:43:25 +0200] rev 28058
dropped parameter prefix for class theorems
wenzelm [Thu, 28 Aug 2008 22:26:23 +0200] rev 28057
added charset (from isabelle_process.scala);
added fifo_reader -- also works on Cygwin;
wenzelm [Thu, 28 Aug 2008 22:26:22 +0200] rev 28056
moved charset to isabelle_system.scala;
IsabelleSystem.fifo_reader;
wenzelm [Thu, 28 Aug 2008 22:26:21 +0200] rev 28055
provide HOME_JVM=HOME to prevent implicit cygpath mangling;
haftmann [Thu, 28 Aug 2008 22:09:20 +0200] rev 28054
restructured and split code serializer module
haftmann [Thu, 28 Aug 2008 22:08:11 +0200] rev 28053
no parameter prefix for class interpretation
haftmann [Thu, 28 Aug 2008 22:08:02 +0200] rev 28052
updated
wenzelm [Thu, 28 Aug 2008 20:29:40 +0200] rev 28051
tuned fold_lines;
wenzelm [Thu, 28 Aug 2008 20:19:45 +0200] rev 28050
fold_lines: simplified, more efficient due to String.fields;
wenzelm [Thu, 28 Aug 2008 19:34:51 +0200] rev 28049
rm fifo after open;
wenzelm [Thu, 28 Aug 2008 19:31:55 +0200] rev 28048
dummy setup for completion;
wenzelm [Thu, 28 Aug 2008 19:31:13 +0200] rev 28047
create named pipe;
wenzelm [Thu, 28 Aug 2008 19:29:59 +0200] rev 28046
added is_cygwin;
added exec2, which joins stdout/stderr;
tuned thread arrangement;
wenzelm [Thu, 28 Aug 2008 19:29:58 +0200] rev 28045
join stdout/stderr, eliminated Kind.STDERR;
messages are read from separate fifo (ensures that spurious stdout from shell wrappers, Poly/ML runtime system etc. do not spoil message protocol);
private output, output_raw;
wenzelm [Thu, 28 Aug 2008 19:29:57 +0200] rev 28044
explicit output stream, typically a named pipe;
wenzelm [Thu, 28 Aug 2008 19:29:56 +0200] rev 28043
refined option -W: output stream;
krauss [Thu, 28 Aug 2008 17:54:18 +0200] rev 28042
more function -> fun
krauss [Thu, 28 Aug 2008 15:33:33 +0200] rev 28041
quicksort: function -> fun
krauss [Thu, 28 Aug 2008 15:24:30 +0200] rev 28040
corrected some typos
wenzelm [Thu, 28 Aug 2008 00:49:54 +0200] rev 28039
fixed atom_to_xml: literal "name" attribute;
wenzelm [Thu, 28 Aug 2008 00:33:19 +0200] rev 28038
exported atom_to_xml;
wenzelm [Thu, 28 Aug 2008 00:33:17 +0200] rev 28037
changed Markup print mode to YXML -- explicitly decode messages before being issued;
changed Output print mode to plain default -- no escaping;
simplified pgml_sym: produce Pgml.pgmlatom, no special treatment of Ctrl/Raw;
removed unused issue_pgips;
removed obsolete delay_msgs feature -- the script parser never fails, but produces inline error markup;
removed obsolete wrap_pgml;
explicit transformation of messages (pgml_terms and message_content);
remove obsolete split_markup workaround;
misc tuning;
wenzelm [Thu, 28 Aug 2008 00:33:15 +0200] rev 28036
tuned;
wenzelm [Thu, 28 Aug 2008 00:33:13 +0200] rev 28035
present_token: disable print_mode, which is YXML now;
wenzelm [Thu, 28 Aug 2008 00:33:11 +0200] rev 28034
text_of Malformed: explode with spaces -- Output.output/escape ineffective by default;
wenzelm [Thu, 28 Aug 2008 00:33:09 +0200] rev 28033
removed obsolete XML.Output workaround;
wenzelm [Thu, 28 Aug 2008 00:33:08 +0200] rev 28032
added get_int;
wenzelm [Thu, 28 Aug 2008 00:33:07 +0200] rev 28031
removed obsolete get_string;
moved get_int to property.ML;
wenzelm [Thu, 28 Aug 2008 00:33:04 +0200] rev 28030
removed obsolete ProofGeneral/pgml_isabelle.ML;
huffman [Wed, 27 Aug 2008 23:46:33 +0200] rev 28029
simplify definition of vector_space locale (use axclasses instead of inheriting from field and ab_group_add classes)
wenzelm [Wed, 27 Aug 2008 20:36:27 +0200] rev 28028
renamed Buffer.write to File.write_buffer;
added scalable iterator fold_lines;
tuned;
wenzelm [Wed, 27 Aug 2008 20:36:26 +0200] rev 28027
renamed Buffer.write to File.write_buffer;
wenzelm [Wed, 27 Aug 2008 20:36:25 +0200] rev 28026
load buffer.ML before file.ML;
wenzelm [Wed, 27 Aug 2008 20:36:23 +0200] rev 28025
replaced find_substring by first_field;
ballarin [Wed, 27 Aug 2008 17:54:31 +0200] rev 28024
Consistent naming of theorems in interpretation.
wenzelm [Wed, 27 Aug 2008 16:32:48 +0200] rev 28023
simplified parse_attrib (find_substring instead of space_explode);
wenzelm [Wed, 27 Aug 2008 16:32:18 +0200] rev 28022
added find_substring;
haftmann [Wed, 27 Aug 2008 12:01:59 +0200] rev 28021
added HOL/ex/Numeral.thy
wenzelm [Wed, 27 Aug 2008 12:00:28 +0200] rev 28020
get rid of tabs;
wenzelm [Wed, 27 Aug 2008 11:49:50 +0200] rev 28019
Property lists.
wenzelm [Wed, 27 Aug 2008 11:49:14 +0200] rev 28018
added General/properties.ML;
wenzelm [Wed, 27 Aug 2008 11:48:54 +0200] rev 28017
type Properties.T;
haftmann [Wed, 27 Aug 2008 11:24:35 +0200] rev 28016
proper error message
haftmann [Wed, 27 Aug 2008 11:24:34 +0200] rev 28015
proper handling of type variabl names
haftmann [Wed, 27 Aug 2008 11:24:32 +0200] rev 28014
completing arities after subclass instance
haftmann [Wed, 27 Aug 2008 11:24:31 +0200] rev 28013
untabification
haftmann [Wed, 27 Aug 2008 11:24:29 +0200] rev 28012
tuned code generator setup
urbanc [Wed, 27 Aug 2008 04:47:30 +0200] rev 28011
added equivariance lemmas for ex1 and the
huffman [Wed, 27 Aug 2008 01:27:33 +0200] rev 28010
add lemmas about Rats similar to those about Reals
huffman [Tue, 26 Aug 2008 23:49:46 +0200] rev 28009
move real_vector class proofs into vector_space and group_hom locales
krauss [Tue, 26 Aug 2008 18:59:52 +0200] rev 28008
added distributivity of relation composition over union [simp]
wenzelm [Tue, 26 Aug 2008 16:36:30 +0200] rev 28007
tuned append;
wenzelm [Tue, 26 Aug 2008 16:36:11 +0200] rev 28006
command: symbols.encode;
ballarin [Tue, 26 Aug 2008 16:04:22 +0200] rev 28005
Reorganisation of registration code.
krauss [Tue, 26 Aug 2008 14:15:44 +0200] rev 28004
function package: name primitive defs "f_sumC_def" instead of "f_sum_def" to avoid clashes
wenzelm [Tue, 26 Aug 2008 12:20:52 +0200] rev 28003
purge classes after compilation;
wenzelm [Tue, 26 Aug 2008 12:17:58 +0200] rev 28002
renamed Isabelle-repository to isabelle;
nipkow [Tue, 26 Aug 2008 12:07:06 +0200] rev 28001
Defined rationals (Rats) globally in Rational.
Chractarized them with a few lemmas in RealDef, one of them from Sqrt.
wenzelm [Tue, 26 Aug 2008 11:42:46 +0200] rev 28000
replaced /home/isabelle/html-data/isabelle-repos by /home/isabelle-repository/repos;
wenzelm [Mon, 25 Aug 2008 23:27:56 +0200] rev 27999
moved new Symbol.Interpretation into plugin;
wenzelm [Mon, 25 Aug 2008 22:42:04 +0200] rev 27998
promoted to EBPlugin;
tuned;
wenzelm [Mon, 25 Aug 2008 22:26:26 +0200] rev 27997
explicitly depend on isabelle-Pure.jar and isabelle-scala-library.jar;
wenzelm [Mon, 25 Aug 2008 22:05:30 +0200] rev 27996
tuned;
wenzelm [Mon, 25 Aug 2008 21:59:36 +0200] rev 27995
isabelle process: pick options/args from properties;
wenzelm [Mon, 25 Aug 2008 21:58:54 +0200] rev 27994
removed unused ConsolePlugin dependency;
added menu item;
added some Isabelle options;
wenzelm [Mon, 25 Aug 2008 20:01:17 +0200] rev 27993
simplified exceptions: use plain error function / RuntimeException;
wenzelm [Mon, 25 Aug 2008 16:52:11 +0200] rev 27992
added try_result;
wenzelm [Sun, 24 Aug 2008 21:15:48 +0200] rev 27991
misc reorganization;
simplified consumer thread;
more robust stop;
wenzelm [Sun, 24 Aug 2008 21:15:46 +0200] rev 27990
Kind: added is_control;
more robust kill/exit;
tuned interfaces;
wenzelm [Sun, 24 Aug 2008 21:15:44 +0200] rev 27989
get: allow null;
wenzelm [Sun, 24 Aug 2008 19:24:27 +0200] rev 27988
misc tuning of names;
wenzelm [Sun, 24 Aug 2008 19:02:22 +0200] rev 27987
rearranged source files;
wenzelm [Sun, 24 Aug 2008 18:57:43 +0200] rev 27986
init_message: class markup in message body, not header;
wenzelm [Sun, 24 Aug 2008 18:11:20 +0200] rev 27985
repackaged as isabelle.jedit;
wenzelm [Sun, 24 Aug 2008 17:23:42 +0200] rev 27984
untabify: silently turn tab into space if column information is unavailable;
haftmann [Sun, 24 Aug 2008 14:42:26 +0200] rev 27983
corrected cache handling for class operations
haftmann [Sun, 24 Aug 2008 14:42:24 +0200] rev 27982
default replaces arbitrary
haftmann [Sun, 24 Aug 2008 14:42:22 +0200] rev 27981
tuned import order
wenzelm [Sun, 24 Aug 2008 14:24:03 +0200] rev 27980
activated \<A>, \<a>, \<AA>, \<aa>;
disabled \<RR>, \<II> which overlap with codepoints for \<Re>, \<Im>, remapped to unofficial place within Isabelle font;
wenzelm [Sat, 23 Aug 2008 23:44:31 +0200] rev 27979
* Isabelle/lib/classes/Pure.jar;
* Status messages;
* Homegrown Isabelle font;
wenzelm [Sat, 23 Aug 2008 23:24:16 +0200] rev 27978
jars: removed obsolete Java process wrapper (cf. new Pure.jar);
wenzelm [Sat, 23 Aug 2008 23:21:50 +0200] rev 27977
obsolete;
wenzelm [Sat, 23 Aug 2008 23:20:43 +0200] rev 27976
obsolete -- superceded by Pure.jar (Scala version);
wenzelm [Sat, 23 Aug 2008 23:17:11 +0200] rev 27975
updated to Pure.jar;
wenzelm [Sat, 23 Aug 2008 23:07:46 +0200] rev 27974
added exec;
private posix_prefix;
wenzelm [Sat, 23 Aug 2008 23:07:44 +0200] rev 27973
moved class Result into static object, removed dynamic tree method;
removed unused Symbol.Interpretation;
class Result: added is_raw, is_system;
disabled console echo;
added interrupt, kill;
IsabelleSystem.exec;
wenzelm [Sat, 23 Aug 2008 23:07:43 +0200] rev 27972
symbolic message markup;
init message: class property;
wenzelm [Sat, 23 Aug 2008 23:07:41 +0200] rev 27971
renamed Markup.MALFORMED to Markup.BAD;
wenzelm [Sat, 23 Aug 2008 23:07:39 +0200] rev 27970
added position, messages;
renamed messages to content, malformed to bad;
wenzelm [Sat, 23 Aug 2008 23:07:38 +0200] rev 27969
added messages and process information;
wenzelm [Sat, 23 Aug 2008 23:07:36 +0200] rev 27968
Position properties.
wenzelm [Sat, 23 Aug 2008 23:07:34 +0200] rev 27967
added General/position.scala;
wenzelm [Sat, 23 Aug 2008 23:07:30 +0200] rev 27966
adapted to new IsabelleProcess from Pure.jar;
IsabellePlugin.result_content decodes symbols;
wenzelm [Sat, 23 Aug 2008 23:07:28 +0200] rev 27965
include ../../classes/Pure.jar;
nipkow [Sat, 23 Aug 2008 21:06:32 +0200] rev 27964
added const Rational
added more function puzzles
wenzelm [Sat, 23 Aug 2008 19:42:17 +0200] rev 27963
YXML.parse_failsafe;
removed full_markup, YXML mode (default);
renamed output_command to command;
renamed output_ML to ML;
tuned;
wenzelm [Sat, 23 Aug 2008 19:42:16 +0200] rev 27962
shell_prefix: physical /bin/env on Cygwin;
wenzelm [Sat, 23 Aug 2008 19:42:15 +0200] rev 27961
removed full_markup mode (default);
removed YXML mode (default);
added XML mode;
message: class attribute, fail for malformed YXML;
wenzelm [Sat, 23 Aug 2008 19:42:14 +0200] rev 27960
added parse_failsafe;
wenzelm [Sat, 23 Aug 2008 19:42:13 +0200] rev 27959
refer to symbolic Markup;
wenzelm [Sat, 23 Aug 2008 19:42:12 +0200] rev 27958
Common markup elements.
wenzelm [Sat, 23 Aug 2008 19:42:11 +0200] rev 27957
added General/markup.scala;
wenzelm [Sat, 23 Aug 2008 17:55:27 +0200] rev 27956
BadVariable: toString;
wenzelm [Sat, 23 Aug 2008 17:55:26 +0200] rev 27955
use java.util.concurrent.LinkedBlockingQueue, which blocks as required;
IsabelleProcessException: toString;
Result: improved toString;
Result: raw markup for stdout/stderr;
cmdline: proper executable name, added YXML mode;
wenzelm [Sat, 23 Aug 2008 17:55:26 +0200] rev 27954
append_string: proper backslash in character escapes;
wenzelm [Sat, 23 Aug 2008 17:22:54 +0200] rev 27953
added getenv;
renamed get_setting to getenv_strict;
added shell_prefix (for Cygwin);
wenzelm [Sat, 23 Aug 2008 17:22:53 +0200] rev 27952
tuned;
wenzelm [Sat, 23 Aug 2008 17:22:52 +0200] rev 27951
Isabelle outer syntax.
wenzelm [Sat, 23 Aug 2008 17:22:51 +0200] rev 27950
added Tools/isabelle_process.scala, Tools/isabelle_syntax.scala;
scalac -deprecation;
wenzelm [Sat, 23 Aug 2008 17:22:51 +0200] rev 27949
Isabelle process management -- always reactive due to multi-threaded I/O.
wenzelm [Sat, 23 Aug 2008 11:48:52 +0200] rev 27948
renamed DOM to document, add xml version and optional stylesheets;
wenzelm [Fri, 22 Aug 2008 21:25:19 +0200] rev 27947
tuned comments;
added document object model (DOM);
wenzelm [Thu, 21 Aug 2008 22:06:17 +0200] rev 27946
parse_attrib: proper index of name end!
wenzelm [Thu, 21 Aug 2008 21:42:16 +0200] rev 27945
tuned parse performance: avoid splitting terminal Y chunk;
wenzelm [Thu, 21 Aug 2008 21:27:07 +0200] rev 27944
parse_attrib: more efficient due to indexOf('=');
wenzelm [Thu, 21 Aug 2008 20:53:31 +0200] rev 27943
replaced Pattern.split by chunks iterator (more efficient, resembles ML version more closely);
wenzelm [Thu, 21 Aug 2008 20:51:41 +0200] rev 27942
tuned comment;
wenzelm [Thu, 21 Aug 2008 19:19:31 +0200] rev 27941
added iterator over content;
wenzelm [Thu, 21 Aug 2008 17:42:59 +0200] rev 27940
proper ISABELLE_ROOT_JVM on Cygwin;
wenzelm [Thu, 21 Aug 2008 16:02:54 +0200] rev 27939
pattern: proper "." not "[.]"!
tuned;
wenzelm [Thu, 21 Aug 2008 15:27:28 +0200] rev 27938
recode: proper result for unmatched symbols;
wenzelm [Thu, 21 Aug 2008 15:20:00 +0200] rev 27937
more robust pattern: look at longer matches first, added catch-all case;
more private fields;
reworked Recoder: more direct char/string operations, avoids inefficiency of large alternatives (java.util.regex does not optimize regexps);
wenzelm [Thu, 21 Aug 2008 13:05:37 +0200] rev 27936
added get_setting;
removed obsolete ISABELLE_HOME, ISABELLE_HOME_USER;
added platform_path, which expands variables and performs basic cygwin conversion;
wenzelm [Thu, 21 Aug 2008 13:05:31 +0200] rev 27935
read_symbols: proper IsabelleSystem.platform_path;