src/HOL/HOL.thy
Fri, 26 Sep 2003 10:34:57 +0200 paulson misc tidying
Tue, 23 Sep 2003 15:42:01 +0200 paulson some basic new lemmas
Sun, 22 Dec 2002 15:02:40 +0100 nipkow removed some problems with print translations
Sun, 22 Dec 2002 10:43:43 +0100 nipkow added print translations tha avoid eta contraction for important binders.
Thu, 21 Nov 2002 17:40:11 +0100 nipkow *** empty log message ***
Thu, 10 Oct 2002 14:21:49 +0200 berghofe Added choice_eq.
Mon, 30 Sep 2002 16:09:05 +0200 berghofe Fixed problem with induct_conj_curry: variable C should have type prop.
Mon, 30 Sep 2002 15:44:21 +0200 nipkow modified induct method
Mon, 02 Sep 2002 11:07:26 +0200 nipkow order_less_irrefl: [simp] -> [iff]
Fri, 30 Aug 2002 16:42:45 +0200 paulson removal of blast.overloaded
Mon, 05 Aug 2002 21:16:36 +0200 wenzelm special syntax for index "1" (plain numeral hidden by "1" symbol in HOL);
Wed, 31 Jul 2002 16:10:24 +0200 nipkow added mk_left_commute to HOL.thy and used it "everywhere"
Wed, 24 Jul 2002 22:15:55 +0200 wenzelm simplified locale predicates;
Wed, 24 Jul 2002 00:10:52 +0200 wenzelm predicate defs via locales;
Mon, 25 Feb 2002 20:48:14 +0100 wenzelm clarified syntax of ``long'' statements: fixes/assumes/shows;
Fri, 15 Feb 2002 20:41:19 +0100 wenzelm tuned;
Sun, 06 Jan 2002 16:51:04 +0100 wenzelm "_not_equal" dummy constant;
Fri, 04 Jan 2002 19:29:30 +0100 wenzelm tuned ``syntax (output)'';
Mon, 10 Dec 2001 15:16:49 +0100 berghofe Replaced several occurrences of "blast" by "rules".
Wed, 05 Dec 2001 03:19:14 +0100 wenzelm tuned declarations (rules, sym, etc.);
Tue, 04 Dec 2001 02:01:13 +0100 wenzelm setup "rules" method;
Sat, 01 Dec 2001 18:52:32 +0100 wenzelm renamed class "term" to "type" (actually "HOL.type");
Sat, 24 Nov 2001 16:54:10 +0100 wenzelm converted simp lemmas;
Wed, 21 Nov 2001 00:32:10 +0100 wenzelm tuned;
Mon, 19 Nov 2001 20:46:05 +0100 wenzelm induct method: localize rews for rule;
Mon, 12 Nov 2001 20:22:51 +0100 wenzelm lemmas induct_atomize = atomize_conj ...;
Fri, 09 Nov 2001 00:09:47 +0100 wenzelm eliminated old "symbols" syntax, use "xsymbols" instead;
Sat, 03 Nov 2001 01:33:54 +0100 wenzelm tuned;
Wed, 31 Oct 2001 21:58:04 +0100 wenzelm removed obsolete (rule equal_intr_rule);
Wed, 31 Oct 2001 01:20:42 +0100 wenzelm renamed inductive_XXX to induct_XXX;
Sun, 28 Oct 2001 21:14:56 +0100 wenzelm tuned declaration of rules;
Fri, 26 Oct 2001 23:59:13 +0200 wenzelm atomize_conj;
Thu, 18 Oct 2001 20:59:33 +0200 wenzelm setup generic cases and induction (from Inductive.thy);
Sun, 14 Oct 2001 22:08:29 +0200 wenzelm moved rulify to ObjectLogic;
Sun, 14 Oct 2001 20:01:42 +0200 wenzelm judgment Trueprop;
Fri, 12 Oct 2001 12:05:46 +0200 wenzelm declare impE iffD1 iffD2 as elim of Pure;
Fri, 05 Oct 2001 21:49:15 +0200 wenzelm added axclass "one" and polymorphic const "1";
Thu, 04 Oct 2001 15:42:48 +0200 wenzelm non-oriented infix = and ~= (output only);
Wed, 25 Jul 2001 13:13:01 +0200 paulson partial restructuring to reduce dependence on Axiom of Choice
Sun, 22 Jul 2001 21:30:05 +0200 wenzelm declare trans [trans] (*overridden in theory Calculation*);
Fri, 20 Jul 2001 21:52:54 +0200 wenzelm added "The" (definite description operator) (by Larry);
Sat, 18 Nov 2000 19:45:05 +0100 wenzelm symbol syntax for "abs";
Fri, 10 Nov 2000 19:02:37 +0100 wenzelm added axclass inverse and consts inverse, divide (infix "/");
Fri, 03 Nov 2000 21:31:11 +0100 wenzelm "atomize" for classical tactics;
Fri, 15 Sep 2000 15:30:50 +0200 paulson the final renaming: selectI -> someI
Wed, 13 Sep 2000 22:29:17 +0200 wenzelm \<epsilon>: syntax (input);
Thu, 07 Sep 2000 20:49:39 +0200 wenzelm removed rulify_attrib_setup;
Tue, 05 Sep 2000 21:06:01 +0200 wenzelm improved meson setup;
Tue, 05 Sep 2000 18:47:03 +0200 wenzelm tuned setup;
Tue, 05 Sep 2000 10:14:36 +0200 paulson loads Tools/meson.ML: meson_tac installed by default
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;
Fri, 04 Aug 2000 22:56:52 +0200 wenzelm lemmas atomize = all_eq imp_eq;
Tue, 01 Aug 2000 11:58:27 +0200 wenzelm added all_eq, imp_eq (for blast);
Sun, 16 Jul 2000 20:48:35 +0200 wenzelm syntax (symbols) "op o" moved from HOL to Fun;
Tue, 13 Jun 2000 18:34:59 +0200 wenzelm rename @case to _case_syntax (improves on low-level errors);
Wed, 24 May 2000 18:47:43 +0200 paulson installing the plus_ac0 axclass
Tue, 23 May 2000 18:22:19 +0200 paulson new type class "zero" so that 0 can be overloaded
Fri, 05 May 2000 18:24:06 +0200 nipkow Added constant abs.
Fri, 31 Mar 2000 21:59:37 +0200 wenzelm setup cong_attrib_setup;
less more (0) -100 -60 tip