src/HOL/simpdata.ML
Mon, 12 Sep 2005 18:20:32 +0200 haftmann introduced new-style AList operations
Wed, 31 Aug 2005 15:46:34 +0200 wenzelm simp_implies: proper named infix;
Tue, 02 Aug 2005 19:47:13 +0200 wenzelm added unfold_tac (Simplifier.inherit_bounds);
Tue, 02 Aug 2005 16:50:55 +0200 ballarin Turned simp_implies into binary operator.
Fri, 01 Jul 2005 13:54:12 +0200 berghofe Implemented trick (due to Tobias Nipkow) for fine-tuning simplification
Tue, 28 Jun 2005 15:27:45 +0200 paulson Constant "If" is now local
Thu, 03 Mar 2005 12:43:01 +0100 skalberg Move towards standard functions.
Sun, 13 Feb 2005 17:15:14 +0100 skalberg Deleted Library.option type.
Sat, 18 Dec 2004 17:14:33 +0100 schirmer added simproc for Let
Mon, 06 Sep 2004 17:37:35 +0200 nipkow made mult_mono_thms generic.
Fri, 14 May 2004 16:53:15 +0200 paulson new atomize theorem
Thu, 04 Mar 2004 12:06:07 +0100 paulson new material from Avigad, and simplified treatment of division by 0
Mon, 09 Dec 2002 10:38:56 +0100 ballarin Fixed bug in simpdata.ML that prevented the use of congruence rules from a
Mon, 30 Sep 2002 16:12:16 +0200 berghofe Removed nRS again because extract_rews now takes care of preserving names.
Thu, 19 Sep 2002 16:00:27 +0200 nipkow preserve names of rewrite rules when transforming them
Tue, 06 Aug 2002 11:22:05 +0200 wenzelm sane interface for simprocs;
Thu, 28 Feb 2002 17:46:46 +0100 paulson fixing nat_combine_numerals simprocs (again)
Sat, 12 Jan 2002 16:37:58 +0100 wenzelm renamed forall_elim_vars_safe to gen_all;
Mon, 17 Dec 2001 14:23:10 +0100 nipkow mods due to mor powerful simprocs for 1-point rules (quantifier1).
Wed, 12 Dec 2001 12:40:02 +0100 nipkow Removed pointless backtracking from arith_tac
Sat, 24 Nov 2001 16:54:10 +0100 wenzelm converted simp lemmas;
Fri, 23 Nov 2001 19:20:58 +0100 wenzelm tuned;
Sat, 03 Nov 2001 18:42:38 +0100 wenzelm proper use of bind_thm(s);
Thu, 04 Oct 2001 15:40:31 +0200 wenzelm removed hol_rewrite_cterm (use full_rewrite_cterm from Pure);
Fri, 28 Sep 2001 17:19:46 +0200 berghofe mksimps and mk_eq_True no longer raise THM exception.
Fri, 31 Aug 2001 16:29:18 +0200 berghofe Proof of True_implies_equals is stored with "open" derivation to
Wed, 25 Jul 2001 13:13:01 +0200 paulson partial restructuring to reduce dependence on Axiom of Choice
Fri, 20 Jul 2001 21:58:19 +0200 wenzelm HOL_ss: the_eq_trivial, the_sym_eq_trivial;
Thu, 31 May 2001 16:52:02 +0200 oheimb streamlined addIffs/delIffs, added warnings
Thu, 29 Mar 2001 13:59:54 +0200 nipkow generalization of 1 point rules for ALL
Fri, 23 Mar 2001 10:10:53 +0100 nipkow added one point simprocs for bounded quantifiers
Fri, 09 Mar 2001 19:05:48 +0100 nipkow arith_tac now copes with propositional reasoning as well.
Tue, 20 Feb 2001 18:47:06 +0100 oheimb debugging: replaced gen_all by forall_elim_vars_safe
Fri, 02 Feb 2001 22:19:23 +0100 wenzelm added hol_simplify, hol_rewrite_cterm;
Tue, 30 Jan 2001 18:57:24 +0100 oheimb added if_def2
Tue, 17 Oct 2000 10:21:12 +0200 paulson renaming of contrapos rules
Fri, 15 Sep 2000 12:39:57 +0200 paulson renamed (most of...) the select rules
Thu, 07 Sep 2000 20:51:31 +0200 wenzelm eliminated rulify setup (now in Provers/rulify.ML);
Wed, 06 Sep 2000 16:54:12 +0200 wenzelm tuned;
Wed, 06 Sep 2000 13:32:25 +0200 nipkow imp_cong bound at thm level.
Tue, 05 Sep 2000 18:46:36 +0200 wenzelm iff declarations moved to clasimp.ML;
Mon, 04 Sep 2000 21:19:27 +0200 wenzelm added safe_mk_meta_eq;
Sat, 02 Sep 2000 21:47:50 +0200 wenzelm added 'iff del' att;
Wed, 30 Aug 2000 10:21:19 +0200 nipkow Fixed rulify.
Tue, 29 Aug 2000 00:55:31 +0200 wenzelm cong setup now part of Simplifier;
Thu, 03 Aug 2000 11:51:11 +0200 paulson new theorem neq_commute
Tue, 18 Jul 2000 21:08:40 +0200 wenzelm * HOL: removed obsolete expand_if = split_if; theorems if_splits =
Wed, 28 Jun 2000 10:47:20 +0200 paulson make_elim -> cla_make_elim; tidied
Fri, 02 Jun 2000 17:47:41 +0200 oheimb added eta_contract_eq, also to simpset
Wed, 24 May 2000 18:44:49 +0200 paulson installing the plus_ac0 simprules
Fri, 31 Mar 2000 22:39:06 +0200 wenzelm added cong atts;
Fri, 31 Mar 2000 22:00:36 +0200 wenzelm change_global/local_css move to Provers/clasimp.ML;
Wed, 15 Mar 2000 18:47:28 +0100 wenzelm splitter setup;
Fri, 07 Jan 2000 11:06:03 +0100 paulson tidied parentheses
Tue, 05 Oct 1999 15:24:58 +0200 berghofe Rule not_not is now stored in theory (needed by Inductive).
Wed, 29 Sep 1999 14:38:03 +0200 wenzelm bind_thms;
Tue, 28 Sep 1999 15:12:50 +0200 paulson AC rules for equality
Thu, 23 Sep 1999 13:06:31 +0200 paulson tidied; added lemma restrict_to_left
Tue, 21 Sep 1999 19:11:07 +0200 nipkow Mod because of new solver interface.
Thu, 26 Aug 1999 19:04:19 +0200 wenzelm iff_attrib_setup;
Wed, 25 Aug 1999 20:49:02 +0200 wenzelm proper bootstrap of HOL theory and packages;
Mon, 16 Aug 1999 17:24:28 +0200 oheimb re-added refl in safe_solver
Thu, 29 Jul 1999 12:44:57 +0200 paulson added parentheses to cope with a possible reduction of the precedence of unary
Mon, 19 Jul 1999 15:24:35 +0200 paulson getting rid of qed_goal
Sat, 10 Jul 1999 21:48:27 +0200 wenzelm handle THM/TERM exn;
Thu, 08 Jul 1999 13:38:41 +0200 paulson Now if_weak_cong is a standard congruence rule
Tue, 27 Apr 1999 10:44:17 +0200 wenzelm "iff" attribute;
Wed, 17 Mar 1999 16:53:46 +0100 wenzelm Theory.sign_of;
Wed, 03 Mar 1999 11:15:18 +0100 paulson expandshort
Mon, 01 Mar 1999 18:37:23 +0100 paulson simpler proofs of congruence rules
Thu, 14 Jan 1999 13:18:09 +0100 nipkow More arith refinements.
Thu, 26 Nov 1998 12:18:51 +0100 nipkow Added a general refutation tactic which works by putting things into nnf first.
Thu, 24 Sep 1998 17:16:06 +0200 oheimb simplified CLASIMP_DATA
Wed, 09 Sep 1998 17:34:58 +0200 nipkow Proved and added rewrite rule (@x. x=y) = y to simpset.
Wed, 12 Aug 1998 17:40:18 +0200 oheimb minor adaption for SML/NJ
Wed, 12 Aug 1998 16:21:18 +0200 oheimb the splitter is now defined as a functor
Thu, 06 Aug 1998 15:48:13 +0200 paulson even more tidying of Goal commands
Thu, 30 Jul 1998 19:18:50 +0200 wenzelm made SML/NJ happy;
Thu, 30 Jul 1998 19:02:52 +0200 wenzelm functorized Clasimp module;
Fri, 24 Jul 1998 13:36:49 +0200 berghofe Added functions addIffs and delIffs which operate on clasimpsets.
Thu, 14 May 1998 16:50:09 +0200 oheimb extended addsplits and delsplits to handle also split rules for assumptions
Mon, 27 Apr 1998 16:45:11 +0200 nipkow Added a few lemmas.
Sat, 04 Apr 1998 12:29:07 +0200 wenzelm no open Simplifier;
Thu, 02 Apr 1998 13:48:28 +0200 paulson changed if_bool_eq to if_bool_eq_conj and added if_bool_eq_disj
Fri, 13 Mar 1998 18:15:14 +0100 wenzelm moved addsplits [expand_if] from HOL_basic_ss to HOL_ss;
Thu, 12 Mar 1998 13:17:13 +0100 oheimb renamed not1_or to disj_not1, not2_or to disj_not2
Tue, 10 Mar 1998 18:31:32 +0100 oheimb new rewrite rules not1_or, not2_or, and if_eq_cancel
Fri, 06 Mar 1998 15:19:29 +0100 nipkow expand_if is now by default part of the simpset.
Wed, 04 Mar 1998 13:14:11 +0100 nipkow Reorganized simplifier. May now reorient rules.
Sat, 28 Feb 1998 15:41:17 +0100 nipkow Splitters via named loopers.
Wed, 25 Feb 1998 20:25:27 +0100 oheimb factored out common code of HOL/simpdata.ML and FOL/simpdata.ML concerning
Wed, 25 Feb 1998 15:51:24 +0100 oheimb changed wrapper mechanism of classical reasoner
Fri, 20 Feb 1998 17:56:39 +0100 nipkow Congruence rules use == in premises now.
Wed, 18 Feb 1998 18:42:54 +0100 oheimb corrected problem with auto_tac: now uses a variant of depth_tac that avoids
Thu, 08 Jan 1998 17:42:26 +0100 oheimb replaced fn _ => by K
Wed, 24 Dec 1997 10:02:30 +0100 paulson New Auto_tac (by Oheimb), and new syntax (without parens), and expandshort
Wed, 03 Dec 1997 10:50:02 +0100 paulson Tidying and some comments
Fri, 28 Nov 1997 11:00:42 +0100 paulson Added comments
Fri, 28 Nov 1997 07:41:24 +0100 nipkow Removed dead code.
Fri, 28 Nov 1997 07:37:06 +0100 nipkow Moved the quantifier elimination simp procs into Provers.
Wed, 12 Nov 1997 12:30:15 +0100 oheimb simpdata.ML: renamed split_prem_tac to split_asm_tac, added split_if_asm
Fri, 07 Nov 1997 18:05:25 +0100 oheimb added split_prem_tac
Fri, 07 Nov 1997 18:02:15 +0100 oheimb changed libraray function find to find_index_eq, currying it
Tue, 04 Nov 1997 13:35:13 +0100 wenzelm removed old datatype_info;
Tue, 04 Nov 1997 12:59:01 +0100 nipkow Logic.loops -> Logic.rewrite_rule_ok
Mon, 03 Nov 1997 12:09:37 +0100 wenzelm adapted to new implicit simpset;
Thu, 30 Oct 1997 09:45:03 +0100 nipkow For each datatype `t' there is now a theorem `split_t_case' of the form
Fri, 17 Oct 1997 15:25:12 +0200 nipkow setloop split_tac -> addsplits
Fri, 17 Oct 1997 11:00:50 +0200 paulson New trivial rewrites
Thu, 16 Oct 1997 15:23:53 +0200 paulson New simprules imp_disj1, imp_disj2
Thu, 16 Oct 1997 14:12:15 +0200 nipkow Various new lemmas. Improved conversion of equations to rewrite rules:
Fri, 10 Oct 1997 19:02:28 +0200 wenzelm fixed dots;
Tue, 02 Sep 1997 17:02:02 +0200 nipkow Added True_implies_equals
Wed, 06 Aug 1997 01:13:46 +0200 berghofe Moved some functions which used to be part of thy_data.ML
Fri, 25 Jul 1997 13:18:09 +0200 wenzelm added prems argument to simplification procedures;
Thu, 24 Jul 1997 11:20:12 +0200 nipkow Deleted comment.
Thu, 24 Jul 1997 11:12:18 +0200 nipkow List.ML: added lemmas by Stefan Merz.
Wed, 23 Jul 1997 17:43:42 +0200 nipkow Prod.ML: Added split_paired_EX and lots of comments about failed attempts to
Wed, 23 Jul 1997 11:07:36 +0200 wenzelm tuned congs: standard;
Tue, 22 Jul 1997 11:14:18 +0200 paulson Removal of the tactical STATE
less more (0) -120 tip