Fri, 10 Oct 1997 15:47:41 +0200 wenzelm added longid syntax;
Fri, 10 Oct 1997 15:46:50 +0200 wenzelm added longid;
Fri, 10 Oct 1997 15:44:48 +0200 wenzelm decode: qualified is always const;
Fri, 10 Oct 1997 14:51:58 +0200 wenzelm tuned;
Thu, 09 Oct 1997 18:01:27 +0200 wenzelm \n at end;
Thu, 09 Oct 1997 17:45:03 +0200 wenzelm ensure that dots in formulas are followed by non-idents;
Thu, 09 Oct 1997 17:20:15 +0200 wenzelm *** empty log message ***
Thu, 09 Oct 1997 15:06:49 +0200 wenzelm no longer handles consts "" -- use syntax instead;
Thu, 09 Oct 1997 15:04:21 +0200 wenzelm removed open;
Thu, 09 Oct 1997 15:03:06 +0200 wenzelm fixed infix syntax;
Thu, 09 Oct 1997 15:01:11 +0200 wenzelm added TLA stuff;
Thu, 09 Oct 1997 15:00:41 +0200 wenzelm fixed oracle;
Thu, 09 Oct 1997 14:59:36 +0200 wenzelm removed declIffOracle;
Thu, 09 Oct 1997 14:56:52 +0200 wenzelm changed preference order of prtab entries;
Thu, 09 Oct 1997 14:55:24 +0200 wenzelm fixed infix syntax;
Thu, 09 Oct 1997 14:55:05 +0200 wenzelm improved oracles: named, many per theory;
Thu, 09 Oct 1997 14:53:31 +0200 wenzelm improved oracle: name;
Thu, 09 Oct 1997 14:52:36 +0200 wenzelm fixed get_axiom, invoke_oracle;
Thu, 09 Oct 1997 14:51:10 +0200 wenzelm print_theory: added oracles;
Thu, 09 Oct 1997 14:50:39 +0200 wenzelm tuned exports;
Thu, 09 Oct 1997 14:39:44 +0200 wenzelm fixed axiom names;
Wed, 08 Oct 1997 12:15:59 +0200 wenzelm symbols syntax;
Wed, 08 Oct 1997 11:50:33 +0200 wenzelm A formalization of TLA in HOL -- by Stephan Merz;
Tue, 07 Oct 1997 18:02:42 +0200 wenzelm improved types of add_XXX funs (xtyp etc.);
Tue, 07 Oct 1997 18:02:02 +0200 wenzelm improved types of add_XXX funs (xtyp etc.);
Tue, 07 Oct 1997 17:58:50 +0200 wenzelm tuned decode;
Tue, 07 Oct 1997 17:58:01 +0200 wenzelm tuned internal mapping table;
Tue, 07 Oct 1997 17:08:48 +0200 wenzelm tuned;
Tue, 07 Oct 1997 17:06:05 +0200 wenzelm tuned warning msg;
Tue, 07 Oct 1997 12:37:53 +0200 wenzelm tuned;
Tue, 07 Oct 1997 12:29:34 +0200 wenzelm The Isabelle Logo;
Mon, 06 Oct 1997 20:00:31 +0200 wenzelm fixed 'begin';
Mon, 06 Oct 1997 19:39:40 +0200 wenzelm optional begin keyword;
Mon, 06 Oct 1997 19:16:57 +0200 wenzelm "->" made syntax;
Mon, 06 Oct 1997 19:15:22 +0200 wenzelm eliminated raise_term;
Mon, 06 Oct 1997 19:15:02 +0200 wenzelm eliminated raise_term, raise_typ;
Mon, 06 Oct 1997 19:13:55 +0200 wenzelm add_arities_i;
Mon, 06 Oct 1997 19:13:29 +0200 wenzelm TODO: handle internal / external names;
Mon, 06 Oct 1997 19:11:56 +0200 wenzelm now supports qualified names (intern vs. extern) !!!
Mon, 06 Oct 1997 19:07:14 +0200 wenzelm eliminated raise_term, raise_typ;
Mon, 06 Oct 1997 18:59:49 +0200 wenzelm tuned read_cterms;
Mon, 06 Oct 1997 18:57:17 +0200 wenzelm eliminated raise_term, raise_typ;
Mon, 06 Oct 1997 18:43:32 +0200 wenzelm new internal forms: add_classes_i, add_classrel_i, add_defsort_i, add_arities_i
Mon, 06 Oct 1997 18:41:39 +0200 wenzelm tuned;
Mon, 06 Oct 1997 18:41:09 +0200 wenzelm now uses new Sign.pretty_sort;
Mon, 06 Oct 1997 18:40:24 +0200 wenzelm eliminated raise_term, raise_typ;
Mon, 06 Oct 1997 18:39:54 +0200 wenzelm now uses Syntax.simple_str_of_sort;
Mon, 06 Oct 1997 18:39:25 +0200 wenzelm added simple_str_of_sort;
Mon, 06 Oct 1997 18:29:43 +0200 wenzelm eliminated raise_term;
Mon, 06 Oct 1997 18:29:11 +0200 wenzelm added 'path' section;
Mon, 06 Oct 1997 18:27:55 +0200 wenzelm added pretty_sort;
Mon, 06 Oct 1997 18:25:04 +0200 wenzelm fixed raw_term_sorts (again!);
Mon, 06 Oct 1997 18:23:13 +0200 wenzelm eliminated raise_ast, raise_term, raise_typ;
Mon, 06 Oct 1997 18:22:22 +0200 wenzelm added sort_to_ast;
Mon, 06 Oct 1997 18:21:00 +0200 wenzelm eliminated raise_ast;
Mon, 06 Oct 1997 18:20:15 +0200 wenzelm RAW target;
Mon, 06 Oct 1997 09:26:00 +0200 wenzelm syntactic constants;
Fri, 03 Oct 1997 10:32:50 +0200 paulson Routine tidying up
Thu, 02 Oct 1997 22:54:00 +0200 wenzelm fully qualified names: Theory.add_XXX;
Wed, 01 Oct 1997 18:19:44 +0200 wenzelm fully qualified name: Theory.set_oracle;
Wed, 01 Oct 1997 18:19:18 +0200 wenzelm exported separator;
Wed, 01 Oct 1997 18:13:41 +0200 wenzelm fully qualified names: Theory.add_XXX;
Wed, 01 Oct 1997 17:43:42 +0200 wenzelm moved theory stuff (add_defs etc.) here from drule.ML;
Wed, 01 Oct 1997 17:42:32 +0200 wenzelm moved theory stuff (add_defs etc.) to theory.ML;
Wed, 01 Oct 1997 17:41:20 +0200 wenzelm fully qualified name: Theory.merge_thy_list;
Wed, 01 Oct 1997 17:40:09 +0200 wenzelm fully qualified names: Theory.add_XXX;
Wed, 01 Oct 1997 17:36:51 +0200 wenzelm added name_space.ML;
Wed, 01 Oct 1997 17:32:38 +0200 wenzelm added split_last;
Wed, 01 Oct 1997 14:30:38 +0200 wenzelm Hierarchically structured name spaces.
Wed, 01 Oct 1997 13:42:18 +0200 paulson Strengthened the possibility property for resumption so that it could have
Wed, 01 Oct 1997 13:41:38 +0200 paulson Fixed ServerResume to check for ServerHello instead of making a new NB
Wed, 01 Oct 1997 12:07:24 +0200 paulson Exchanged the M and SID fields of the FINISHED messages to simplify proofs;
Wed, 01 Oct 1997 12:07:07 +0200 paulson Exchanged the M and SID fields of the FINISHED messages to simplify proofs
Wed, 01 Oct 1997 11:30:55 +0200 paulson Auto update
Tue, 30 Sep 1997 17:33:16 +0200 berghofe SYNC
Tue, 30 Sep 1997 17:32:33 +0200 berghofe Removed "browse.tex".
Tue, 30 Sep 1997 17:31:19 +0200 berghofe Added section describing the theory browser.
Tue, 30 Sep 1997 17:29:32 +0200 berghofe Updated usage information for tool "usedir".
Tue, 30 Sep 1997 17:28:54 +0200 berghofe Theory browser stuff has been moved to "present.tex".
Tue, 30 Sep 1997 16:19:27 +0200 wenzelm obsolete;
Tue, 30 Sep 1997 16:12:38 +0200 wenzelm ISABELLE_USEDIR_OPTIONS="-i true"
Tue, 30 Sep 1997 12:53:54 +0200 berghofe Changed html data directory and names of graph files.
Tue, 30 Sep 1997 12:52:15 +0200 berghofe There is now one single option -i for generating theory browsing
Tue, 30 Sep 1997 12:49:16 +0200 berghofe Modified some links.
Tue, 30 Sep 1997 11:03:55 +0200 paulson Client, Server certificates now sent using the separate Certificate rule,
Mon, 29 Sep 1997 15:39:28 +0200 wenzelm tuned;
Mon, 29 Sep 1997 15:16:22 +0200 wenzelm superficial;
Mon, 29 Sep 1997 15:11:27 +0200 wenzelm obsolete;
Mon, 29 Sep 1997 15:08:47 +0200 wenzelm margin 76 (2nd try :-);
Mon, 29 Sep 1997 14:12:02 +0200 wenzelm fixed href to html library;
Mon, 29 Sep 1997 14:11:18 +0200 wenzelm improved warning;
Mon, 29 Sep 1997 14:10:52 +0200 wenzelm default margin 76 (to accomodate warning and error default output);
Mon, 29 Sep 1997 12:13:43 +0200 paulson Step_tac -> Safe_tac
Mon, 29 Sep 1997 11:56:04 +0200 paulson Much tidying including step_tac -> clarify_tac or safe_tac; sometimes
Mon, 29 Sep 1997 11:52:25 +0200 paulson Step_tac -> Safe_tac
Mon, 29 Sep 1997 11:51:52 +0200 paulson Much tidying including "qed" instead of result(), and even qed_spec_mp,
Mon, 29 Sep 1997 11:51:09 +0200 paulson Previously loaded the WRONG THEORY, ignoring Confluence...
Mon, 29 Sep 1997 11:49:33 +0200 paulson Now using qed_spec_mp
Mon, 29 Sep 1997 11:48:48 +0200 paulson result() -> qed; Step_tac -> Safe_tac
Mon, 29 Sep 1997 11:47:01 +0200 paulson Step_tac -> Safe_tac
Mon, 29 Sep 1997 11:46:33 +0200 paulson Renamed XA, XB to PA, PB and removed the certificate from Client Verify
Mon, 29 Sep 1997 11:45:52 +0200 paulson Default simpset tactics now dereference "simpset"
Mon, 29 Sep 1997 11:44:56 +0200 paulson Added Safe_tac; all other default claset tactics now dereference "claset"
Mon, 29 Sep 1997 11:42:15 +0200 paulson fast_tac HOL_cs -> Fast_tac, etc.
Mon, 29 Sep 1997 11:40:03 +0200 paulson result() -> qed
Mon, 29 Sep 1997 11:37:02 +0200 paulson Step_tac -> Safe_tac
Mon, 29 Sep 1997 11:36:44 +0200 paulson Tidied proof of r_comp_rtrancl_eq
Mon, 29 Sep 1997 11:32:25 +0200 paulson qed_spec_mp, normalize_thm, etc. copied in from HOL.ML
Mon, 29 Sep 1997 11:31:56 +0200 paulson Step_tac -> Safe_tac
Mon, 29 Sep 1997 11:31:13 +0200 paulson Safe_tac, Safe_step_tac, and minor corrections including \tt -> \texttt
Mon, 29 Sep 1997 11:28:23 +0200 paulson Safe_tac; qed_spec_mp in FOL
Fri, 26 Sep 1997 10:21:14 +0200 paulson Minor tidying to use Clarify_tac, etc.
Fri, 26 Sep 1997 10:12:04 +0200 wenzelm eliminated rules;
Thu, 25 Sep 1997 13:25:50 +0200 paulson Clarify_tac and some textual improvements
Thu, 25 Sep 1997 13:23:41 +0200 paulson Clarify_tac; general reorganization
Thu, 25 Sep 1997 12:32:14 +0200 paulson Deleted obsolete version of clarify_tac
Thu, 25 Sep 1997 12:25:29 +0200 paulson Deleted the unused list_mk_disj
Thu, 25 Sep 1997 12:24:53 +0200 paulson Deleted the unused gtake and recoded enumerate to use foldl
Thu, 25 Sep 1997 12:20:24 +0200 paulson Deleted an obsolete step in TrustServerFinished
Thu, 25 Sep 1997 12:19:41 +0200 paulson Deleted obsolete axioms inj_serverK and isSym_serverK
Thu, 25 Sep 1997 12:14:41 +0200 paulson Tidied proofs, using Clarify_tac
Thu, 25 Sep 1997 12:13:18 +0200 paulson Changed some proofs to use Clarify_tac
Thu, 25 Sep 1997 12:10:07 +0200 paulson Prints warnings using the "warning" function instead of "writeln"
Thu, 25 Sep 1997 12:09:41 +0200 paulson Generalized and exported biresolution_from_nets_tac to allow the declaration
Thu, 25 Sep 1997 12:08:08 +0200 paulson Addition of clarify_tac, clarify_step_tac, Clarify_tac, Clarify_step_tac
Wed, 24 Sep 1997 12:27:53 +0200 paulson sessionK now indexed by nat instead of bool.
Wed, 24 Sep 1997 12:26:14 +0200 paulson Tidied some proofs using clarify_tac
Wed, 24 Sep 1997 12:25:32 +0200 paulson clarify_tac and a new simprule
Wed, 24 Sep 1997 12:24:41 +0200 paulson Names and saves the theorem parts_spies_subset_used
Wed, 24 Sep 1997 10:51:52 +0200 wenzelm pure_trfuns: added constraint;
Tue, 23 Sep 1997 17:35:07 +0200 wenzelm added handle_error: ('a -> 'b) -> 'a -> 'b error;
Tue, 23 Sep 1997 08:44:57 +0200 wenzelm index.html obsolete;
Mon, 22 Sep 1997 17:38:55 +0200 wenzelm Pure: fixed idt/idts vs. pttrn/pttrns syntactic categories;
Mon, 22 Sep 1997 17:37:48 +0200 wenzelm acks;
Mon, 22 Sep 1997 17:37:24 +0200 wenzelm added Cambridge fs;
Mon, 22 Sep 1997 17:37:03 +0200 wenzelm fixed pttrn syntax;
Mon, 22 Sep 1997 17:35:52 +0200 wenzelm fixed LAM <x,y,zs>.b syntax (may break some unusual cases);
Mon, 22 Sep 1997 17:31:57 +0200 wenzelm tuned pattern syntax;
Mon, 22 Sep 1997 17:31:28 +0200 wenzelm tuned lambda_ast_tr, idtyp_ast_tr' to accomodate fix of idt/idts
Mon, 22 Sep 1997 17:29:42 +0200 wenzelm fixed idt/idts vs. pttrn/pttrns;
Mon, 22 Sep 1997 16:08:45 +0200 paulson Added Cambridge font server
Mon, 22 Sep 1997 14:46:56 +0200 wenzelm obsolete;
Mon, 22 Sep 1997 13:17:29 +0200 paulson Simplified SpyKeys to use sessionK instead of clientK and serverK
Fri, 19 Sep 1997 18:27:31 +0200 paulson First working version with Oops event for session keys
Fri, 19 Sep 1997 16:12:21 +0200 paulson Full version of TLS including session resumption, but no Oops
Fri, 19 Sep 1997 16:11:24 +0200 paulson Deleted the obsolete theorem analz_UN1_synth
Thu, 18 Sep 1997 13:24:04 +0200 paulson Global change: lost->bad and sees Spy->spies
Wed, 17 Sep 1997 16:40:52 +0200 paulson Deleted the redundant identifier Says_imp_sees_Spy'
Wed, 17 Sep 1997 16:39:43 +0200 paulson New proof of respond_Spy_not_see_session_key
Wed, 17 Sep 1997 16:38:34 +0200 paulson Removed the simprule imp_disjL from the analz_image_..._ss to boost speed
Wed, 17 Sep 1997 16:37:40 +0200 paulson Fixed comments
Wed, 17 Sep 1997 16:37:27 +0200 paulson Spy can see Notes of the compromised agents
Wed, 17 Sep 1997 16:37:21 +0200 paulson Now with the sessionK constant and new events ClientAccepts and ServerAccepts
Tue, 16 Sep 1997 14:40:01 +0200 paulson Addition of SessionIDs to the Hello and Finished messages
Tue, 16 Sep 1997 14:04:10 +0200 paulson Deleted the redundant simprule not_parts_not_analz
Tue, 16 Sep 1997 13:58:02 +0200 paulson Deleted the redundant simprule not_parts_not_analz
Tue, 16 Sep 1997 13:54:41 +0200 paulson Having "addcongs [if_weak_cong]" in analz_image_..._ss makes simplification
Tue, 16 Sep 1997 13:32:22 +0200 paulson TLS now with a distinction between premaster secret and master secret
Fri, 12 Sep 1997 10:45:51 +0200 mueller extended adm_tac;
Thu, 11 Sep 1997 16:20:56 +0200 wenzelm replaced print_goals_ref hook by print_current_goals_fn and
Thu, 11 Sep 1997 16:16:03 +0200 wenzelm removed print_goals_ref (which was broken anyway);
Thu, 11 Sep 1997 12:24:28 +0200 paulson Split base cases from "msg" to "atomic" in order
Thu, 11 Sep 1997 12:22:31 +0200 paulson Now uses the generic induct_tac
Thu, 11 Sep 1997 12:21:34 +0200 paulson auto update
Wed, 10 Sep 1997 14:18:12 +0200 nipkow Added Larry's test for preventing a datatype shadowing a theory.
Tue, 09 Sep 1997 12:09:06 +0200 nipkow Example from HOLCF paper.
Tue, 09 Sep 1997 12:08:28 +0200 nipkow Loads HoareEx now.
Tue, 09 Sep 1997 11:15:32 +0200 mueller adm_tac extended
Tue, 09 Sep 1997 11:14:20 +0200 mueller moved extended adm_tac to new place
Mon, 08 Sep 1997 10:12:28 +0200 paulson added ".ML" extension in "use" command
Fri, 05 Sep 1997 12:24:13 +0200 paulson Renamed "evs" to "evs1", "evs2", etc. in protocol inductive definition
Thu, 04 Sep 1997 17:57:56 +0200 paulson set_of_list
Thu, 04 Sep 1997 17:43:16 +0200 paulson Deleted an obsolete description of rewrite_cterm. The current version uses
Wed, 03 Sep 1997 16:25:30 +0200 mueller some minor changes;
Wed, 03 Sep 1997 16:24:46 +0200 mueller new extended adm tactic introduced;
Tue, 02 Sep 1997 17:02:02 +0200 nipkow Added True_implies_equals
Tue, 02 Sep 1997 16:10:26 +0200 nipkow Added Larry's equal_intr_rule
Tue, 02 Sep 1997 11:25:32 +0200 oheimb added case_prover
Thu, 21 Aug 1997 12:57:24 +0200 paulson Simplified the statement of A_trusts_NS2
Thu, 21 Aug 1997 12:56:29 +0200 paulson Replacing impOfSubs analz_mono by analz_insertI should improve convergence
Thu, 21 Aug 1997 12:55:10 +0200 paulson Renamed set_of_list to set, and relevant theorems too
Thu, 21 Aug 1997 12:54:20 +0200 paulson Replaced Suc(Suc 0) by 2; it improves readability a little
Thu, 21 Aug 1997 12:53:23 +0200 paulson Renamed theorems of the form set_of_list_XXX to set_XXX
Sun, 10 Aug 1997 12:28:34 +0200 nipkow Added select1_equality
Fri, 08 Aug 1997 11:22:59 +0200 wenzelm added append_file;
Fri, 08 Aug 1997 00:11:11 +0200 berghofe This file has moved to Distribution/lib/images.
Fri, 08 Aug 1997 00:09:26 +0200 berghofe This file has moved to Distribution/lib/html.
Thu, 07 Aug 1997 23:48:29 +0200 berghofe Removed references to simplifier.
Thu, 07 Aug 1997 23:46:36 +0200 berghofe Modified parse error message.
Thu, 07 Aug 1997 23:45:24 +0200 berghofe Startup script for Isabelle theory browser.
Thu, 07 Aug 1997 23:43:30 +0200 berghofe Modified graph data directory.
Thu, 07 Aug 1997 23:39:28 +0200 berghofe Added some commands for building theory browser.
Thu, 07 Aug 1997 23:37:53 +0200 berghofe Added new environment variable ISABELLE_BROWSER_INFO.
Thu, 07 Aug 1997 23:35:32 +0200 berghofe Added some code for generating theory browsing data.
Thu, 07 Aug 1997 23:34:31 +0200 berghofe Gif images which are copied to $ISABELLE_BROWSER_INFO when
Thu, 07 Aug 1997 23:32:24 +0200 berghofe Index file which is copied to $ISABELLE_BROWSER_INFO
Wed, 06 Aug 1997 15:07:53 +0200 wenzelm added str_of_classrel;
Wed, 06 Aug 1997 15:07:33 +0200 wenzelm added "Proving ..." msgs;
Wed, 06 Aug 1997 14:42:44 +0200 wenzelm renamed use_string to use_strings;
Wed, 06 Aug 1997 14:35:52 +0200 wenzelm removed smlnj-1.07;
Wed, 06 Aug 1997 14:15:05 +0200 wenzelm prs instead of TextIO.output;
Wed, 06 Aug 1997 14:12:29 +0200 wenzelm tuned copy_file;
Wed, 06 Aug 1997 14:12:03 +0200 wenzelm tuned names;
Wed, 06 Aug 1997 14:11:08 +0200 wenzelm tuned;
Wed, 06 Aug 1997 14:10:22 +0200 wenzelm ThmDatabase;
Wed, 06 Aug 1997 14:09:50 +0200 wenzelm added read_file, write_file;
Wed, 06 Aug 1997 11:58:50 +0200 wenzelm tuned;
Wed, 06 Aug 1997 11:57:52 +0200 wenzelm use ThySyn.add_syntax;
Wed, 06 Aug 1997 11:57:20 +0200 wenzelm tuned comments;
Wed, 06 Aug 1997 11:56:31 +0200 wenzelm oops;
Wed, 06 Aug 1997 11:52:16 +0200 wenzelm eliminated ThySynData and ThySynFun;
Wed, 06 Aug 1997 11:19:59 +0200 wenzelm obsolete!
Wed, 06 Aug 1997 01:18:31 +0200 berghofe Replaced "init_thy_reader" by "set_parser".
Wed, 06 Aug 1997 01:17:42 +0200 berghofe Removed references to "thy_data.ML".
Wed, 06 Aug 1997 01:13:46 +0200 berghofe Moved some functions which used to be part of thy_data.ML
Wed, 06 Aug 1997 01:12:03 +0200 berghofe Moved functions contained in this file to HOL.ML, datatype.ML,
Wed, 06 Aug 1997 00:47:20 +0200 berghofe Replaced "init_thy_reader" by "set_parser".
Wed, 06 Aug 1997 00:45:09 +0200 berghofe Removed reference to "thy_data.ML".
Wed, 06 Aug 1997 00:44:25 +0200 berghofe The functions in this file have been moved to "cladata.ML"
Wed, 06 Aug 1997 00:41:40 +0200 berghofe Moved functions from file "thy_data.ML".
Wed, 06 Aug 1997 00:39:13 +0200 berghofe Replaced "init_thy_reader" by "set_parser".
Wed, 06 Aug 1997 00:37:21 +0200 berghofe Replaced "init_thy_reader" by set_parser.
Wed, 06 Aug 1997 00:33:13 +0200 berghofe Added some new dependencies for files in subdirectory Thy.
Wed, 06 Aug 1997 00:29:54 +0200 berghofe Added function "file_exists".
Wed, 06 Aug 1997 00:29:02 +0200 berghofe Removed function file_exists (now included in library.ML)
Wed, 06 Aug 1997 00:26:19 +0200 berghofe Moved functions for theory information storage / retrieval
Wed, 06 Aug 1997 00:24:49 +0200 berghofe This file now contains all functions for generating html
Wed, 06 Aug 1997 00:23:01 +0200 berghofe Moved several functions:
Wed, 06 Aug 1997 00:18:34 +0200 berghofe Moved "qed" - functions etc. from thy_read.ML to thm_database.ML.
Wed, 06 Aug 1997 00:15:14 +0200 berghofe Added some additional "use" commands for new files
Wed, 06 Aug 1997 00:06:47 +0200 berghofe Source files for Isabelle theory graph browser.
Wed, 06 Aug 1997 00:04:53 +0200 berghofe Makefile for GraphBrowser
Tue, 05 Aug 1997 17:26:01 +0200 wenzelm added getenv;
Tue, 05 Aug 1997 17:21:24 +0200 wenzelm removed smlnj-1.07;
Tue, 05 Aug 1997 17:03:11 +0200 wenzelm cleaned up;
Tue, 05 Aug 1997 17:02:50 +0200 wenzelm tuned comments;
Tue, 05 Aug 1997 17:01:02 +0200 wenzelm removed ML-Systems/smlnj-1.07.ML;
Tue, 05 Aug 1997 16:44:46 +0200 wenzelm SML/NJ 1.07 no longer supported!
Tue, 05 Aug 1997 16:43:54 +0200 wenzelm cleaned up;
Tue, 05 Aug 1997 16:22:17 +0200 nipkow Added example mapf which requires a special congruence rule.
(0) -3000 -1000 -240 +240 +1000 +3000 +10000 +30000 tip