Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+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.
corrected class antiquotation
2008-10-02, by haftmann
max_threads_value always 1 for dummy version;
2008-10-02, by wenzelm
simplified Exn.EXCEPTIONS, flatten nested occurrences;
2008-10-02, by wenzelm
simplified Exn.EXCEPTIONS;
2008-10-02, by wenzelm
major cleanup of hoare_tac.ML: just one copy for Hoare.thy and HoareAbort.thy (only 1 line different), refrain from inspecting the main goal, proper context;
2008-10-02, by wenzelm
tuned
2008-10-02, by haftmann
Yet another proof of Newman's lemma, this time using the coherent logic prover.
2008-10-02, by berghofe
unit_source: more rigid parsing, stop after final qed;
2008-10-01, by wenzelm
excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
2008-10-01, by wenzelm
replaced can_defer by is_relevant (negation);
2008-10-01, by wenzelm
datatype transition: internal trans field is maintained in reverse order;
2008-10-01, by wenzelm
future_proof: protect conclusion of deferred proof state;
2008-10-01, by wenzelm
future_schedule: back to one group for all loader tasks;
2008-10-01, by wenzelm
tuned comments;
2008-10-01, by wenzelm
fixed
2008-10-01, by haftmann
renamed promise to future, tuned related interfaces;
2008-10-01, by wenzelm
more robust treatment of Interrupt (cf. exn.ML);
2008-10-01, by wenzelm
more robust treatment of Interrupt;
2008-10-01, by wenzelm
more robust treatment of Interrupt (cf. exn.ML);
2008-10-01, by wenzelm
removed release_results (cf. Exn.release_all, Exn.release_first);
2008-10-01, by wenzelm
more precise join_futures, improved termination;
2008-10-01, by wenzelm
added more_antiquote.ML
2008-10-01, by haftmann
extract Isabelle dist name correctly
2008-10-01, by kleing
unit_source: explicit treatment of 'oops' proofs;
2008-09-30, by wenzelm
promise_proof: proper statement with empty vars;
2008-09-30, by wenzelm
load_thy: more precise treatment of improper cmd or proof (notably 'oops');
2008-09-30, by wenzelm
schedule_tasks: single theory is loaded concurrently as well (cf. concurrent Toplevel.excursion);
2008-09-30, by wenzelm
added unit_source: commands with proof;
2008-09-30, by wenzelm
begin_proof: avoid race condition wrt. skip_proofs flag;
2008-09-30, by wenzelm
load_thy: Toplevel.excursion based on units of command/proof pairs;
2008-09-30, by wenzelm
more command categories;
2008-09-30, by wenzelm
renamed Future.fork_irrelevant to Future.fork_background;
2008-09-30, by wenzelm
export explicit joint_futures, removed Theory.at_end hook;
2008-09-30, by wenzelm
tuned
2008-09-30, by haftmann
turned process_thy into present_thy, which merely does presentation (wrt. persistent intermediate states);
2008-09-30, by wenzelm
Toplevel.commit_exit: position;
2008-09-30, by wenzelm
export setmp_thread_position;
2008-09-30, by wenzelm
simplified process_file, eliminated Toplevel.excursion;
2008-09-30, by wenzelm
clarified codegen interfaces
2008-09-30, by haftmann
tuned
2008-09-30, by haftmann
reorganized examples
2008-09-30, by haftmann
fixed slips
2008-09-30, by haftmann
re-canibalised manual
2008-09-30, by haftmann
slightly different command line for makedist_mercurial
2008-09-30, by kleing
put_thms: ContextPosition.set_visible false;
2008-09-29, by wenzelm
added type pp, which helps installing polymorphic pretty printers;
2008-09-29, by wenzelm
added str_of;
2008-09-29, by wenzelm
install_pp Future.T (polyml only);
2008-09-29, by wenzelm
report_token/parse_token: back to context-less version;
2008-09-29, by wenzelm
back to plain Position.report for regular references;
2008-09-29, by wenzelm
back to plain Position.report for regular references;
2008-09-29, by wenzelm
promise global proofs;
2008-09-29, by wenzelm
renamed report to report_visible;
2008-09-29, by wenzelm
code example: back to individual ML commands, which are now thread-safe;
2008-09-29, by wenzelm
ContextPosition.report;
2008-09-29, by wenzelm
target update: invisible context position avoids duplication of reports etc.;
2008-09-29, by wenzelm
Context position visibility.
2008-09-29, by wenzelm
added context_position.ML;
2008-09-29, by wenzelm
more precise redundancy check
2008-09-29, by haftmann
clarified dependencies between arith tools
2008-09-29, by haftmann
separate HOL-Main image
2008-09-29, by haftmann
polished code generator setup
2008-09-29, by haftmann
added theory antiquotation
2008-09-29, by haftmann
tuned comments;
2008-09-29, by wenzelm
handle _ should be avoided (spurious Interrupt will spoil the game);
2008-09-29, by wenzelm
added norm_export_morphism;
2008-09-29, by wenzelm
added exit_global, exit_result, exit_result_global;
2008-09-29, by wenzelm
LocalTheory.exit_global;
2008-09-29, by wenzelm
HOL no longer depends on HOL-Plain;
2008-09-28, by wenzelm
setmp_noncritical;
2008-09-28, by wenzelm
join earlier promises first;
2008-09-28, by wenzelm
proper setmp_thread_data for nested execute (cf. join_loop);
2008-09-28, by wenzelm
promise_result: enforce strictly sequential dependencies, via serial numbers;
2008-09-28, by wenzelm
do not cvs update for doc test (switching to mercurial, update done outside
2008-09-28, by kleing
use mercurial repository for isatest
2008-09-28, by kleing
thread_data: include thread name, export access;
2008-09-28, by wenzelm
setmp_noncritical;
2008-09-27, by wenzelm
dequeue_towards: return bound for unfinished tasks;
2008-09-27, by wenzelm
moved release_results to future.ML;
2008-09-27, by wenzelm
added release_results (formerly in par_list.ML);
2008-09-27, by wenzelm
Future.release_results;
2008-09-27, by wenzelm
more tracing;
2008-09-27, by wenzelm
Theory.checkpoint for main operations, admits concurrent proofs;
2008-09-27, by wenzelm
promise: include check into future body, i.e. joined results are always valid;
2008-09-27, by wenzelm
proper transfer of theorems that involve classes being instantiated here;
2008-09-27, by wenzelm
HOL_USEDIR_OPTIONS no longer applies to HOL-Plain (main HOL is rebuilt from Pure);
2008-09-27, by wenzelm
eliminated polymorphic equality;
2008-09-26, by wenzelm
added subset operation;
2008-09-26, by wenzelm
Added fresh_star_const.
2008-09-26, by berghofe
Added some more theorems to NominalData.
2008-09-26, by berghofe
Added some more lemmas that are useful in proof of strong induction rule.
2008-09-26, by berghofe
removed obsolete name convention "func"
2008-09-26, by haftmann
fixed typo
2008-09-26, by haftmann
clarified function transformator interface
2008-09-26, by haftmann
op = vs. eq
2008-09-26, by haftmann
moved future_scheduler flag to skip_proof.ML;
2008-09-25, by wenzelm
added future_scheduler (from thy_info.ML);
2008-09-25, by wenzelm
simplified promise;
2008-09-25, by wenzelm
simplified Thm.promise;
2008-09-25, by wenzelm
explicit checkpoint for low-level (global) theory operations admits concurrent SkipProof.prove;
2008-09-25, by wenzelm
explicit checkpoint for low-level (global) theory operations, admits concurrent proofs;
2008-09-25, by wenzelm
circumvent problem with code redundancy
2008-09-25, by haftmann
clarifed redundancy policy
2008-09-25, by haftmann
tuned comments;
2008-09-25, by wenzelm
added release_results;
2008-09-25, by wenzelm
abtract types: plain datatype with opaque signature matching;
2008-09-25, by wenzelm
prove: error with original thread position;
2008-09-25, by wenzelm
explicit type OrdList.T;
2008-09-25, by wenzelm
(temporary workaround)
2008-09-25, by haftmann
(temporal deactivation)
2008-09-25, by haftmann
non left-linear equations for nbe
2008-09-25, by haftmann
non left-linear equations for nbe
2008-09-25, by haftmann
map_force
2008-09-25, by haftmann
matchess
2008-09-25, by haftmann
burrow_fst
2008-09-25, by haftmann
discontinued special treatment of op = vs. eq_class.eq
2008-09-25, by haftmann
report: produce individual status messages;
2008-09-24, by wenzelm
protocol change: remapped message codes to make room for nested system messages (e.g. for protocol proxy);
2008-09-24, by wenzelm
protocol change: remapped message codes to make room for nested system messages (e.g. for protocol proxy);
2008-09-24, by wenzelm
init: OuterKeyword.report;
2008-09-24, by wenzelm
prove_multi: immediate;
2008-09-23, by wenzelm
added promise_result, prove_promise;
2008-09-23, by wenzelm
Corrected call of SUBPROOF in coherent_tac that used wrong context.
2008-09-23, by berghofe
fixed outer syntax
2008-09-23, by haftmann
case default fallback for NBE
2008-09-23, by haftmann
fixed quickcheck parameter syntax
2008-09-23, by haftmann
renamed rtype to typerep
2008-09-23, by haftmann
added fold_rev;
2008-09-23, by wenzelm
added del_node, which is more efficient for sparse graphs;
2008-09-23, by wenzelm
IntGraph.del_node;
2008-09-23, by wenzelm
join_results: special case for empty list, works without multithreading;
2008-09-23, by wenzelm
added dest_deriv, removed external type deriv;
2008-09-23, by wenzelm
added conditional add_oracles, keep oracles_of_proof private;
2008-09-23, by wenzelm
Thm.proof_of;
2008-09-23, by wenzelm
Added coherent logic prover.
2008-09-22, by berghofe
New prover for coherent logic.
2008-09-22, by berghofe
Added setup for coherent logic prover.
2008-09-22, by berghofe
Added examples for coherent logic prover.
2008-09-22, by berghofe
Examples for coherent logic prover.
2008-09-22, by berghofe
made the perm_simp tactic to understand options such as (no_asm)
2008-09-22, by urbanc
type thm: fully internal derivation, no longer exported;
2008-09-22, by wenzelm
added is_finished;
2008-09-22, by wenzelm
added Promise constructor, which is similar to Oracle but may be replaced later;
2008-09-22, by wenzelm
removed deriv.ML which is now incorporated into thm.ML;
2008-09-22, by wenzelm
added reject_draft;
2008-09-22, by wenzelm
type thm: fully internal derivation, no longer exported;
2008-09-22, by wenzelm
generic quickcheck framework
2008-09-22, by haftmann
TEMPORARY: make batch run happy
2008-09-22, by haftmann
absolute Library path
2008-09-22, by haftmann
different session branches for HOL-Plain vs. Plain
2008-09-22, by haftmann
temporary workaround for class constants
2008-09-22, by haftmann
corrected sort intersection
2008-09-22, by haftmann
some steps towards generic quickcheck framework
2008-09-22, by haftmann
fixed headers
2008-09-22, by haftmann
added some fragments from website
2008-09-22, by haftmann
made SML/NJ happy;
2008-09-20, by wenzelm
Isar toplevel editor model.
2008-09-19, by wenzelm
future tasks: support boolean priorities (true = high, false = low/irrelevant);
2008-09-19, by wenzelm
output_sync is now public;
2008-09-19, by wenzelm
added props_text (from isar_syn.ML);
2008-09-19, by wenzelm
moved Isar editor commands from isar_syn.ML to isar.ML;
2008-09-19, by wenzelm
moved Isar editor commands from isar_syn.ML to isar.ML;
2008-09-19, by wenzelm
added Isar/isar.scala;
2008-09-19, by wenzelm
avoid using implicit assumptions
2008-09-19, by huffman
add theory graph to ZF document
2008-09-19, by huffman
made SMLNJ happy
2008-09-19, by haftmann
jar: include sources;
2008-09-18, by wenzelm
tuned;
2008-09-18, by wenzelm
eval_term: CRITICAL due to eval_result;
2008-09-18, by wenzelm
begin_theory: Theory.checkpoint for immediate uses ensures that ML evaluation always starts with non-draft @{theory};
2008-09-18, by wenzelm
updated generated file;
2008-09-18, by wenzelm
simplified oracle interface;
2008-09-18, by wenzelm
show: non-critical testing;
2008-09-18, by wenzelm
added deriv.ML: Abstract derivations based on raw proof terms.
2008-09-18, by wenzelm
termination prover for "fun" can be configured using context data.
2008-09-18, by krauss
updated generated file;
2008-09-18, by wenzelm
unchecked $ISABELLE_HOME_USER/etc/settings;
2008-09-18, by wenzelm
use_text/use_file now depend on explicit ML name space;
2008-09-17, by wenzelm
threads work only for Poly/ML 5.2 or later;
2008-09-17, by wenzelm
* ML bindings produced via Isar commands are stored within the Isar context.
2008-09-17, by wenzelm
added ML_prf;
2008-09-17, by wenzelm
updated generated file;
2008-09-17, by wenzelm
added inherit_env;
2008-09-17, by wenzelm
added map_contexts;
2008-09-17, by wenzelm
ML_prf: inherit env for all contexts within the proof;
2008-09-17, by wenzelm
shutdown only if Multithreading.available;
2008-09-17, by wenzelm
ML_Context.evaluate: proper context (for ML environment);
2008-09-17, by wenzelm
ML_Context.evaluate: proper context (for ML environment);
2008-09-17, by wenzelm
simplified ML_Context.eval_in -- expect immutable Proof.context value;
2008-09-17, by wenzelm
proper thm antiquotations within ML solve obscure context problems (due to update of ML environment);
2008-09-17, by wenzelm
simplified ML_Context.eval_in -- expect immutable Proof.context value;
2008-09-17, by wenzelm
explicit handling of ML environment within generic context;
2008-09-17, by wenzelm
added ML_prf;
2008-09-17, by wenzelm
use_text/use_file now depend on explicit ML name space;
2008-09-17, by wenzelm
ML name space -- dummy version of Poly/ML 5.2 facility.
2008-09-17, by wenzelm
added ML-Systems/ml_name_space.ML;
2008-09-17, by wenzelm
use ML_prf within proofs;
2008-09-17, by wenzelm
local @{context};
2008-09-17, by wenzelm
moved global ML bindings to global place;
2008-09-17, by wenzelm
back to dynamic the_context(), because static @{theory} is invalidated if ML environment changes within the same code block;
2008-09-17, by wenzelm
updated generated file;
2008-09-17, by wenzelm
wf_finite_psubset[simp], in_finite_psubset[simp]
2008-09-17, by krauss
Public interface to interpretation morphism.
2008-09-17, by ballarin
moved term_of syntax to separate theory
2008-09-17, by haftmann
removed obsolete theory
2008-09-17, by haftmann
added quickcheck.ML
2008-09-17, by haftmann
tuned comments;
2008-09-16, by wenzelm
multithreading for Poly/ML 5.1 is no longer supported;
2008-09-16, by wenzelm
tuned;
2008-09-16, by wenzelm
updated system manual;
2008-09-16, by wenzelm
Proof General / Emacs interface wrapper;
2008-09-16, by wenzelm
Proof General: option -I is obsolete;
2008-09-16, by wenzelm
added PROOFGENERAL_HOME;
2008-09-16, by wenzelm
separate emacs tool for Proof General / Emacs;
2008-09-16, by wenzelm
added quickcheck stub
2008-09-16, by haftmann
removed babel again
2008-09-16, by haftmann
celver code lemma avoid type ambiguity problem with Haskell
2008-09-16, by haftmann
a sophisticated char/nibble conversion combinator
2008-09-16, by haftmann
moved term_of syntax to separate theory
2008-09-16, by haftmann
SimpleThread.fork;
2008-09-16, by wenzelm
Simplified thread fork interface.
2008-09-16, by wenzelm
added Concurrent/simple_thread.ML;
2008-09-16, by wenzelm
updated generated file;
2008-09-16, by wenzelm
misc tuning and modernization;
2008-09-16, by wenzelm
check setting and tool;
2008-09-16, by wenzelm
Clearer separation of interpretation frontend and backend.
2008-09-16, by ballarin
No interpretation of locale with dangling type frees.
2008-09-16, by ballarin
Do not rely on locale assumption in interpretation.
2008-09-16, by ballarin
The metis method now fails in the usual manner, rather than raising an exception,
2008-09-16, by paulson
Fixed typo in locale declaration.
2008-09-16, by ballarin
added babel
2008-09-16, by haftmann
explicit size of characters
2008-09-16, by haftmann
dropped superfluous code lemmas
2008-09-16, by haftmann
evaluation using code generator
2008-09-16, by haftmann
generic value command
2008-09-16, by haftmann
converted symbols.tex;
2008-09-15, by wenzelm
tuned;
2008-09-15, by wenzelm
converted misc.tex;
2008-09-15, by wenzelm
tuned;
2008-09-15, by wenzelm
generated files;
2008-09-15, by wenzelm
converted present.tex;
2008-09-15, by wenzelm
basic setup for generated document sources (cf. IsarRef/isar-ref.tex);
2008-09-15, by wenzelm
load underscore package after iman etc.;
2008-09-15, by wenzelm
tuned comment;
2008-09-15, by wenzelm
added formal markup for setting, executable, tool;
2008-09-15, by wenzelm
basic setup for generated document sources (cf. IsarRef/isar-ref.tex);
2008-09-15, by wenzelm
converted basics.tex to theory file;
2008-09-15, by wenzelm
added isatt markup;
2008-09-15, by wenzelm
New outline for codegen tutorial -- draft
2008-09-14, by haftmann
added extern_fact (local or global);
2008-09-12, by wenzelm
print raw (internal) result names;
2008-09-12, by wenzelm
more procise printing of fact names;
2008-09-12, by wenzelm
pretty_fact: extern fact name wrt. the given context, assuming that is the proper one for presentation;
2008-09-12, by wenzelm
cancel, shutdown: notify_all;
2008-09-11, by wenzelm
finish: Future.shutdown last;
2008-09-11, by wenzelm
eliminated requests, use global state variables uniformly;
2008-09-11, by wenzelm
finish: Future.shutdown;
2008-09-11, by wenzelm
added is_empty;
2008-09-11, by wenzelm
shutdown: global join-and-shutdown operation;
2008-09-11, by wenzelm
added focus, which indicates a particular collection of high-priority tasks;
2008-09-11, by wenzelm
some general notes on future values;
2008-09-11, by wenzelm
separate Concurrent/ROOT.ML;
2008-09-11, by wenzelm
Parallel list combinators.
2008-09-11, by wenzelm
added Concurrent/par_list.ML;
2008-09-11, by wenzelm
added interrupt_task (external id);
2008-09-10, by wenzelm
tuned;
2008-09-10, by wenzelm
future_schedule: uninterruptible join;
2008-09-10, by wenzelm
added future_scheduler (default false);
2008-09-10, by wenzelm
replaced join_all by join_results, which returns Exn.results;
2008-09-10, by wenzelm
workers: explicit activity flag;
2008-09-10, by wenzelm
future: allow explicit group;
2008-09-10, by wenzelm
cancel: invalidate group implicitly, via bool ref;
2008-09-10, by wenzelm
auto_flush: uniform block buffering for all output streams;
2008-09-10, by wenzelm
auto_flush stdout, stderr as well;
2008-09-09, by wenzelm
proper values of no_interrupts, regular_interrupts;
2008-09-09, by wenzelm
cancel: check_scheduler;
2008-09-09, by wenzelm
simplified dequeue: provide Thread.self internally;
2008-09-09, by wenzelm
eliminated cache, access queue efficiently via IntGraph.get_first;
2008-09-09, by wenzelm
export get_first from underlying table;
2008-09-09, by wenzelm
out_stream: block-buffered, with separate autoflush thread (every 50ms);
2008-09-09, by wenzelm
babel: removed unnecessary "french" option, which actually enables french section names etc. on some LaTeX installations;
2008-09-09, by wenzelm
added comment
2008-09-09, by nipkow
human-readable printing of TaskQueue.task/group;
2008-09-09, by wenzelm
* Changed defaults for unify configuration options;
2008-09-09, by wenzelm
inherit group from running thread, or create a new one -- make it harder to re-use canceled groups;
2008-09-09, by wenzelm
job: explicit 'ok' status -- false for canceled jobs;
2008-09-09, by wenzelm
Overall exception handler in order to insulate our users from low-level bugs.
2008-09-09, by paulson
more careful exception handling in order to prevent backtracking; miscellaneous tidying up.
2008-09-09, by paulson
Increasing the default limits in order to prevent unnecessary failures.
2008-09-09, by paulson
send: broadcast condition while locked!
2008-09-08, by wenzelm
proper signature constraint;
2008-09-08, by wenzelm
tuned Mailbox.send;
2008-09-08, by wenzelm
removed unused sync_interrupts;
2008-09-08, by wenzelm
moved thread data to future.ML (again);
2008-09-08, by wenzelm
more interrupt operations;
2008-09-08, by wenzelm
moved task, thread_data, group, queue to task_queue.ML;
2008-09-08, by wenzelm
Ordered queue of grouped tasks.
2008-09-08, by wenzelm
added Concurrent/task_queue.ML;
2008-09-08, by wenzelm
await: SYNCHRONIZED wait!
2008-09-08, by wenzelm
tuned check_cache;
2008-09-08, by wenzelm
added sync_interrupts, regular_interrupts;
2008-09-07, by wenzelm
added sync_interrupts, regular_interrupts;
2008-09-07, by wenzelm
opaque signature constraint abstracts local type abbrev;
2008-09-07, by wenzelm
tuned;
2008-09-07, by wenzelm
added change_result;
2008-09-07, by wenzelm
Functional threads as future values.
2008-09-07, by wenzelm
added Concurrent/future.ML;
2008-09-07, by wenzelm
Default (mostly dummy) implementation of thread structures.
2008-09-07, by wenzelm
*** MESSAGE REFERS TO PREVIOUS VERSION ***
2008-09-07, by wenzelm
*** empty log message ***
2008-09-07, by wenzelm
explicit use of universal.ML and dummy_thread.ML;
2008-09-07, by wenzelm
added no_interrupts;
2008-09-07, by wenzelm
added no_interrupts;
2008-09-07, by wenzelm
tuned;
2008-09-07, by wenzelm
send: broadcast to all waiting threads;
2008-09-07, by wenzelm
added ML-Systems/thread_dummy.ML;
2008-09-07, by wenzelm
dropped "run" marker in monad syntax
2008-09-06, by haftmann
multithreading.ML provides dummy thread structures;
2008-09-05, by wenzelm
different bookkeeping for code equations
2008-09-05, by haftmann
renamed structure CodeTarget to Code_Target
2008-09-05, by haftmann
instances comm_semiring_0_cancel < comm_semiring_0, comm_ring < comm_semiring_0_cancel
2008-09-05, by huffman
proper header;
2008-09-04, by wenzelm
added receive_timeout;
2008-09-04, by wenzelm
check WRAPPER_OUTPUT node type;
2008-09-04, by wenzelm
init: disallow "" as out stream;
2008-09-04, by wenzelm
fixed deps: no Concurrent/receiver.ML yet;
2008-09-04, by wenzelm
Concurrent message exchange via mailbox -- with unbounded queueing.
2008-09-04, by wenzelm
added Concurrent/mailbox.ML;
2008-09-04, by wenzelm
reorganize subsections
2008-09-04, by huffman
rename INF_drop_prefix to INFM_drop_prefix
2008-09-04, by huffman
add lemma power_Suc2; generalize power_minus from class comm_ring_1 to ring_1
2008-09-04, by huffman
move diff_add_cancel, add_diff_cancel from class ab_group_add to group_add
2008-09-04, by huffman
tuned signature;
2008-09-04, by wenzelm
added General/queue.ML;
2008-09-04, by wenzelm
Efficient queues.
2008-09-04, by wenzelm
moved Multithreading.task/schedule to Concurrent/schedule.ML
2008-09-04, by wenzelm
multithreading.ML provides dummy thread structures;
2008-09-04, by wenzelm
moved Multithreading.task/schedule to Concurrent/schedule.ML;
2008-09-04, by wenzelm
provide dummy thread structures, including proper Thread.getLocal/setLocal;
2008-09-04, by wenzelm
Thread.getLocal/setLocal;
2008-09-04, by wenzelm
Scheduling -- multiple threads working on a queue of tasks.
2008-09-04, by wenzelm
added Concurrent/schedule.ML;
2008-09-04, by wenzelm
update tags
2008-09-03, by convert-repo
use /home/isabelle/mercurial/bin/hg wrapper;
2008-09-03, by wenzelm
exclude large .mov files;
2008-09-03, by wenzelm
simplified add_axiom: no hyps;
2008-09-03, by wenzelm
discontinued local axioms -- too difficult to implement, too easy to produce nonsense;
2008-09-03, by wenzelm
axiomatization is now global-only;
2008-09-03, by wenzelm
added const_decl;
2008-09-03, by wenzelm
simplified specify_const: canonical args, global deps;
2008-09-03, by wenzelm
declare_const: Name.binding, store/report position;
2008-09-03, by wenzelm
Sign.declare_const: Name.binding;
2008-09-03, by wenzelm
removed ex/Puzzle
2008-09-03, by nipkow
added qualified: string -> binding -> binding;
2008-09-03, by wenzelm
Name.qualified;
2008-09-03, by wenzelm
theorem dependency hook: check previous state;
2008-09-03, by wenzelm
added pos_of;
2008-09-03, by wenzelm
-> AFP
2008-09-03, by nipkow
simplified Toplevel.add_hook: cover successful transactions only;
2008-09-03, by wenzelm
retired Ben Porter's DenumRat in favour of the shorter proof in
2008-09-03, by kleing
made SML/NJ happy;
2008-09-02, by wenzelm
refined theorem dependency output: previous state needs to contain a theory (not empty toplevel);
2008-09-02, by wenzelm
* Generic Toplevel.add_hook interface allows to analyze the result of
2008-09-02, by wenzelm
Replaced Library/NatPair by Nat_Int_Bij.
2008-09-02, by nipkow
added new_thms_deps (operates on global facts, some name_hint approximation);
2008-09-02, by wenzelm
theorem dependency output: Toplevel.add_hook, ProofGeneralPgip.new_thms_deps;
2008-09-02, by wenzelm
added add_hook interface for post-transition hooks;
2008-09-02, by wenzelm
tuned;
2008-09-02, by wenzelm
ProofDisplay.print_results;
2008-09-02, by wenzelm
no pervasive bindings;
2008-09-02, by wenzelm
Streamlined parts of Complex/ex/DenumRat and AFP/Integration/Rats and
2008-09-02, by nipkow
distributed literal code generation out of central infrastructure
2008-09-02, by haftmann
* Result facts now refer to the *full* internal name;
2008-09-02, by wenzelm
* Name bindings in higher specification mechanisms;
2008-09-02, by wenzelm
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);
2008-09-02, by wenzelm
updated generated file;
2008-09-02, by wenzelm
Interpretation commands no longer accept interpretation attributes.
2008-09-02, by ballarin
type Attrib.binding abbreviates Name.binding without attributes;
2008-09-02, by wenzelm
explicit type Name.binding for higher-specification elements;
2008-09-02, by wenzelm
explicit type Name.binding for higher-specification elements;
2008-09-02, by wenzelm
explicit type Name.binding for higher-specification elements;
2008-09-02, by wenzelm
explicit type Name.binding for higher-specification elements;
2008-09-02, by wenzelm
explicit type Name.binding for higher-specification elements;
2008-09-02, by wenzelm
added binding;
2008-09-02, by wenzelm
added fixed_decl, fact_decl, local_fact_decl;
2008-09-02, by wenzelm
name_thm etc.: pass position;
2008-09-02, by wenzelm
added type binding -- generic name bindings;
2008-09-02, by wenzelm
name/var morphism operates on Name.binding;
2008-09-02, by wenzelm
adapted to class instantiation compliance
2008-09-02, by haftmann
It appears that the code generator (Stefan's) needs some laws that appear superfluous: {..n} = set ...
2008-09-01, by nipkow
renamed lemma
2008-09-01, by nipkow
moved more lemmas here from AFP/Integration/Rats
2008-09-01, by nipkow
moved lemma into SetInterval where it belongs
2008-09-01, by nipkow
cleaned up code generation for {.._} and {..<_}
2008-09-01, by nipkow
*** empty log message ***
2008-09-01, by nipkow
extended interface to preferences to allow adding new ones
2008-09-01, by nipkow
Prover is set via menu now
2008-09-01, by nipkow
restructured code generation of literals
2008-09-01, by haftmann
IsabelleSystem.mk_fifo, IsabelleSystem.rm_fifo;
2008-08-29, by wenzelm
init: more explicit protocol of open/remove rendezvous;
2008-08-29, by wenzelm
use hardwired /tmp -- fifo only work on local file-system;
2008-08-29, by wenzelm
separate module for code output
2008-08-29, by haftmann
fixed names of class assumptions
2008-08-29, by haftmann
dropped parameter prefix for class theorems
2008-08-29, by haftmann
added charset (from isabelle_process.scala);
2008-08-28, by wenzelm
moved charset to isabelle_system.scala;
2008-08-28, by wenzelm
provide HOME_JVM=HOME to prevent implicit cygpath mangling;
2008-08-28, by wenzelm
restructured and split code serializer module
2008-08-28, by haftmann
no parameter prefix for class interpretation
2008-08-28, by haftmann
updated
2008-08-28, by haftmann
tuned fold_lines;
2008-08-28, by wenzelm
fold_lines: simplified, more efficient due to String.fields;
2008-08-28, by wenzelm
rm fifo after open;
2008-08-28, by wenzelm
dummy setup for completion;
2008-08-28, by wenzelm
create named pipe;
2008-08-28, by wenzelm
added is_cygwin;
2008-08-28, by wenzelm
join stdout/stderr, eliminated Kind.STDERR;
2008-08-28, by wenzelm
explicit output stream, typically a named pipe;
2008-08-28, by wenzelm
refined option -W: output stream;
2008-08-28, by wenzelm
more function -> fun
2008-08-28, by krauss
quicksort: function -> fun
2008-08-28, by krauss
corrected some typos
2008-08-28, by krauss
fixed atom_to_xml: literal "name" attribute;
2008-08-28, by wenzelm
exported atom_to_xml;
2008-08-28, by wenzelm
changed Markup print mode to YXML -- explicitly decode messages before being issued;
2008-08-28, by wenzelm
tuned;
2008-08-28, by wenzelm
present_token: disable print_mode, which is YXML now;
2008-08-28, by wenzelm
text_of Malformed: explode with spaces -- Output.output/escape ineffective by default;
2008-08-28, by wenzelm
removed obsolete XML.Output workaround;
2008-08-28, by wenzelm
added get_int;
2008-08-28, by wenzelm
removed obsolete get_string;
2008-08-28, by wenzelm
removed obsolete ProofGeneral/pgml_isabelle.ML;
2008-08-28, by wenzelm
simplify definition of vector_space locale (use axclasses instead of inheriting from field and ab_group_add classes)
2008-08-27, by huffman
renamed Buffer.write to File.write_buffer;
2008-08-27, by wenzelm
renamed Buffer.write to File.write_buffer;
2008-08-27, by wenzelm
load buffer.ML before file.ML;
2008-08-27, by wenzelm
replaced find_substring by first_field;
2008-08-27, by wenzelm
Consistent naming of theorems in interpretation.
2008-08-27, by ballarin
simplified parse_attrib (find_substring instead of space_explode);
2008-08-27, by wenzelm
added find_substring;
2008-08-27, by wenzelm
added HOL/ex/Numeral.thy
2008-08-27, by haftmann
get rid of tabs;
2008-08-27, by wenzelm
Property lists.
2008-08-27, by wenzelm
added General/properties.ML;
2008-08-27, by wenzelm
type Properties.T;
2008-08-27, by wenzelm
proper error message
2008-08-27, by haftmann
proper handling of type variabl names
2008-08-27, by haftmann
completing arities after subclass instance
2008-08-27, by haftmann
untabification
2008-08-27, by haftmann
tuned code generator setup
2008-08-27, by haftmann
added equivariance lemmas for ex1 and the
2008-08-27, by urbanc
add lemmas about Rats similar to those about Reals
2008-08-27, by huffman
move real_vector class proofs into vector_space and group_hom locales
2008-08-26, by huffman
added distributivity of relation composition over union [simp]
2008-08-26, by krauss
tuned append;
2008-08-26, by wenzelm
command: symbols.encode;
2008-08-26, by wenzelm
Reorganisation of registration code.
2008-08-26, by ballarin
function package: name primitive defs "f_sumC_def" instead of "f_sum_def" to avoid clashes
2008-08-26, by krauss
purge classes after compilation;
2008-08-26, by wenzelm
renamed Isabelle-repository to isabelle;
2008-08-26, by wenzelm
Defined rationals (Rats) globally in Rational.
2008-08-26, by nipkow
replaced /home/isabelle/html-data/isabelle-repos by /home/isabelle-repository/repos;
2008-08-26, by wenzelm
moved new Symbol.Interpretation into plugin;
2008-08-25, by wenzelm
promoted to EBPlugin;
2008-08-25, by wenzelm
explicitly depend on isabelle-Pure.jar and isabelle-scala-library.jar;
2008-08-25, by wenzelm
tuned;
2008-08-25, by wenzelm
isabelle process: pick options/args from properties;
2008-08-25, by wenzelm
removed unused ConsolePlugin dependency;
2008-08-25, by wenzelm
simplified exceptions: use plain error function / RuntimeException;
2008-08-25, by wenzelm
added try_result;
2008-08-25, by wenzelm
misc reorganization;
2008-08-24, by wenzelm
Kind: added is_control;
2008-08-24, by wenzelm
get: allow null;
2008-08-24, by wenzelm
misc tuning of names;
2008-08-24, by wenzelm
rearranged source files;
2008-08-24, by wenzelm
init_message: class markup in message body, not header;
2008-08-24, by wenzelm
repackaged as isabelle.jedit;
2008-08-24, by wenzelm
untabify: silently turn tab into space if column information is unavailable;
2008-08-24, by wenzelm
corrected cache handling for class operations
2008-08-24, by haftmann
default replaces arbitrary
2008-08-24, by haftmann
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip