1998-04-27 paulson New proof of apply_equality and new thm Pi_image_cons
1998-04-24 oheimb improved split_all_tac significantly
1998-04-24 oheimb improved keyboard modifiers
1998-04-24 oheimb added ASCII translation of subseteq
1998-04-24 paulson tidied; div & mod
1998-04-24 oheimb *** empty log message ***
1998-04-22 wenzelm added no_syn;
1998-04-22 wenzelm added mk_cond_defpair, mk_defpair;
1998-04-22 nipkow Modifications due to improved simplifier.
1998-04-22 nipkow Tried to speed up the rewriter by eta-contracting all patterns beforehand and
1998-04-21 oheimb improved pair_tac to call prune_params_tac afterwards
1998-04-21 oheimb split_all_tac is now added to claset() _before_ other safe tactics
1998-04-21 oheimb made proof of zmult_congruent2 more stable
1998-04-21 oheimb simplification of explicit theory usage and merges
1998-04-21 oheimb removed split_all_tac from claset() globally within IOA
1998-04-21 oheimb made modifications of the simpset() local
1998-04-21 oheimb layout improvement
1998-04-21 paulson expandshort; new gcd_induct with inbuilt case analysis
1998-04-21 paulson Renamed mod_XXX_cancel to mod_XXX_self
1998-04-20 paulson New laws for mod
1998-04-20 paulson proving fib(gcd(m,n)) = gcd(fib m, fib n)
1998-04-19 wenzelm fixed comment;
1998-04-10 paulson Fixed bug in inductive sections to allow disjunctive premises;
1998-04-10 paulson bug fixes
1998-04-10 paulson can prove the empty relation to be WF
1998-04-10 paulson Fixed bug in inductive sections to allow disjunctive premises;
1998-04-09 paulson Clearer description of recdef, including use of {}
1998-04-09 paulson Simplified the syntax description; mentioned FOL vs HOL
1998-04-07 oheimb *** empty log message ***
1998-04-07 oheimb replaced option_map_SomeD by option_map_eq_Some (RS iffD1)
1998-04-07 oheimb made split_all_tac as safe wrapper more defensive:
1998-04-04 wenzelm no open Simplifier;
1998-04-04 wenzelm tuned fail;
1998-04-04 wenzelm type_error;
1998-04-04 wenzelm tuned comments;
1998-04-04 wenzelm no open Simplifier;
1998-04-04 wenzelm replaced thy_data by thy_setup;
1998-04-04 wenzelm type_error;
1998-04-04 wenzelm replaced thy_data by setup;
1998-04-04 wenzelm removed simple;
1998-04-04 wenzelm added triv_goal, rev_triv_goal (for Isar);
1998-04-04 wenzelm added Goal_def;
1998-04-04 wenzelm replaced thy_data by thy_setup;
1998-04-04 wenzelm added local_theory (for Isar);
1998-04-04 wenzelm tuned trace msgs;
1998-04-03 wenzelm tuned names;
1998-04-03 wenzelm added get_tthm(s), store_tthms(s);
1998-04-03 wenzelm tuned comments;
1998-04-03 wenzelm added attribute.ML;
1998-04-03 wenzelm Theorem tags and attributes.
1998-04-03 paulson UNITY
1998-04-03 oheimb repaired incompatibility with new SML version by eta-expansion
1998-04-03 paulson New target HOL-UNITY
1998-04-03 paulson New UNITY theory
1998-04-03 paulson Tidied proofs
1998-04-03 paulson Tidied proofs by getting rid of case_tac
1998-04-03 oheimb improved \tt appearance of many ASCII special symbols like #
1998-04-02 oheimb split_all_tac now fails if there is nothing to split
1998-04-02 paulson new theorems
1998-04-02 paulson changed if_bool_eq to if_bool_eq_conj
1998-04-02 paulson changed if_bool_eq to if_bool_eq_conj and added if_bool_eq_disj
1998-04-02 paulson New theorems card_Diff_le and card_insert_le; tidied
1998-04-02 oheimb introduced functions for updating the wrapper lists
1998-04-02 oheimb *** empty log message ***
1998-03-30 oheimb merge_cs now also merges safe and unsafe wrappers
1998-03-30 oheimb generalized appearance of trancl_into_rtrancl and r_into_trancl
1998-03-30 oheimb adapted proof of finite_converse
1998-03-30 oheimb added wf_converse_trancl, adapted proof of wfrec
1998-03-30 oheimb added caveat
1998-03-30 oheimb added introduction and elimination rules for Univalent
1998-03-30 oheimb added Univalent_rel_pow
1998-03-30 oheimb removed superfluous use_thy
1998-03-30 oheimb removed superfluous translations
1998-03-24 wenzelm added try, single, many;
1998-03-24 oheimb added cproj', and therefore extended prj
1998-03-24 oheimb added cproj', and therefore extended prj
1998-03-24 oheimb improved checks
1998-03-24 oheimb added o2s
1998-03-24 oheimb added finite_acyclic_wf_converse: corrected 8bit chars
1998-03-24 oheimb added acyclicI
1998-03-24 oheimb added finite_acyclic_wf_converse
1998-03-23 paulson more thms
1998-03-16 paulson inverse -> converse
1998-03-16 paulson inverse -> converse
1998-03-16 paulson re-ordered proofs
1998-03-13 wenzelm moved addsplits [expand_if] from HOL_basic_ss to HOL_ss;
1998-03-12 oheimb renamed not1_or to disj_not1, not2_or to disj_not2
1998-03-12 oheimb improved coding of delWrapper and delSWrapper
1998-03-12 oheimb addloop: added warning in case of overwriting a looper
1998-03-12 nipkow Made mutual simplification of prems a special case.
1998-03-12 nipkow Used merge_alists for loopers.
1998-03-12 paulson New, stronger rewrites
1998-03-12 paulson The theorem nat_neqE, and some tidying
1998-03-12 paulson New laws, mostly generalizing old "pred" ones
1998-03-11 paulson spy_analz_tac now handles individual conjuncts properly
1998-03-11 paulson new theorem
1998-03-11 paulson New theorem Image_eq_UN; deleted the silly vimage_inverse_Image
1998-03-11 paulson Arith.thy -> thy; proved a few new theorems
1998-03-11 nipkow New Asm_full_simp_tac shortens proof.
1998-03-11 nipkow Simplifier
1998-03-11 nipkow More Lex.
1998-03-11 nipkow New Asm_full_simp_tac led to a loop.
1998-03-10 nipkow Mod because of new simplifier.
1998-03-10 nipkow Mod because of not1_or.
1998-03-10 nipkow Updated proofs because of new simplifier.
1998-03-10 nipkow Updated proofs because of new simplification tactics.
1998-03-10 nipkow Adapted proofs because of new simplification tactics.
1998-03-10 nipkow The new asm_lr_simp_tac is the old asm_full_simp_tac.
1998-03-10 oheimb renamed is_chain to chain, is_tord to tord, replaced chain_finite by chfin
1998-03-10 oheimb added not1_or and if_eq_cancel to simpset()
1998-03-10 oheimb added not1_or and if_eq_cancel to simpset()
1998-03-10 oheimb new rewrite rules not1_or, not2_or, and if_eq_cancel
1998-03-10 oheimb renamed smart_tac to force_tac, slight improvement of force_tac
1998-03-10 nipkow Asm_full_simp_tac now reorients asm c = t to t = c.
1998-03-10 wenzelm adhoc fix of is_blank;
1998-03-10 nipkow New scanner in abstract form.
1998-03-10 nipkow New simplifier flag for mutual simplification.
1998-03-10 nipkow Removed expand_split from simpset.
1998-03-09 wenzelm removed pred;
1998-03-09 wenzelm eliminated pred function;
1998-03-09 wenzelm Symbol.explode;
1998-03-09 wenzelm replaced $LOGNAME by $USER;
1998-03-09 wenzelm tuned;
1998-03-09 wenzelm Symbol.is_*;
1998-03-09 wenzelm adapted to new scanner, baroque chars;
1998-03-09 wenzelm Symbol.input;
1998-03-09 wenzelm adapted to symbols, scan;
1998-03-09 wenzelm Generic scanners (for potentially infinite input) -- replaces Scanner;
1998-03-09 wenzelm adapted to new scanner and abroque chars;
1998-03-09 wenzelm read_var;
1998-03-09 wenzelm Symbol.output;
1998-03-09 wenzelm tuned syntax error msg;
1998-03-09 wenzelm Symbol.explode;
1998-03-09 wenzelm scan.ML, symbol.ML;
1998-03-09 wenzelm adapted to new scanners and baroque chars;
1998-03-09 wenzelm tuned some names;
1998-03-09 wenzelm adapted to baroque chars;
1998-03-09 wenzelm added merge_alists;
1998-03-09 wenzelm Syntax.indexname;
1998-03-09 wenzelm tuned comment;
1998-03-09 wenzelm tuned;
1998-03-09 wenzelm replaced Pure/Syntax/symbol_font.ML by Pure/Syntax/symbol.ML;
1998-03-09 wenzelm replaced Pure/Syntax/symbol_font.ML by Pure/Syntax/symbol.ML;
1998-03-07 nipkow Removed `addsplits [expand_if]'
1998-03-06 wenzelm added clasimp.ML;
1998-03-06 nipkow Removed superfluous `op'
1998-03-06 nipkow *** empty log message ***
1998-03-06 nipkow Added delspilts, Addsplits, Delsplits.
1998-03-06 nipkow expand_if is now by default part of the simpset.
1998-03-05 paulson New theorem and simprules
1998-03-04 nipkow Reorganized simplifier. May now reorient rules.
1998-03-04 nipkow Reorganized simplifier. May now reorient rules.
1998-03-04 nipkow Reorganized simplifier. May now reorient rules.
1998-03-03 paulson Better simplification allows deletion of parts of proofs
1998-03-03 paulson New theorem
1998-03-03 paulson New theorems
1998-03-03 paulson New theorems; tidied
1998-03-03 paulson New theorem diff_Suc_le_Suc_diff; tidied another proof
1998-03-03 paulson auto generated
1998-02-28 nipkow Modified def.
1998-02-28 nipkow Splitters via named loopers.
1998-02-28 nipkow Little reorganization. Loop tactics have names now.
1998-02-28 nipkow Tried to reorganize rewriter a little. More to be done.
1998-02-27 oheimb added minimal description of rep_cs: corrections
1998-02-27 oheimb added minimal description of rep_cs
1998-02-27 oheimb added minimal description of rep_ss
1998-02-27 paulson "choice" moved to Set.ML
1998-02-27 paulson New absorbsion laws, etc
1998-02-27 paulson Vimage
1998-02-27 paulson New vimage laws
1998-02-26 oheimb added smart_tac
1998-02-26 oheimb removed superfluous addss
1998-02-26 paulson New theory, Vimage
1998-02-26 paulson Proved choice and bchoice; changed Fun.thy -> thy
1998-02-26 wenzelm *** empty log message ***
1998-02-26 wenzelm added clasimp.ML;
1998-02-25 oheimb renamed rep_claset to rep_cs
1998-02-25 oheimb factored out common code of HOL/simpdata.ML and FOL/simpdata.ML concerning
1998-02-25 oheimb changed wrapper mechanism of classical reasoner
1998-02-25 oheimb added split_all_tac to claset()
1998-02-25 oheimb changed wrapper mechanism of classical reasoner
1998-02-24 paulson New theory of the inverse image of a function
1998-02-24 nipkow Added some lemmas.
1998-02-23 paulson Catches bad elim rules, handling exception OPTION
1998-02-23 paulson New laws for union
1998-02-23 paulson New laws for id
1998-02-22 nipkow New induction schemas for lists (length and snoc).
1998-02-20 nipkow *** empty log message ***
1998-02-20 nipkow Congruence rules use == in premises now.
1998-02-20 nipkow Congruence rules use == in premises now.
1998-02-20 oheimb minor improvements
1998-02-20 oheimb re-arranged bindings for many function keys
1998-02-20 oheimb extended input syntax to handle names of special keys
1998-02-20 oheimb moved Ctrl entry before Alt entry
1998-02-20 paulson New theorem eq_imp_le
1998-02-19 paulson Four new Union/Intersection laws
1998-02-18 oheimb corrected problem with auto_tac: now uses a variant of depth_tac that avoids
1998-02-18 wenzelm added New Jersey mirror;
1998-02-18 nipkow Improved loop-test for rewrite rules a little.
1998-02-18 wenzelm tuned comment;
1998-02-13 wenzelm added append (curried);
1998-02-12 wenzelm *** empty log message ***
1998-02-12 wenzelm Sign.merge vs. Sign.nontriv_merge;
1998-02-12 wenzelm tuned comments;
1998-02-12 wenzelm oops;
1998-02-12 wenzelm tuned print_cs;
1998-02-12 wenzelm updated;
1998-02-12 wenzelm tuned;
1998-02-12 wenzelm added explicit signature;
1998-02-12 wenzelm improved comments;
1998-02-12 wenzelm fixed add_trrules: intern root;
1998-02-12 wenzelm export map_trrule;
1998-02-12 wenzelm tuned add_trrules;
1998-02-12 wenzelm improved is_letter etc.;
1998-02-10 paulson New Addsimps for Compl rules
1998-02-10 paulson New AddIffs le_0_eq and neq0_conv
1998-02-09 nipkow Replaced ALLNEWSUBGOALS by THEN_ALL_NEW
1998-02-09 nipkow Used THEN_ALL_NEW.
1998-02-07 paulson moved freeze_thaw to drule.ML
1998-02-07 paulson Tidying; rotate_prems; moved freeze_thaw from tactic.ML
1998-02-07 paulson AC and other rewrite rules for Un and Int
1998-02-07 paulson auto update
1998-02-07 paulson Added reference to rotate_prems
1998-02-06 nipkow filter_size -> length_filter
1998-02-06 nipkow Added `remdups'
1998-02-06 wenzelm added Vartab: TABLE;
1998-02-05 wenzelm added param;
1998-02-05 wenzelm added THEN_ALL_NEW;
1998-02-05 paulson New theorem Image_id
1998-02-05 paulson New theorem order_eq_refl
1998-02-05 paulson New max, min theorems
1998-02-05 paulson Added some more explicit guarantees of key secrecy for agents
1998-02-05 paulson Fixed a lot of overfull and underfull lines (hboxes)
1998-02-05 paulson Updated the description of how to set up hyp_subst_tac
1998-02-02 paulson New example, Pow_Sigma_bij
1998-02-02 paulson fixed WWW links
1998-02-02 paulson Three new facts about Image
1998-02-02 paulson Replaced \\1 by $1 as Perl itself asked me to...
1998-01-30 paulson Fixed the description of recdef
1998-01-30 wenzelm tuned msgs;
(0) -3000 -1000 -240 +240 +1000 +3000 +10000 +30000 tip