2002-02-21 wenzelm updated title;
2002-02-21 kleing new MicroJava document
2002-02-21 kleing fix toc
2002-02-21 wenzelm fixed document;
2002-02-21 wenzelm tr: quote argument;
2002-02-21 kleing new document
2002-02-20 berghofe Removed superfluous lookup of theorems in Relation.thy
2002-02-20 berghofe Moved change_type to proofterm.ML
2002-02-20 berghofe New function strip_comb (cterm version of Term.strip_comb).
2002-02-20 berghofe New function change_type for changing type assignments of theorems,
2002-02-20 berghofe New function for eliminating definitions in proof term.
2002-02-20 berghofe Converted to new theory format.
2002-02-19 wenzelm added is_quasi;
2002-02-19 wenzelm removed obscure functions bump_int_list, bump_list, bump_string;
2002-02-19 wenzelm Symbol.bump_string;
2002-02-19 wenzelm tuned;
2002-02-19 wenzelm Paulson:1989;
2002-02-19 wenzelm "isatool usedir -D output HOL Test && isatool document Test/output";
2002-02-16 kleing fixed copy_all
2002-02-16 wenzelm converted/deleted equalities.ML, mono.ML, subset.ML (see Set.thy);
2002-02-15 wenzelm removed unused unmask_interrupt;
2002-02-15 wenzelm clarified copy_all;
2002-02-15 wenzelm moved copy_all to Thy/present.ML;
2002-02-15 wenzelm replaced nodups by distinct;
2002-02-15 wenzelm tuned;
2002-02-15 paulson a new definition of "restrict"
2002-02-14 wenzelm made MLWorks happy;
2002-02-14 nipkow *** empty log message ***
2002-02-14 nipkow nodups -> distinct
2002-02-14 nipkow nodups -> distinct
2002-02-13 paulson deleted some redundant 'addS*Es [equalityC*E]'s
2002-02-13 paulson new function lemmas
2002-02-13 paulson tidied. no more special simpset (super_ss)
2002-02-13 paulson new lemmas for closure under Union
2002-02-12 wenzelm eliminated Pure/Isar/comment.ML;
2002-02-12 wenzelm ANTIQUOTE_FAIL;
2002-02-12 wenzelm eliminated Isar/comment.ML;
2002-02-12 wenzelm tuned;
2002-02-12 wenzelm added isabelle-hol-book;
2002-02-12 wenzelm * Isar/Pure: marginal comments ``--'' may now occur just anywhere in the text;
2002-02-12 wenzelm got rid of explicit marginal comments (now stripped earlier from input);
2002-02-12 wenzelm tuned;
2002-02-11 wenzelm ML-Systems/smlnj-compiler.ML compatibility tweak;
2002-02-11 wenzelm include SVC_Test;
2002-02-07 berghofe Theorems are only "pre-named" if the do not already have names.
2002-02-06 berghofe Added function could_unify to speed up rewriting of proof terms.
2002-02-06 berghofe Indexes of variables in expanded proofs are now incremented to avoid clashes.
2002-02-05 wenzelm moved SVC stuff to ex;
2002-02-05 berghofe New function maxidx_of_proof.
2002-02-04 paulson New-style versions of these old examples
2002-02-02 berghofe Rewrite procedure now works for both compact and full proof objects.
2002-01-30 wenzelm escape_mfix;
2002-01-30 wenzelm added literal;
2002-01-30 wenzelm prep_mixfix': proper use of Syntax.literal;
2002-01-30 wenzelm tuned;
2002-01-30 paulson mu-syntax for the LEAST operator
2002-01-30 paulson Multiset: added the translation Mult(A) => A-||>nat-{0}
2002-01-28 wenzelm tuned;
2002-01-28 wenzelm GPLed;
2002-01-28 wenzelm tuned header;
2002-01-28 wenzelm tuned;
2002-01-28 schirmer Bali added
2002-01-28 schirmer Isabelle/Bali sources;
2002-01-26 wenzelm Isar cases/induct: no backtracking;
2002-01-26 wenzelm cases: really append cases_default;
2002-01-26 wenzelm generic DETERM;
2002-01-25 paulson ZF
2002-01-24 wenzelm copy_files *.sty;
2002-01-24 wenzelm cond_print_result_rule: priority (again) instead of slightly
2002-01-24 wenzelm fixed subgoal_tac; fails on non-existent subgoal;
2002-01-24 wenzelm copy_styles replaces overly conservative update_styles;
2002-01-24 wenzelm Springer LNCS 2283;
2002-01-24 wenzelm updated;
2002-01-24 wenzelm iff del: less_Suc0 -- luckily this does NOT affect the printed text;
2002-01-23 wenzelm delsimps [less_Suc0];
2002-01-23 wenzelm less_Suc0;
2002-01-23 wenzelm error "Unexpected end of input";
2002-01-23 wenzelm reorganized code for predicate text;
2002-01-23 wenzelm tuned;
2002-01-23 wenzelm * HOL: nat_number_of;
2002-01-23 paulson A few more standard simprules, TCs, etc.
2002-01-22 wenzelm qualified_result replaces qualified;
2002-01-22 wenzelm added locale_facts(_i) interface (useful for simple ML proof tools);
2002-01-21 wenzelm full_proofs;
2002-01-21 wenzelm * Pure/show_hyps reset by default (in accordance to existing Isar practice);
2002-01-21 wenzelm reset show_hyps by default (in accordance to existing Isar practice);
2002-01-21 wenzelm save library;
2002-01-21 wenzelm full_atomize;
2002-01-21 wenzelm wild guess at polyml-4.1.2;
2002-01-21 wenzelm options -l and -t;
2002-01-21 berghofe Removed timing function.
2002-01-21 paulson new simprules and classical rules
2002-01-21 berghofe Tuned name mangling function.
2002-01-21 berghofe Made some proofs constructive.
2002-01-21 berghofe datatype_codegen now checks type of constructor.
2002-01-21 nipkow *** empty log message ***
2002-01-21 paulson lexical tidying
2002-01-21 paulson slight re-use of code
2002-01-19 kleing fixed typos
2002-01-18 wenzelm rewrite_term: removed rew0, so no on-the-fly eta-contraction;
2002-01-18 wenzelm fixed document setup of HOL-Library;
2002-01-18 wenzelm tuned;
2002-01-18 paulson tidied
2002-01-18 paulson OOPS
2002-01-18 paulson tweaks
2002-01-18 wenzelm moved document sources to proper place, *within* Library/Library (!);
2002-01-17 wenzelm cover polyml-4.1.2;
2002-01-17 wenzelm RuleCases.make interface based on term instead of thm;
2002-01-17 wenzelm RuleCases.make interface based on term instead of thm;
2002-01-17 wenzelm atomize_term replaces atomize_cterm;
2002-01-17 wenzelm ObjectLogic.atomize_term replaces ObjectLogic.atomize_cterm;
2002-01-17 wenzelm Thm.prop_of;
2002-01-17 wenzelm Tactic.norm_hhf renamed to Tactic.norm_hhf_rule;
2002-01-17 wenzelm added prop_of: thm -> term (at last!);
2002-01-17 wenzelm added add_term_free_names (more precise/efficient than add_term_names);
2002-01-17 wenzelm renamed norm_hhf to norm_hhf_rule;
2002-01-17 wenzelm added is_norm_hhf (from logic.ML);
2002-01-17 wenzelm MetaSimplifier.rewrite_term replaces slow Tactic.rewrite_cterm;
2002-01-17 wenzelm MetaSimplifier.rewrite_term replaces slow Tactic.rewrite_cterm;
2002-01-17 wenzelm eta_contract with sharing (by berghofe);
(0) -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip