Wed, 02 Nov 2005 11:02:29 +0100 urbanc added the collection of lemmas "supp_at"
Tue, 01 Nov 2005 23:55:53 +0100 urbanc some minor tweaks in some proofs (nothing extraordinary)
Tue, 01 Nov 2005 23:54:29 +0100 urbanc tunings of some comments (nothing serious)
Mon, 31 Oct 2005 16:35:15 +0100 haftmann nth_*, fold_index refined
Mon, 31 Oct 2005 16:00:15 +0100 haftmann fold_index replacing foldln
Mon, 31 Oct 2005 01:43:22 +0100 nipkow A few new lemmas
Sun, 30 Oct 2005 10:55:56 +0100 urbanc tuned my last commit
Sun, 30 Oct 2005 10:37:57 +0100 urbanc simplified the abs_supp_approx proof and tuned some comments in
Sat, 29 Oct 2005 15:01:25 +0200 urbanc Changed Simplifier.simp_modifiers to Simplifier.simp_modifiers'.
Sat, 29 Oct 2005 14:37:32 +0200 urbanc 1) have adjusted the swapping of the result type
Fri, 28 Oct 2005 22:37:57 +0200 wenzelm tuned;
Fri, 28 Oct 2005 22:32:55 +0200 wenzelm lthms_containing: not o valid_thms;
Fri, 28 Oct 2005 22:28:15 +0200 wenzelm added fact_tac, some_fact_tac;
Fri, 28 Oct 2005 22:28:13 +0200 wenzelm renamed Goal constant to prop, more general protect/unprotect interfaces;
Fri, 28 Oct 2005 22:28:12 +0200 wenzelm renamed Goal constant to prop, more general protect/unprotect interfaces;
Fri, 28 Oct 2005 22:28:11 +0200 wenzelm added fact method;
Fri, 28 Oct 2005 22:28:09 +0200 wenzelm tuned ProofContext.export interfaces;
Fri, 28 Oct 2005 22:28:07 +0200 wenzelm syntax for literal facts;
Fri, 28 Oct 2005 22:28:06 +0200 wenzelm removed try_dest_Goal, use Logic.unprotect;
Fri, 28 Oct 2005 22:28:04 +0200 wenzelm added cgoal_of;
Fri, 28 Oct 2005 22:28:03 +0200 wenzelm accomodate simplified Thm.lift_rule;
Fri, 28 Oct 2005 22:28:02 +0200 wenzelm export cong_modifiers, simp_modifiers';
Fri, 28 Oct 2005 22:28:00 +0200 wenzelm certify_term: tuned monomorphic consts;
Fri, 28 Oct 2005 22:27:59 +0200 wenzelm datatype thmref: added Fact;
Fri, 28 Oct 2005 22:27:58 +0200 wenzelm Logic.lift_all;
Fri, 28 Oct 2005 22:27:57 +0200 wenzelm renamed Goal constant to prop, more general protect/unprotect interfaces;
Fri, 28 Oct 2005 22:27:56 +0200 wenzelm renamed Goal.norm_hhf_rule to Goal.norm_hhf;
Fri, 28 Oct 2005 22:27:55 +0200 wenzelm renamed Goal constant to prop, more general protect/unprotect interfaces;
Fri, 28 Oct 2005 22:27:54 +0200 wenzelm added add_local/add_global;
Fri, 28 Oct 2005 22:27:52 +0200 wenzelm added incr_indexes;
Fri, 28 Oct 2005 22:27:51 +0200 wenzelm renamed Goal constant to prop;
Fri, 28 Oct 2005 22:27:47 +0200 wenzelm accomodate simplified Thm.lift_rule;
Fri, 28 Oct 2005 22:27:46 +0200 wenzelm Logic.unprotect;
Fri, 28 Oct 2005 22:27:44 +0200 wenzelm literal facts;
Fri, 28 Oct 2005 22:27:41 +0200 wenzelm * Pure/Isar: literal facts;
Fri, 28 Oct 2005 22:26:10 +0200 wenzelm tuned;
Fri, 28 Oct 2005 20:18:37 +0200 webertj unnecessary imports removed
Fri, 28 Oct 2005 18:53:26 +0200 urbanc fixed case names in the weak induction principle and
Fri, 28 Oct 2005 18:22:26 +0200 berghofe Implemented proof of weak induction theorem.
Fri, 28 Oct 2005 17:59:07 +0200 berghofe Added "deepen" method.
Fri, 28 Oct 2005 17:27:49 +0200 haftmann circumvented smlnj value restriction
Fri, 28 Oct 2005 17:27:04 +0200 haftmann added extraction interface for code generator
Fri, 28 Oct 2005 16:43:46 +0200 urbanc Added (optional) arguments to the tactics
Fri, 28 Oct 2005 16:35:40 +0200 haftmann cleaned up nth, nth_update, nth_map and nth_string functions
Fri, 28 Oct 2005 13:52:57 +0200 berghofe Removed legacy prove_goalw_cterm command.
Fri, 28 Oct 2005 12:22:34 +0200 paulson got rid of obsolete prove_goalw_cterm
Fri, 28 Oct 2005 09:36:19 +0200 haftmann swapped add_datatype result
Fri, 28 Oct 2005 09:35:04 +0200 haftmann removed obfuscating PStrStrTab
Fri, 28 Oct 2005 08:40:55 +0200 haftmann reachable - abandoned foldl_map in favor of fold_map
Fri, 28 Oct 2005 02:30:53 +0200 mengj Added Tools/res_hol_clause.ML
Fri, 28 Oct 2005 02:30:12 +0200 mengj Added a new file res_hol_clause.ML to Reconstruction.thy. This file is used to translate HOL formulae into FOL clauses.
Fri, 28 Oct 2005 02:29:01 +0200 mengj Added "writeln_strs" to the signature
Fri, 28 Oct 2005 02:28:20 +0200 mengj Added several new functions that are used to prove HOL goals. Added new methods "vampireH" and "eproverH" that can prove both FOL and HOL goals. The old "vampire" and "eprover" methods are renamed to "vampireF" and "eproverF"; they can only prove FOL goals.
Fri, 28 Oct 2005 02:27:19 +0200 mengj Added new functions to handle HOL goals and lemmas.
Fri, 28 Oct 2005 02:25:57 +0200 mengj Added several new functions that convert HOL Isabelle rules to FOL axiom clauses. The original functions that convert FOL rules to clauses stay with the same names; the new functions have "H" at the end of their names.
Fri, 28 Oct 2005 02:24:58 +0200 mengj Added several functions to the signature.
Fri, 28 Oct 2005 02:23:49 +0200 mengj A new file that defines datatypes representing FOL clauses that are derived from HOL formulae. This file also has functions that convert lambda terms to combinator expressions, and functions that convert clauses to TPTP format.
Thu, 27 Oct 2005 18:25:33 +0200 paulson sorted lemma lists
Thu, 27 Oct 2005 13:59:06 +0200 wenzelm * HOL: alternative iff syntax;
Thu, 27 Oct 2005 13:54:43 +0200 wenzelm consts: monomorphic;
Thu, 27 Oct 2005 13:54:42 +0200 wenzelm removed inappropriate monomorphic test;
Thu, 27 Oct 2005 13:54:40 +0200 wenzelm replaced Defs.monomorphic by Sign.monomorphic;
Thu, 27 Oct 2005 13:54:38 +0200 wenzelm alternative iff syntax for equality on booleans, with print_mode 'iff';
Thu, 27 Oct 2005 08:14:05 +0200 haftmann added module Pure/General/rat.ML
Wed, 26 Oct 2005 16:31:53 +0200 paulson tidied away duplicate thm
Tue, 25 Oct 2005 18:38:21 +0200 wenzelm EVERY;
Tue, 25 Oct 2005 18:18:59 +0200 wenzelm traceIt: plain term;
Tue, 25 Oct 2005 18:18:58 +0200 wenzelm val legacy = ref false;
Tue, 25 Oct 2005 18:18:57 +0200 wenzelm prove_raw: cterms, explicit asms;
Tue, 25 Oct 2005 18:18:49 +0200 wenzelm avoid legacy goals;
Sat, 22 Oct 2005 01:22:10 +0200 wenzelm legacy = ref true for the time being -- avoid volumious warnings;
Fri, 21 Oct 2005 18:20:29 +0200 wenzelm tuned;
Fri, 21 Oct 2005 18:17:00 +0200 wenzelm avoid OldGoals shortcuts;
Fri, 21 Oct 2005 18:16:57 +0200 wenzelm * Legacy goal package: reduced interface to the bare minimum required to keep existing proof scripts running.
Fri, 21 Oct 2005 18:15:00 +0200 wenzelm Internal goals.
Fri, 21 Oct 2005 18:14:59 +0200 wenzelm renamed triv_goal to goalI, rev_triv_goal to goalD;
Fri, 21 Oct 2005 18:14:58 +0200 wenzelm tuned header;
Fri, 21 Oct 2005 18:14:57 +0200 wenzelm Goal.norm_hhf_rule;
Fri, 21 Oct 2005 18:14:56 +0200 wenzelm export add_binds_i;
Fri, 21 Oct 2005 18:14:55 +0200 wenzelm load_file: setmp OldGoals.legacy true;
Fri, 21 Oct 2005 18:14:54 +0200 wenzelm improved check_result;
Fri, 21 Oct 2005 18:14:53 +0200 wenzelm Goal.prove_plain;
Fri, 21 Oct 2005 18:14:52 +0200 wenzelm do not export find_thms;
Fri, 21 Oct 2005 18:14:51 +0200 wenzelm use obsolete goals.ML here;
Fri, 21 Oct 2005 18:14:50 +0200 wenzelm Goal.conclude;
Fri, 21 Oct 2005 18:14:49 +0200 wenzelm moved SELECT_GOAL to goal.ML;
Fri, 21 Oct 2005 18:14:48 +0200 wenzelm moved norm_hhf_rule, prove etc. to goal.ML;
Fri, 21 Oct 2005 18:14:47 +0200 wenzelm added simplification tactics and rules (from meta_simplifier.ML);
Fri, 21 Oct 2005 18:14:46 +0200 wenzelm moved various simplification tactics and rules to simplifier.ML;
Fri, 21 Oct 2005 18:14:45 +0200 wenzelm warn_obsolete for goal commands -- danger of disrupting a local proof context;
Fri, 21 Oct 2005 18:14:44 +0200 wenzelm renamed triv_goal to goalI, rev_triv_goal to goalD;
Fri, 21 Oct 2005 18:14:43 +0200 wenzelm added goal.ML;
Fri, 21 Oct 2005 18:14:42 +0200 wenzelm added goal.ML;
Fri, 21 Oct 2005 18:14:41 +0200 wenzelm Goal.norm_hhf_rule, Goal.init;
Fri, 21 Oct 2005 18:14:40 +0200 wenzelm avoid triv_goal and home-grown meta_allE;
Fri, 21 Oct 2005 18:14:38 +0200 wenzelm OldGoals;
Fri, 21 Oct 2005 18:14:37 +0200 wenzelm proper header;
Fri, 21 Oct 2005 18:14:36 +0200 wenzelm avoid home-grown meta_allE;
Fri, 21 Oct 2005 18:14:34 +0200 wenzelm Goal.prove;
Fri, 21 Oct 2005 18:14:32 +0200 wenzelm avoid shortcuts from OldGoals;
Fri, 21 Oct 2005 16:34:22 +0200 wenzelm added simplified settings for Poly/ML 4.x (commented out);
Fri, 21 Oct 2005 16:22:59 +0200 wenzelm reverted (accidental?) change of 1.148;
Fri, 21 Oct 2005 14:49:49 +0200 haftmann abandoned rational number functions in favor of General/rat.ML
Fri, 21 Oct 2005 14:49:04 +0200 haftmann introduced functions from Pure/General/rat.ML
Fri, 21 Oct 2005 14:47:37 +0200 haftmann slight corrections
Fri, 21 Oct 2005 10:32:59 +0200 haftmann substantially improved integration of website into distribution framework
Fri, 21 Oct 2005 10:32:04 +0200 haftmann substantially improved integration of website into distribution framework
Fri, 21 Oct 2005 10:27:02 +0200 haftmann substantially improved integration of website into distribution framework
Fri, 21 Oct 2005 10:21:38 +0200 haftmann substantially improved integration of website into distribution framework
Fri, 21 Oct 2005 09:54:03 +0200 haftmann towards an improved website/makedist integration
Fri, 21 Oct 2005 09:18:27 +0200 haftmann towards an improved website/makedist integration
Fri, 21 Oct 2005 09:08:42 +0200 haftmann added default distinfo.mak
Fri, 21 Oct 2005 09:05:52 +0200 haftmann towards an improved website/makedist integration
Fri, 21 Oct 2005 09:05:52 +0200 haftmann towards an improved website/makedist integration
Fri, 21 Oct 2005 08:23:45 +0200 haftmann added rounding functions
Fri, 21 Oct 2005 02:57:22 +0200 mengj Merged theory ResAtpOracle.thy into ResAtpMethods.thy
Wed, 19 Oct 2005 21:53:34 +0200 wenzelm obsolete;
Wed, 19 Oct 2005 21:52:50 +0200 wenzelm removed add_inductive_x;
Wed, 19 Oct 2005 21:52:49 +0200 wenzelm removed obsolete add_datatype_x;
Wed, 19 Oct 2005 21:52:48 +0200 wenzelm removed obsolete thy_syntax.ML;
Wed, 19 Oct 2005 21:52:47 +0200 wenzelm removed obsolete old_symbol_source;
Wed, 19 Oct 2005 21:52:46 +0200 wenzelm removed obsolete non-Isar theory format and old Isar theory headers;
Wed, 19 Oct 2005 21:52:45 +0200 wenzelm removed old-style theory format;
Wed, 19 Oct 2005 21:52:44 +0200 wenzelm avoid lagacy read function;
Wed, 19 Oct 2005 21:52:43 +0200 wenzelm added thm(s) retrieval functions (from goals.ML);
Wed, 19 Oct 2005 21:52:42 +0200 wenzelm removed obsolete old-locales;
Wed, 19 Oct 2005 21:52:41 +0200 wenzelm removed obsolete axclass_tac, add_inst_subclass_x, add_inst_arity_x;
Wed, 19 Oct 2005 21:52:40 +0200 wenzelm removed obsolete Thy/thy_parse.ML, Thy/thy_scan.ML, Thy/thy_syn.ML;
Wed, 19 Oct 2005 21:52:38 +0200 wenzelm removed obsolete old-style syntax;
Wed, 19 Oct 2005 21:52:37 +0200 wenzelm removed obsolete IOA/meta_theory/ioa_package.ML;
Wed, 19 Oct 2005 21:52:36 +0200 wenzelm removed obsolete domain/interface.ML, IOA/meta_theory/ioa_package.ML;
Wed, 19 Oct 2005 21:52:35 +0200 wenzelm removed obsolete domain/interface.ML;
Wed, 19 Oct 2005 21:52:34 +0200 wenzelm removed obsolete add_typedef_x;
Wed, 19 Oct 2005 21:52:33 +0200 wenzelm removed print_exn (better let the toplevel do this);
Wed, 19 Oct 2005 21:52:32 +0200 wenzelm removed obsolete add_recdef_old;
Wed, 19 Oct 2005 21:52:31 +0200 wenzelm removed obsolete HOL/thy_syntax.ML;
Wed, 19 Oct 2005 21:52:30 +0200 wenzelm * Theory syntax: discontinued non-Isar format and old Isar headers;
Wed, 19 Oct 2005 21:52:29 +0200 wenzelm replaced commafy by existing commas;
Wed, 19 Oct 2005 21:52:28 +0200 wenzelm updated;
Wed, 19 Oct 2005 21:52:27 +0200 wenzelm isatool fixheaders;
Wed, 19 Oct 2005 21:52:07 +0200 wenzelm fix headers;
Wed, 19 Oct 2005 17:21:53 +0200 haftmann added table functor instance for pairs of strings
Wed, 19 Oct 2005 17:19:52 +0200 haftmann added subgraph
Wed, 19 Oct 2005 17:19:37 +0200 haftmann added join
Wed, 19 Oct 2005 16:32:09 +0200 haftmann slight improvements for website
Wed, 19 Oct 2005 14:51:12 +0200 wenzelm moved VAMPIRE_HOME, E_HOME to section "External reasoning tools" -- commented out by default!
Wed, 19 Oct 2005 13:59:33 +0200 mengj More functions are added to the signature of ResClause
Wed, 19 Oct 2005 10:25:46 +0200 mengj *** empty log message ***
Wed, 19 Oct 2005 06:46:45 +0200 nipkow added 2 lemmas
Wed, 19 Oct 2005 06:33:24 +0200 mengj Added files in order to use external ATPs as oracles and invoke these ATPs by calling Isabelle methods (currently "vampire" and "eprover").
Tue, 18 Oct 2005 17:59:37 +0200 wenzelm simplified interfaces proof/proof' etc.: perform ProofHistory.apply(s)/current internally;
Tue, 18 Oct 2005 17:59:36 +0200 wenzelm tuned error msg;
Tue, 18 Oct 2005 17:59:35 +0200 wenzelm renamed atomize_rule to atomize_cterm;
Tue, 18 Oct 2005 17:59:34 +0200 wenzelm ObjectLogic.atomize_cterm;
Tue, 18 Oct 2005 17:59:33 +0200 wenzelm use simplified Toplevel.proof etc.;
Tue, 18 Oct 2005 17:59:32 +0200 wenzelm back: Toplevel.actual/skip_proof;
Tue, 18 Oct 2005 17:59:31 +0200 wenzelm renamed set_context to context;
Tue, 18 Oct 2005 17:59:30 +0200 wenzelm renamed set_context to context;
Tue, 18 Oct 2005 17:59:29 +0200 wenzelm functor: no Simplifier argument;
Tue, 18 Oct 2005 17:59:28 +0200 wenzelm moved helper lemma to HilbertChoice.thy;
Tue, 18 Oct 2005 17:59:27 +0200 wenzelm Simplifier.theory_context;
Tue, 18 Oct 2005 17:59:26 +0200 wenzelm added lemma exE_some (from specification_package.ML);
Tue, 18 Oct 2005 17:59:25 +0200 wenzelm Simplifier.theory_context;
Tue, 18 Oct 2005 17:59:24 +0200 wenzelm tuned error msg;
Tue, 18 Oct 2005 17:59:23 +0200 wenzelm Simplifier.context/theory_context;
Tue, 18 Oct 2005 17:59:22 +0200 wenzelm updated;
Tue, 18 Oct 2005 15:08:38 +0200 paulson new interface to make_conjecture_clauses
Mon, 17 Oct 2005 23:10:25 +0200 wenzelm * Simplifier: simpset of a running simplification process contains a proof context;
Mon, 17 Oct 2005 23:10:24 +0200 wenzelm added type_solver (uses Simplifier.the_context);
Mon, 17 Oct 2005 23:10:23 +0200 wenzelm added pos/negDivAlg_induct declarations (from Main.thy);
Mon, 17 Oct 2005 23:10:22 +0200 wenzelm moved pos/negDivAlg_induct declarations to Integ/IntDiv.thy;
Mon, 17 Oct 2005 23:10:21 +0200 wenzelm removed obsolete/experimental context components (superceded by Simplifier.the_context);
Mon, 17 Oct 2005 23:10:20 +0200 wenzelm added set/addloop' for simpset dependent loopers;
Mon, 17 Oct 2005 23:10:19 +0200 wenzelm functor: no Simplifier argument;
Mon, 17 Oct 2005 23:10:18 +0200 wenzelm change_claset(_of): more abtract interface;
Mon, 17 Oct 2005 23:10:17 +0200 wenzelm functor: no Simplifier argument;
Mon, 17 Oct 2005 23:10:16 +0200 wenzelm tuned;
Mon, 17 Oct 2005 23:10:15 +0200 wenzelm Simplifier.inherit_context instead of Simplifier.inherit_bounds;
Mon, 17 Oct 2005 23:10:13 +0200 wenzelm change_claset/simpset;
Mon, 17 Oct 2005 23:10:10 +0200 wenzelm change_claset/simpset;
Mon, 17 Oct 2005 19:19:29 +0200 berghofe Improved proof of injectivity theorems to make it work on
Mon, 17 Oct 2005 18:34:51 +0200 berghofe Fixed bug in proof of support theorem (it failed on constructors with no arguments).
Mon, 17 Oct 2005 17:42:24 +0200 berghofe Implemented proofs for support and freshness theorems.
Mon, 17 Oct 2005 17:40:34 +0200 urbanc deleted leading space in the definition of fresh
Mon, 17 Oct 2005 12:30:57 +0200 berghofe Initial revision.
Sat, 15 Oct 2005 00:14:30 +0200 wenzelm tuned;
Sat, 15 Oct 2005 00:09:20 +0200 wenzelm tuned comment;
Sat, 15 Oct 2005 00:09:07 +0200 wenzelm added ML_type, ML_struct;
Sat, 15 Oct 2005 00:08:15 +0200 wenzelm more;
Sat, 15 Oct 2005 00:08:14 +0200 wenzelm * antiquotations ML_type, ML_struct;
Sat, 15 Oct 2005 00:08:13 +0200 wenzelm added guess;
Sat, 15 Oct 2005 00:08:12 +0200 wenzelm added antiquotations ML_type, ML_struct;
Sat, 15 Oct 2005 00:08:11 +0200 wenzelm use perl for test/stat;
Sat, 15 Oct 2005 00:08:10 +0200 wenzelm export strip_params;
Sat, 15 Oct 2005 00:08:09 +0200 wenzelm note_thmss, read/cert_vars etc.: natural argument order;
Sat, 15 Oct 2005 00:08:08 +0200 wenzelm goal statements: before_qed argument;
Sat, 15 Oct 2005 00:08:07 +0200 wenzelm added 'guess', which derives the obtained context from the course of reasoning;
Sat, 15 Oct 2005 00:08:06 +0200 wenzelm added primitive_text, succeed_text;
Sat, 15 Oct 2005 00:08:05 +0200 wenzelm goal statements: accomodate before_qed argument;
Sat, 15 Oct 2005 00:08:04 +0200 wenzelm goal statements: accomodate before_qed argument;
Sat, 15 Oct 2005 00:08:03 +0200 wenzelm added 'guess';
Sat, 15 Oct 2005 00:08:02 +0200 wenzelm tuned;
Sat, 15 Oct 2005 00:08:01 +0200 wenzelm added no_facts;
Sat, 15 Oct 2005 00:08:00 +0200 wenzelm tuned comments;
Sat, 15 Oct 2005 00:07:59 +0200 wenzelm updated;
Fri, 14 Oct 2005 15:34:56 +0200 paulson signature changes
Fri, 14 Oct 2005 14:36:39 +0200 haftmann added module rat.ML for rational numbers
Fri, 14 Oct 2005 13:04:38 +0200 isatest longer time out for test (kleing)
Fri, 14 Oct 2005 11:36:14 +0200 paulson deletion of Tools/res_types_sorts; removal of absolute numbering of clauses
Fri, 14 Oct 2005 10:19:50 +0200 paulson deletion of Tools/res_types_sorts; removal of absolute numbering of clauses
Thu, 13 Oct 2005 11:58:22 +0200 wenzelm obsolete;
Wed, 12 Oct 2005 18:17:48 +0200 webertj counter added to SAT signature
Wed, 12 Oct 2005 17:06:22 +0200 webertj no proof reconstruction when quick_and_dirty is set
Wed, 12 Oct 2005 10:49:07 +0200 paulson tidying
Wed, 12 Oct 2005 03:02:18 +0200 huffman domain package generates compactness lemmas for new constructors
Wed, 12 Oct 2005 03:01:30 +0200 huffman add ML bindings for compactness lemmas
Wed, 12 Oct 2005 03:01:09 +0200 huffman added compactness theorems
Wed, 12 Oct 2005 01:43:37 +0200 huffman added compactness lemmas; cleaned up
Tue, 11 Oct 2005 23:47:29 +0200 huffman added compactness theorems in locale iso
Tue, 11 Oct 2005 23:27:49 +0200 huffman added several theorems in locale iso
Tue, 11 Oct 2005 23:27:14 +0200 huffman added xsymbols syntax for pairs; cleaned up
Tue, 11 Oct 2005 23:23:39 +0200 huffman added theorem typedef_compact
Tue, 11 Oct 2005 23:22:12 +0200 huffman rearranged subsections; added theorems expand_cfun_eq, expand_cfun_less
Tue, 11 Oct 2005 23:19:50 +0200 huffman cleaned up; renamed less_fun to expand_fun_less
Tue, 11 Oct 2005 17:30:00 +0200 nipkow added hd lemma
Tue, 11 Oct 2005 15:04:11 +0200 paulson simplifying the treatment of clausification
Tue, 11 Oct 2005 15:03:36 +0200 paulson simplifying the treatment of nameless theorems
Tue, 11 Oct 2005 14:02:33 +0200 wenzelm expand: error on undefined/empty env variable;
Tue, 11 Oct 2005 14:02:32 +0200 wenzelm added assert;
Tue, 11 Oct 2005 13:30:17 +0200 wenzelm tuned;
Tue, 11 Oct 2005 13:28:08 +0200 wenzelm added string_of_pid;
Tue, 11 Oct 2005 13:28:07 +0200 wenzelm raw symbols: allow non-ASCII chars (e.g. UTF-8);
Tue, 11 Oct 2005 13:28:06 +0200 wenzelm moved string_of_pid to ML-Systems;
Tue, 11 Oct 2005 13:28:05 +0200 wenzelm ML_SUFFIX in targets (experimental);
Tue, 11 Oct 2005 13:28:04 +0200 wenzelm cleanup backup images;
Mon, 10 Oct 2005 15:35:29 +0200 paulson small tidy-up of utility functions
Mon, 10 Oct 2005 14:43:45 +0200 wenzelm updated print_tac;
Mon, 10 Oct 2005 05:46:17 +0200 huffman add names to infix declarations
Mon, 10 Oct 2005 05:30:02 +0200 huffman new syntax translations for continuous lambda abstraction
Mon, 10 Oct 2005 04:38:26 +0200 huffman removed Istrictify; simplified some proofs
(0) -10000 -3000 -1000 -240 +240 +1000 +3000 +10000 +30000 tip