Tue, 13 Aug 2002 21:54:23 +0200 nipkow *** empty log message ***
Tue, 13 Aug 2002 17:42:34 +0200 paulson In ZF/Constructible, moved many results from Satisfies_absolute, etc., to
Tue, 13 Aug 2002 12:16:14 +0200 wenzelm more robust printing of numerals;
Tue, 13 Aug 2002 11:03:11 +0200 paulson new file Constructible/Satisfies_absolute.thy
Mon, 12 Aug 2002 18:01:44 +0200 paulson Lots of new results concerning recursive datatypes, towards absoluteness of
Mon, 12 Aug 2002 17:59:57 +0200 nipkow *** empty log message ***
Mon, 12 Aug 2002 17:48:19 +0200 nipkow *** empty log message ***
Mon, 12 Aug 2002 17:48:15 +0200 nipkow Added Mi and Max on sets, hid Min and Pls on numerals.
Fri, 09 Aug 2002 11:22:18 +0200 nipkow *** empty log message ***
Thu, 08 Aug 2002 23:53:22 +0200 wenzelm transform_error: pass through Interrupt;
Thu, 08 Aug 2002 23:52:55 +0200 wenzelm tuned;
Thu, 08 Aug 2002 23:51:24 +0200 wenzelm exception SIMPROC_FAIL: solid error reporting of simprocs;
Thu, 08 Aug 2002 23:50:23 +0200 wenzelm tuned prove_conv (error reporting done within meta_simplifier.ML);
Thu, 08 Aug 2002 23:49:44 +0200 wenzelm adhoc_freeze_vars;
Thu, 08 Aug 2002 23:48:31 +0200 wenzelm proper instantiation of mk_left_commute;
Thu, 08 Aug 2002 23:47:41 +0200 wenzelm converted;
Thu, 08 Aug 2002 23:46:51 +0200 wenzelm tuned deps;
Thu, 08 Aug 2002 23:46:09 +0200 wenzelm use Tactic.prove instead of prove_goalw_cterm in internal proofs!
Thu, 08 Aug 2002 23:42:49 +0200 wenzelm Tactic.prove, Tactic.prove_standard;
Thu, 08 Aug 2002 23:42:10 +0200 wenzelm * Pure: improved error reporting of simprocs;
Wed, 07 Aug 2002 20:11:07 +0200 wenzelm tuned;
Wed, 07 Aug 2002 20:05:43 +0200 wenzelm mk_left_commute: proper instantiation avoids expensive unification;
Wed, 07 Aug 2002 20:03:38 +0200 wenzelm tuned;
Wed, 07 Aug 2002 20:03:17 +0200 wenzelm Simplifier.simproc(_i);
Wed, 07 Aug 2002 18:32:50 +0200 nipkow Added time example at the end.
Wed, 07 Aug 2002 17:36:05 +0200 wenzelm section on "Rule declarations and methods";
Wed, 07 Aug 2002 16:50:08 +0200 berghofe Removed (now unneeded) declaration of realizer for induction on datatype b.
Wed, 07 Aug 2002 16:49:25 +0200 berghofe Removed (now unneeded) declarations of realizers for induction on lists and letters.
Wed, 07 Aug 2002 16:48:20 +0200 berghofe Added file Tools/datatype_realizer.ML
Wed, 07 Aug 2002 16:47:36 +0200 berghofe Removed (now unneeded) declaration of realizers for induction on natural numbers.
Wed, 07 Aug 2002 16:46:15 +0200 berghofe Module for defining realizers for induction and case analysis theorems
Wed, 07 Aug 2002 16:44:47 +0200 berghofe Added calls to add_dt_realizers.
Wed, 07 Aug 2002 16:43:41 +0200 berghofe Exported function make_tnames.
Wed, 07 Aug 2002 05:54:44 +0200 nipkow Fixed two bugs
Tue, 06 Aug 2002 11:24:27 +0200 wenzelm * Provers: Simplifier.simproc(_i) now provide sane interface for
Tue, 06 Aug 2002 11:22:05 +0200 wenzelm sane interface for simprocs;
Tue, 06 Aug 2002 11:20:47 +0200 wenzelm fixed intern_skolem: disallow internal names (why didn't anybody notice?!?);
Tue, 06 Aug 2002 11:19:52 +0200 wenzelm predefined locales "var" and "struct" (useful for sharing parameters);
Tue, 06 Aug 2002 11:19:00 +0200 wenzelm * Pure: predefined locales "var" and "struct" are useful for sharing
Mon, 05 Aug 2002 21:17:45 +0200 wenzelm protect simplifier operation against spurious exceptions from simprocs;
Mon, 05 Aug 2002 21:17:04 +0200 wenzelm tuned;
Mon, 05 Aug 2002 21:16:36 +0200 wenzelm special syntax for index "1" (plain numeral hidden by "1" symbol in HOL);
Mon, 05 Aug 2002 14:35:33 +0200 berghofe Removed theory NatDef.
Mon, 05 Aug 2002 14:32:56 +0200 berghofe Replaced nat_ind_tac by induct_tac.
Mon, 05 Aug 2002 14:30:06 +0200 berghofe Removed proof of Suc_le_D (already proved in Nat.thy).
Mon, 05 Aug 2002 14:29:20 +0200 berghofe Removed reference to theory NatDef.
Mon, 05 Aug 2002 14:28:31 +0200 berghofe Removed reference to simpset of NatDef.thy
Mon, 05 Aug 2002 14:27:55 +0200 berghofe Legacy ML bindings.
Mon, 05 Aug 2002 14:27:42 +0200 berghofe - Converted to new theory format
Mon, 05 Aug 2002 14:26:54 +0200 berghofe Moved NatDef stuff to theory Nat.
Mon, 05 Aug 2002 12:00:51 +0200 wenzelm updated;
Fri, 02 Aug 2002 21:40:47 +0200 wenzelm added Isabelle LNCSes;
Fri, 02 Aug 2002 21:40:28 +0200 wenzelm fixed long statement: P.opt_thm_name;
Fri, 02 Aug 2002 17:52:51 +0200 wenzelm fixed railroads;
Fri, 02 Aug 2002 11:49:55 +0200 wenzelm typedef: "open" option;
Fri, 02 Aug 2002 11:12:34 +0200 wenzelm declare projected "axioms" as "elim?";
Thu, 01 Aug 2002 18:22:46 +0200 paulson better satisfies rules for is_recfun
Wed, 31 Jul 2002 18:30:25 +0200 paulson some progress towards "satisfies"
Wed, 31 Jul 2002 17:42:38 +0200 nipkow *** empty log message ***
Wed, 31 Jul 2002 16:10:24 +0200 nipkow added mk_left_commute to HOL.thy and used it "everywhere"
Wed, 31 Jul 2002 14:40:40 +0200 paulson separate "axioms" proofs: more flexible for locale reasoning
Wed, 31 Jul 2002 14:39:47 +0200 paulson tweaks involving Separation
Wed, 31 Jul 2002 14:34:08 +0200 paulson new theorem eq_commute
Tue, 30 Jul 2002 11:39:57 +0200 paulson better sats rules for higher-order operators
Tue, 30 Jul 2002 11:38:33 +0200 paulson removal of twos_compl.ML, which is not really needed
Tue, 30 Jul 2002 10:29:34 +0200 isatest - changed date format for proper lexicographical ordering
Tue, 30 Jul 2002 10:28:38 +0200 isatest changed date format for proper lexicographical ordering
Mon, 29 Jul 2002 21:39:22 +0200 wenzelm tuned messages;
Mon, 29 Jul 2002 18:07:53 +0200 wenzelm tuned;
Mon, 29 Jul 2002 00:57:16 +0200 wenzelm eliminate open locales and special ML code;
Sun, 28 Jul 2002 21:09:37 +0200 wenzelm tuned document;
Sat, 27 Jul 2002 21:55:14 +0200 wenzelm make SML/NJ happy;
Fri, 26 Jul 2002 21:09:39 +0200 wenzelm support for split assumptions in cases (hyps vs. prems);
Fri, 26 Jul 2002 21:07:57 +0200 wenzelm tuned;
Thu, 25 Jul 2002 18:29:04 +0200 paulson More lemmas, working towards relativization of "satisfies"
Thu, 25 Jul 2002 10:56:35 +0200 paulson Added the assumption nth_replacement to locale M_datatypes.
Wed, 24 Jul 2002 22:15:55 +0200 wenzelm simplified locale predicates;
Wed, 24 Jul 2002 22:14:42 +0200 wenzelm removed unused locale_facts(_i);
Wed, 24 Jul 2002 22:13:02 +0200 wenzelm tuned;
Wed, 24 Jul 2002 17:59:12 +0200 paulson tweaks, aiming towards relativization of "satisfies"
Wed, 24 Jul 2002 16:16:44 +0200 berghofe Tuned type constraint of function merge_rules to make smlnj happy.
Wed, 24 Jul 2002 00:13:41 +0200 wenzelm AC18: meta-level predicate via locale;
Wed, 24 Jul 2002 00:12:50 +0200 wenzelm tuned view;
Wed, 24 Jul 2002 00:11:56 +0200 wenzelm removed attribute "norm_hhf";
Wed, 24 Jul 2002 00:11:24 +0200 wenzelm adapted fact names;
Wed, 24 Jul 2002 00:10:52 +0200 wenzelm predicate defs via locales;
Wed, 24 Jul 2002 00:09:44 +0200 wenzelm locales: predicate defs;
Wed, 24 Jul 2002 00:08:52 +0200 wenzelm * Pure: locale specifications now produce predicate definitions;
Tue, 23 Jul 2002 15:07:12 +0200 paulson Relativization and Separation for the function "nth"
Mon, 22 Jul 2002 13:55:44 +0200 berghofe Added "nocite" to avoid BibTeX error when proofs are switched off.
Sun, 21 Jul 2002 15:52:39 +0200 berghofe Added program extraction keywords.
Sun, 21 Jul 2002 15:45:41 +0200 berghofe Document for program extraction in HOL.
Sun, 21 Jul 2002 15:44:42 +0200 berghofe Examples for program extraction in HOL.
Sun, 21 Jul 2002 15:43:14 +0200 berghofe Rules for rewriting HOL proofs.
Sun, 21 Jul 2002 15:42:30 +0200 berghofe Added theory for setting up program extraction.
Sun, 21 Jul 2002 15:37:04 +0200 berghofe Added program extraction module.
Fri, 19 Jul 2002 18:44:37 +0200 wenzelm *** empty log message ***
Fri, 19 Jul 2002 18:44:36 +0200 wenzelm accomodate cumulative locale predicates;
Fri, 19 Jul 2002 18:44:07 +0200 wenzelm support locale ``views'' (for cumulative predicates);
Fri, 19 Jul 2002 18:06:31 +0200 paulson Towards relativization and absoluteness of formula_rec
Fri, 19 Jul 2002 13:29:22 +0200 paulson Absoluteness of the function "nth"
Fri, 19 Jul 2002 13:28:19 +0200 paulson A couple of new theorems for Constructible
Thu, 18 Jul 2002 15:21:42 +0200 paulson absoluteness for "formula" and "eclose"
Thu, 18 Jul 2002 12:10:24 +0200 wenzelm define cumulative predicate view;
Thu, 18 Jul 2002 12:09:44 +0200 wenzelm adapted add_locale;
Thu, 18 Jul 2002 12:09:28 +0200 wenzelm adapted locale syntax;
Thu, 18 Jul 2002 12:09:08 +0200 wenzelm fixed inform_file_retracted: remove_thy;
Thu, 18 Jul 2002 12:08:45 +0200 wenzelm ACe_axioms;
Thu, 18 Jul 2002 12:05:51 +0200 wenzelm added satisfy_hyps;
Thu, 18 Jul 2002 12:05:29 +0200 wenzelm quantify LC (conflict with const name of HOL);
Thu, 18 Jul 2002 10:37:55 +0200 paulson new theorems to support Constructible proofs
Wed, 17 Jul 2002 16:41:32 +0200 paulson Formulas (and lists) in M (and L!)
Wed, 17 Jul 2002 15:48:54 +0200 paulson Expressing Lset and L without using length and arity; simplifies Separation
Tue, 16 Jul 2002 20:25:21 +0200 schirmer Added conditional and (&&) and or (||).
Tue, 16 Jul 2002 18:52:26 +0200 wenzelm adapted locales;
Tue, 16 Jul 2002 18:46:59 +0200 wenzelm adapted locales;
Tue, 16 Jul 2002 18:46:13 +0200 wenzelm tuned;
Tue, 16 Jul 2002 18:46:04 +0200 wenzelm adapted locales;
Tue, 16 Jul 2002 18:43:05 +0200 wenzelm rearranged to work without proof contexts;
Tue, 16 Jul 2002 18:42:07 +0200 wenzelm export_standard supercedes export_single;
Tue, 16 Jul 2002 18:41:50 +0200 wenzelm export map_context;
Tue, 16 Jul 2002 18:41:18 +0200 wenzelm assert_propT;
Tue, 16 Jul 2002 18:41:00 +0200 wenzelm proper predicate definitions of locale body;
Tue, 16 Jul 2002 18:40:11 +0200 wenzelm add_locale: adapted args;
Tue, 16 Jul 2002 18:39:55 +0200 wenzelm locale: optional predicate name, or "open";
Tue, 16 Jul 2002 18:39:27 +0200 wenzelm module now right after ProofContext (for locales);
Tue, 16 Jul 2002 18:38:36 +0200 wenzelm avoid "_st" versions of proof data;
Tue, 16 Jul 2002 18:38:11 +0200 wenzelm context rules;
(0) -10000 -3000 -1000 -128 +128 +1000 +3000 +10000 +30000 tip