Thu, 16 Oct 2008 00:18:53 +0200 kleing only test HOL image for smlnj
Wed, 15 Oct 2008 22:12:02 +0200 wenzelm tuned;
Wed, 15 Oct 2008 21:45:02 +0200 wenzelm tuned;
Wed, 15 Oct 2008 21:15:35 +0200 wenzelm generic ATP manager based on threads (by Fabian Immler);
Wed, 15 Oct 2008 21:06:15 +0200 wenzelm added sledgehammer etc.;
Wed, 15 Oct 2008 19:43:11 +0200 wenzelm removed obsolete Complex sessions;
Wed, 15 Oct 2008 16:25:31 +0200 haftmann figure for adaption
Wed, 15 Oct 2008 16:06:59 +0200 ballarin Removed 'includes' (fixed).
Wed, 15 Oct 2008 15:44:15 +0200 ballarin Removed 'includes'.
Wed, 15 Oct 2008 00:18:43 +0200 kleing give more time to do inital loggin and settings read
Wed, 15 Oct 2008 00:18:19 +0200 kleing log start of test session
Tue, 14 Oct 2008 20:10:45 +0200 wenzelm tuned interfaces -- plain prover function, without thread;
Tue, 14 Oct 2008 20:10:44 +0200 wenzelm add_prover: plain prover function, without thread;
Tue, 14 Oct 2008 20:10:43 +0200 wenzelm tuned AtpWrapper interfaces;
Tue, 14 Oct 2008 16:32:26 +0200 haftmann continued codegen tutorial
Tue, 14 Oct 2008 16:01:36 +0200 wenzelm renamed AtpThread to AtpWrapper;
Tue, 14 Oct 2008 15:45:46 +0200 wenzelm adding preferences is now permissive;
Tue, 14 Oct 2008 15:45:45 +0200 wenzelm tuned;
Tue, 14 Oct 2008 15:45:44 +0200 wenzelm adding preferences is now permissive, no error handling here;
Tue, 14 Oct 2008 15:16:13 +0200 wenzelm CRITICAL access to preferences;
Tue, 14 Oct 2008 15:16:12 +0200 wenzelm export generic_pref etc.;
Tue, 14 Oct 2008 15:16:11 +0200 wenzelm renamed kill_all to kill, in conformance with atp_kill command;
Tue, 14 Oct 2008 15:16:09 +0200 wenzelm tuned comments;
Tue, 14 Oct 2008 13:24:07 +0200 nipkow added lemma
Tue, 14 Oct 2008 13:23:31 +0200 nipkow Added liveness analysis
Tue, 14 Oct 2008 13:01:58 +0200 wenzelm info: back to plain printing;
Tue, 14 Oct 2008 13:01:57 +0200 wenzelm added min_elem, upto;
Tue, 14 Oct 2008 13:01:56 +0200 wenzelm added value;
Tue, 14 Oct 2008 13:01:52 +0200 wenzelm simplified synchronized variable access;
Mon, 13 Oct 2008 15:48:40 +0200 wenzelm State variables with synchronized access.
Mon, 13 Oct 2008 15:48:39 +0200 wenzelm added generic combinator for synchronized evaluation (formerly in future.ML);
Mon, 13 Oct 2008 15:48:38 +0200 wenzelm simplified implementation using Synchronized.var;
Mon, 13 Oct 2008 15:48:37 +0200 wenzelm SimpleThread.synchronized;
Mon, 13 Oct 2008 15:48:36 +0200 wenzelm added Concurrent/synchronized.ML;
Mon, 13 Oct 2008 14:04:53 +0200 wenzelm ** Update from Fabian **
Mon, 13 Oct 2008 14:04:29 +0200 wenzelm ** Update from Fabian **
Mon, 13 Oct 2008 14:04:28 +0200 wenzelm ** Update from Fabian **
Mon, 13 Oct 2008 13:56:54 +0200 wenzelm tuned output;
Mon, 13 Oct 2008 13:44:59 +0200 haftmann tuned
Mon, 13 Oct 2008 06:54:25 +0200 urbanc tuned
Sat, 11 Oct 2008 03:54:34 +0200 kleing change DISTPREFIX to not use yet another filesystem
Fri, 10 Oct 2008 16:02:15 +0200 haftmann tuned
Fri, 10 Oct 2008 15:52:45 +0200 haftmann tuned
Fri, 10 Oct 2008 15:23:33 +0200 haftmann tuned
Fri, 10 Oct 2008 06:49:44 +0200 haftmann tuned
Fri, 10 Oct 2008 06:45:53 +0200 haftmann `code func` now just `code`
Fri, 10 Oct 2008 06:45:50 +0200 haftmann some adaption
Fri, 10 Oct 2008 06:45:49 +0200 haftmann using tikz pictures
Fri, 10 Oct 2008 06:45:48 +0200 haftmann tuned default rules of (dvd)
Thu, 09 Oct 2008 21:34:11 +0200 wenzelm replaced str_of by general peek;
Thu, 09 Oct 2008 21:34:05 +0200 wenzelm extra Poly/ML toplevel pretty printing in ML-Systems/install_pp_polyml.ML;
Thu, 09 Oct 2008 21:06:08 +0200 wenzelm fixed spelling;
Thu, 09 Oct 2008 20:53:24 +0200 wenzelm added enabled;
Thu, 09 Oct 2008 20:53:23 +0200 wenzelm added enabled;
Thu, 09 Oct 2008 20:53:22 +0200 wenzelm Multithreading.enabled;
Thu, 09 Oct 2008 20:53:21 +0200 wenzelm moved future_scheduler flag to Concurrent/ROOT.ML;
Thu, 09 Oct 2008 20:53:20 +0200 wenzelm added invalidate_group;
Thu, 09 Oct 2008 20:53:17 +0200 wenzelm added fail-safe interrupt;
Thu, 09 Oct 2008 20:53:16 +0200 wenzelm subject to Multithreading.enabled;
Thu, 09 Oct 2008 20:53:15 +0200 wenzelm future result: Interrupt invalidates group, but pretends success otherwise;
Thu, 09 Oct 2008 20:53:14 +0200 wenzelm added future_scheduler flag (tmp!), from skip_proofs.ML;
Thu, 09 Oct 2008 20:53:13 +0200 wenzelm Dummy version of parallel list combinators -- plain sequential evaluation.
Thu, 09 Oct 2008 20:53:12 +0200 wenzelm added Concurrent/par_list_dummy.ML;
Thu, 09 Oct 2008 20:53:11 +0200 wenzelm improved performance of skolem cache, due to parallel map;
Thu, 09 Oct 2008 20:53:10 +0200 wenzelm SimpleThread.interrupt;
Thu, 09 Oct 2008 20:03:22 +0200 wenzelm report: back to single message;
Thu, 09 Oct 2008 19:24:21 +0200 wenzelm added section label;
Thu, 09 Oct 2008 18:16:07 +0200 haftmann tuned
Thu, 09 Oct 2008 09:18:32 +0200 kleing do logging to MASTERLOG centrally (avoid multiple writers over NFS as
Thu, 09 Oct 2008 08:47:28 +0200 haftmann removed legacy |>>>
Thu, 09 Oct 2008 08:47:27 +0200 haftmann established canonical argument order in SML code generators
Thu, 09 Oct 2008 08:47:26 +0200 haftmann established canonical argument order
Thu, 09 Oct 2008 08:47:25 +0200 haftmann made SMLNJ happy
Wed, 08 Oct 2008 20:37:44 +0200 wenzelm less tracing;
Wed, 08 Oct 2008 20:21:35 +0200 wenzelm Future.joint_results is already uninterruptible;
Wed, 08 Oct 2008 20:21:34 +0200 wenzelm more careful handling of group interrupts;
Wed, 08 Oct 2008 19:32:20 +0200 wenzelm use polyml-cvs, which fixes a serious deadlock problem of Poly/ML runtime vs. GC;
Wed, 08 Oct 2008 19:30:15 +0200 wenzelm added HOL-Main;
Wed, 08 Oct 2008 19:20:29 +0200 wenzelm setmp_noncritical makes it work with future scheduler;
Wed, 08 Oct 2008 18:09:36 +0200 paulson The result of the equality inference rule no longer undergoes factoring.
Wed, 08 Oct 2008 00:25:38 +0200 kleing make the test for experimental sessions in isatest-check actually work
Wed, 08 Oct 2008 00:03:42 +0200 kleing leave a log message when no snapshot is generated
Tue, 07 Oct 2008 16:07:59 +0200 haftmann clarified preprocessor policies
Tue, 07 Oct 2008 16:07:50 +0200 haftmann arbitrary is undefined
Tue, 07 Oct 2008 16:07:40 +0200 haftmann tuned whitespace
Tue, 07 Oct 2008 16:07:33 +0200 haftmann only one theorem table for both code generators
Tue, 07 Oct 2008 16:07:30 +0200 haftmann proper default codegen attribute
Tue, 07 Oct 2008 16:07:25 +0200 haftmann tuned code setup
Tue, 07 Oct 2008 16:07:24 +0200 haftmann code generator more liberal with respect to sort constraints of instance parameters
Tue, 07 Oct 2008 16:07:23 +0200 haftmann more Isar for example
Tue, 07 Oct 2008 16:07:22 +0200 haftmann tuned funpow code generation
Tue, 07 Oct 2008 16:07:21 +0200 haftmann tuned min/max code generation
Tue, 07 Oct 2008 16:07:20 +0200 haftmann dropped superfluous if
Tue, 07 Oct 2008 16:07:18 +0200 haftmann tuned of_nat code generation
Tue, 07 Oct 2008 16:07:16 +0200 haftmann re-introduces axiom subst
Tue, 07 Oct 2008 16:07:14 +0200 haftmann corrected SML undefined
Tue, 07 Oct 2008 11:51:31 +0200 wenzelm updated to official version as of 07-Oct-2008;
Mon, 06 Oct 2008 22:41:21 +0200 wenzelm fold_lines: more tuning, avoiding extra split_last;
Mon, 06 Oct 2008 22:35:03 +0200 wenzelm extra check of PROOFGENERAL_HOME;
Sun, 05 Oct 2008 13:13:48 +0200 kleing needs -b option for isabelle getenv
Sat, 04 Oct 2008 17:51:10 +0200 wenzelm updated generated file;
Sat, 04 Oct 2008 17:50:57 +0200 wenzelm tuned isabelle usage;
Sat, 04 Oct 2008 17:40:58 +0200 wenzelm updated generated file;
Sat, 04 Oct 2008 17:40:56 +0200 wenzelm simplified main Isabelle executables: removed Isabelle and isabelle (replaced by isabelle-process), renamed isatool to isabelle;
Sat, 04 Oct 2008 16:19:49 +0200 wenzelm updated generated file;
Sat, 04 Oct 2008 16:19:00 +0200 wenzelm replaced ISABELLE by ISABELLE_PROCESS;
Sat, 04 Oct 2008 16:05:15 +0200 wenzelm ISABELLE_PROCESS commandline;
Sat, 04 Oct 2008 16:05:09 +0200 wenzelm replaced ISATOOL by ISABELLE_TOOL;
Sat, 04 Oct 2008 16:05:08 +0200 wenzelm ISABELLE_PROCESS replaces ISABELLE and ISABELLE_TOOL replaces ISATOOL -- old bindings stay for a while (legacy feature);
Sat, 04 Oct 2008 14:43:40 +0200 wenzelm eliminated prompt messages;
Sat, 04 Oct 2008 14:29:45 +0200 wenzelm added isabelle_tool version as basic integrity check of platform/distribution;
Sat, 04 Oct 2008 14:29:43 +0200 wenzelm renamed isatool to isabelle_tool in programming interfaces;
Sat, 04 Oct 2008 14:29:42 +0200 wenzelm Theory header keywords.
Sat, 04 Oct 2008 14:29:40 +0200 wenzelm added Thy/thy_header.scala;
Fri, 03 Oct 2008 21:31:27 +0200 wenzelm tuned quotes;
Fri, 03 Oct 2008 21:13:17 +0200 wenzelm factor: proper padding of digits;
Fri, 03 Oct 2008 21:06:39 +0200 wenzelm plain process_id function;
Fri, 03 Oct 2008 21:06:38 +0200 wenzelm removed obsolete Posix/Signal compatibility wrappers;
Fri, 03 Oct 2008 21:06:37 +0200 wenzelm removed obsolete Posix/Signal compatibility wrappers;
Fri, 03 Oct 2008 21:06:36 +0200 wenzelm removed obsolete Posix/Signal compatibility wrappers;
Fri, 03 Oct 2008 20:10:44 +0200 wenzelm do not handle Error (which matches arbitrary exceptions!), but ERROR _;
Fri, 03 Oct 2008 20:10:43 +0200 wenzelm updated to new AtpManager;
Fri, 03 Oct 2008 19:35:18 +0200 wenzelm operate on Proof.state, not Toplevel.state;
Fri, 03 Oct 2008 19:35:17 +0200 wenzelm misc simplifcation and tuning;
Fri, 03 Oct 2008 19:35:16 +0200 wenzelm perform atp_setups here;
Fri, 03 Oct 2008 19:35:15 +0200 wenzelm updated generated file;
Fri, 03 Oct 2008 19:35:14 +0200 wenzelm removed HOL-Plain -- already included in HOL;
Fri, 03 Oct 2008 19:17:37 +0200 wenzelm removed spurious ResAtp.set_prover;
Fri, 03 Oct 2008 17:07:41 +0200 wenzelm simplified thread creation via SimpleThread;
Fri, 03 Oct 2008 17:07:39 +0200 wenzelm simplified thread creation via SimpleThread;
Fri, 03 Oct 2008 16:37:09 +0200 wenzelm version of sledgehammer using threads instead of processes, misc cleanup;
Fri, 03 Oct 2008 15:20:33 +0200 wenzelm removed old/unused setup of raw ATP oracles;
Fri, 03 Oct 2008 14:07:41 +0200 wenzelm tuned;
Fri, 03 Oct 2008 14:06:19 +0200 wenzelm Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
Fri, 03 Oct 2008 13:21:01 +0200 wenzelm added PROOFGENERAL_EMACS, with attempt to find Carbon Emacs;
Fri, 03 Oct 2008 00:21:48 +0200 wenzelm tuned tracing;
Fri, 03 Oct 2008 00:12:13 +0200 wenzelm slower heartbeat;
Thu, 02 Oct 2008 23:52:12 +0200 wenzelm added simple heartbeat thread;
Thu, 02 Oct 2008 23:52:10 +0200 wenzelm time factor: one more digit;
Thu, 02 Oct 2008 23:30:44 +0200 wenzelm more tuning of tracing messages;
Thu, 02 Oct 2008 22:09:22 +0200 wenzelm include factor in timing report;
Thu, 02 Oct 2008 21:21:21 +0200 wenzelm with_attributes: enforces InterruptAsynch => InterruptAsynchOnce to avoid race condition;
Thu, 02 Oct 2008 19:59:01 +0200 wenzelm tracing: ignore failure of any kind;
Thu, 02 Oct 2008 19:59:00 +0200 wenzelm tuned SYNCHRONIZED: outermost Exn.release;
Thu, 02 Oct 2008 19:38:48 +0200 wenzelm program wrapper: controlled_execution ensures proper thread attributes (global default is unsafe due to InterruptAsynch;
Thu, 02 Oct 2008 17:18:36 +0200 haftmann added partiality section
Thu, 02 Oct 2008 17:18:22 +0200 haftmann corrected class antiquotation
Thu, 02 Oct 2008 14:22:45 +0200 wenzelm max_threads_value always 1 for dummy version;
Thu, 02 Oct 2008 14:22:44 +0200 wenzelm simplified Exn.EXCEPTIONS, flatten nested occurrences;
Thu, 02 Oct 2008 14:22:40 +0200 wenzelm simplified Exn.EXCEPTIONS;
Thu, 02 Oct 2008 14:22:36 +0200 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;
Thu, 02 Oct 2008 13:07:33 +0200 haftmann tuned
Thu, 02 Oct 2008 12:17:20 +0200 berghofe Yet another proof of Newman's lemma, this time using the coherent logic prover.
Wed, 01 Oct 2008 22:33:29 +0200 wenzelm unit_source: more rigid parsing, stop after final qed;
Wed, 01 Oct 2008 22:33:28 +0200 wenzelm excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
Wed, 01 Oct 2008 22:33:24 +0200 wenzelm replaced can_defer by is_relevant (negation);
Wed, 01 Oct 2008 20:02:37 +0200 wenzelm datatype transition: internal trans field is maintained in reverse order;
Wed, 01 Oct 2008 18:16:14 +0200 wenzelm future_proof: protect conclusion of deferred proof state;
Wed, 01 Oct 2008 18:16:10 +0200 wenzelm future_schedule: back to one group for all loader tasks;
Wed, 01 Oct 2008 14:17:06 +0200 wenzelm tuned comments;
Wed, 01 Oct 2008 13:33:54 +0200 haftmann fixed
Wed, 01 Oct 2008 12:18:18 +0200 wenzelm renamed promise to future, tuned related interfaces;
Wed, 01 Oct 2008 12:00:05 +0200 wenzelm more robust treatment of Interrupt (cf. exn.ML);
Wed, 01 Oct 2008 12:00:04 +0200 wenzelm more robust treatment of Interrupt;
Wed, 01 Oct 2008 12:00:02 +0200 wenzelm more robust treatment of Interrupt (cf. exn.ML);
Wed, 01 Oct 2008 12:00:01 +0200 wenzelm removed release_results (cf. Exn.release_all, Exn.release_first);
Wed, 01 Oct 2008 12:00:00 +0200 wenzelm more precise join_futures, improved termination;
Wed, 01 Oct 2008 08:42:42 +0200 haftmann added more_antiquote.ML
Wed, 01 Oct 2008 00:09:51 +0200 kleing extract Isabelle dist name correctly
Tue, 30 Sep 2008 23:31:40 +0200 wenzelm unit_source: explicit treatment of 'oops' proofs;
Tue, 30 Sep 2008 23:31:38 +0200 wenzelm promise_proof: proper statement with empty vars;
Tue, 30 Sep 2008 23:31:36 +0200 wenzelm load_thy: more precise treatment of improper cmd or proof (notably 'oops');
Tue, 30 Sep 2008 22:02:55 +0200 wenzelm schedule_tasks: single theory is loaded concurrently as well (cf. concurrent Toplevel.excursion);
Tue, 30 Sep 2008 22:02:53 +0200 wenzelm added unit_source: commands with proof;
Tue, 30 Sep 2008 22:02:51 +0200 wenzelm begin_proof: avoid race condition wrt. skip_proofs flag;
Tue, 30 Sep 2008 22:02:50 +0200 wenzelm load_thy: Toplevel.excursion based on units of command/proof pairs;
Tue, 30 Sep 2008 22:02:47 +0200 wenzelm more command categories;
Tue, 30 Sep 2008 22:02:45 +0200 wenzelm renamed Future.fork_irrelevant to Future.fork_background;
Tue, 30 Sep 2008 22:02:44 +0200 wenzelm export explicit joint_futures, removed Theory.at_end hook;
Tue, 30 Sep 2008 14:30:44 +0200 haftmann tuned
Tue, 30 Sep 2008 14:19:28 +0200 wenzelm turned process_thy into present_thy, which merely does presentation (wrt. persistent intermediate states);
Tue, 30 Sep 2008 14:19:27 +0200 wenzelm Toplevel.commit_exit: position;
Tue, 30 Sep 2008 14:19:26 +0200 wenzelm export setmp_thread_position;
Tue, 30 Sep 2008 14:19:25 +0200 wenzelm simplified process_file, eliminated Toplevel.excursion;
Tue, 30 Sep 2008 12:49:18 +0200 haftmann clarified codegen interfaces
Tue, 30 Sep 2008 12:49:17 +0200 haftmann tuned
Tue, 30 Sep 2008 12:49:16 +0200 haftmann reorganized examples
Tue, 30 Sep 2008 12:49:14 +0200 haftmann fixed slips
Tue, 30 Sep 2008 11:19:47 +0200 haftmann re-canibalised manual
Tue, 30 Sep 2008 04:06:55 +0200 kleing slightly different command line for makedist_mercurial
Mon, 29 Sep 2008 21:45:44 +0200 wenzelm put_thms: ContextPosition.set_visible false;
Mon, 29 Sep 2008 21:26:49 +0200 wenzelm added type pp, which helps installing polymorphic pretty printers;
Mon, 29 Sep 2008 21:26:46 +0200 wenzelm added str_of;
Mon, 29 Sep 2008 21:26:44 +0200 wenzelm install_pp Future.T (polyml only);
Mon, 29 Sep 2008 21:26:41 +0200 wenzelm report_token/parse_token: back to context-less version;
Mon, 29 Sep 2008 21:26:39 +0200 wenzelm back to plain Position.report for regular references;
Mon, 29 Sep 2008 21:26:36 +0200 wenzelm back to plain Position.report for regular references;
Mon, 29 Sep 2008 21:26:32 +0200 wenzelm promise global proofs;
Mon, 29 Sep 2008 21:26:26 +0200 wenzelm renamed report to report_visible;
Mon, 29 Sep 2008 14:59:02 +0200 wenzelm code example: back to individual ML commands, which are now thread-safe;
Mon, 29 Sep 2008 14:41:25 +0200 wenzelm ContextPosition.report;
Mon, 29 Sep 2008 14:41:24 +0200 wenzelm target update: invisible context position avoids duplication of reports etc.;
Mon, 29 Sep 2008 14:41:23 +0200 wenzelm Context position visibility.
Mon, 29 Sep 2008 14:41:22 +0200 wenzelm added context_position.ML;
Mon, 29 Sep 2008 12:32:00 +0200 haftmann more precise redundancy check
Mon, 29 Sep 2008 12:31:59 +0200 haftmann clarified dependencies between arith tools
Mon, 29 Sep 2008 12:31:58 +0200 haftmann separate HOL-Main image
Mon, 29 Sep 2008 12:31:57 +0200 haftmann polished code generator setup
Mon, 29 Sep 2008 12:31:56 +0200 haftmann added theory antiquotation
Mon, 29 Sep 2008 11:46:52 +0200 wenzelm tuned comments;
Mon, 29 Sep 2008 11:46:47 +0200 wenzelm handle _ should be avoided (spurious Interrupt will spoil the game);
Mon, 29 Sep 2008 10:58:04 +0200 wenzelm added norm_export_morphism;
Mon, 29 Sep 2008 10:58:03 +0200 wenzelm added exit_global, exit_result, exit_result_global;
Mon, 29 Sep 2008 10:58:01 +0200 wenzelm LocalTheory.exit_global;
Sun, 28 Sep 2008 14:46:51 +0200 wenzelm HOL no longer depends on HOL-Plain;
Sun, 28 Sep 2008 14:40:43 +0200 wenzelm setmp_noncritical;
Sun, 28 Sep 2008 12:42:35 +0200 wenzelm join earlier promises first;
Sun, 28 Sep 2008 12:23:45 +0200 wenzelm proper setmp_thread_data for nested execute (cf. join_loop);
Sun, 28 Sep 2008 12:23:44 +0200 wenzelm promise_result: enforce strictly sequential dependencies, via serial numbers;
Sun, 28 Sep 2008 09:25:24 +0200 kleing do not cvs update for doc test (switching to mercurial, update done outside
Sun, 28 Sep 2008 09:13:46 +0200 kleing use mercurial repository for isatest
Sun, 28 Sep 2008 00:00:55 +0200 wenzelm thread_data: include thread name, export access;
Sat, 27 Sep 2008 19:35:00 +0200 wenzelm setmp_noncritical;
Sat, 27 Sep 2008 18:18:08 +0200 wenzelm dequeue_towards: return bound for unfinished tasks;
Sat, 27 Sep 2008 18:18:07 +0200 wenzelm moved release_results to future.ML;
Sat, 27 Sep 2008 18:18:06 +0200 wenzelm added release_results (formerly in par_list.ML);
Sat, 27 Sep 2008 18:18:05 +0200 wenzelm Future.release_results;
Sat, 27 Sep 2008 15:37:01 +0200 wenzelm more tracing;
Sat, 27 Sep 2008 15:20:39 +0200 wenzelm Theory.checkpoint for main operations, admits concurrent proofs;
Sat, 27 Sep 2008 15:20:37 +0200 wenzelm promise: include check into future body, i.e. joined results are always valid;
Sat, 27 Sep 2008 15:20:36 +0200 wenzelm proper transfer of theorems that involve classes being instantiated here;
Sat, 27 Sep 2008 14:26:06 +0200 wenzelm HOL_USEDIR_OPTIONS no longer applies to HOL-Plain (main HOL is rebuilt from Pure);
Fri, 26 Sep 2008 19:07:56 +0200 wenzelm eliminated polymorphic equality;
Fri, 26 Sep 2008 17:24:15 +0200 wenzelm added subset operation;
Fri, 26 Sep 2008 14:53:10 +0200 berghofe Added fresh_star_const.
Fri, 26 Sep 2008 14:52:27 +0200 berghofe Added some more theorems to NominalData.
Fri, 26 Sep 2008 14:51:27 +0200 berghofe Added some more lemmas that are useful in proof of strong induction rule.
Fri, 26 Sep 2008 09:10:02 +0200 haftmann removed obsolete name convention "func"
Fri, 26 Sep 2008 09:09:53 +0200 haftmann fixed typo
Fri, 26 Sep 2008 09:09:52 +0200 haftmann clarified function transformator interface
(0) -10000 -3000 -1000 -240 +240 +1000 +3000 +10000 +30000 tip