src/Pure/Isar/locale.ML
Mon, 09 Oct 2006 02:20:04 +0200 wenzelm removed obsolete note_thmss(_i);
Sat, 07 Oct 2006 01:30:58 +0200 wenzelm tuned;
Thu, 21 Sep 2006 19:04:20 +0200 wenzelm member (op =);
Fri, 15 Sep 2006 22:56:13 +0200 wenzelm renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
Wed, 09 Aug 2006 00:12:38 +0200 wenzelm global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
Thu, 03 Aug 2006 14:53:57 +0200 ballarin Updated comments.
Wed, 02 Aug 2006 22:27:01 +0200 wenzelm removed obsolete Drule.frees/vars_of etc.;
Thu, 27 Jul 2006 23:28:28 +0200 wenzelm renamed ProofContext.fix_frees to Variable.fix_frees;
Thu, 27 Jul 2006 13:43:01 +0200 wenzelm moved basic assumption operations from structure ProofContext to Assumption;
Tue, 25 Jul 2006 21:18:02 +0200 wenzelm renamed add_term_varnames to Term.add_varnames (cf. Term.add_vars etc.);
Wed, 19 Jul 2006 19:24:02 +0200 ballarin Strict dfs traversal of imported and registered identifiers.
Tue, 11 Jul 2006 12:24:23 +0200 wenzelm Name.internal;
Tue, 11 Jul 2006 11:19:28 +0200 ballarin Witness theorems of interpretations now transfered to current theory.
Sat, 08 Jul 2006 12:54:47 +0200 wenzelm Element.prove_witness: context;
Fri, 07 Jul 2006 09:39:25 +0200 ballarin Fixed erroneous check-in.
Fri, 07 Jul 2006 09:28:39 +0200 ballarin Internal restructuring: identify no longer computes syntax.
Thu, 06 Jul 2006 23:36:40 +0200 wenzelm removed obsolete locale view;
Tue, 04 Jul 2006 15:45:59 +0200 ballarin Locales no longer generate views. The following functions have changed
Tue, 04 Jul 2006 14:47:01 +0200 ballarin Method intro_locales replaced by intro_locales and unfold_locales.
Thu, 22 Jun 2006 07:08:04 +0200 ballarin Improved handling of defines imported in duplicate.
Tue, 20 Jun 2006 16:46:30 +0200 haftmann fixed sml/nj value restriction problem
Tue, 20 Jun 2006 15:53:44 +0200 ballarin Restructured locales with predicates: import is now an interpretation.
Sat, 17 Jun 2006 19:37:55 +0200 wenzelm Variable.importT_inst;
Thu, 15 Jun 2006 23:10:45 +0200 wenzelm ProofContext: moved variable operations to struct Variable;
Tue, 13 Jun 2006 23:41:31 +0200 wenzelm use Drule.unvarify instead of obsolete Drule.freeze_all;
Wed, 07 Jun 2006 02:01:33 +0200 wenzelm renamed Type.(un)varifyT to Logic.(un)varifyT;
Tue, 06 Jun 2006 10:05:57 +0200 ballarin Improved parameter management of locales.
Mon, 05 Jun 2006 21:54:26 +0200 wenzelm export read/cert_expr;
Fri, 26 May 2006 22:20:06 +0200 wenzelm activate Defines: fix frees;
Tue, 16 May 2006 21:33:16 +0200 wenzelm replaced abbrevs by term_syntax, which is both simpler and more general;
Sun, 07 May 2006 00:22:05 +0200 wenzelm removed 'concl is' patterns;
Thu, 27 Apr 2006 15:06:35 +0200 wenzelm tuned basic list operators (flat, maps, map_filter);
Thu, 13 Apr 2006 12:01:01 +0200 wenzelm use conjunction stuff from conjunction.ML;
Sat, 08 Apr 2006 22:51:26 +0200 wenzelm abbrevs: support print mode;
Mon, 20 Mar 2006 21:29:04 +0100 wenzelm interpret: Proof.assert_forward_or_chain;
Mon, 20 Mar 2006 17:15:35 +0100 ballarin Tuned signature of Locale.add_locale(_i).
Fri, 17 Mar 2006 15:22:40 +0100 ballarin add_locale(_i) returns internal locale name.
Fri, 17 Mar 2006 09:57:25 +0100 ballarin Internal restructuring: local parameters.
Thu, 16 Mar 2006 20:19:25 +0100 ballarin New interface function parameters_of_expr.
Wed, 15 Feb 2006 21:35:11 +0100 wenzelm removed distinct, renamed gen_distinct to distinct;
Sun, 12 Feb 2006 21:34:18 +0100 wenzelm simplified TableFun.join;
Sat, 11 Feb 2006 17:17:53 +0100 wenzelm added abbreviations: activated by init, no expressions yet;
Tue, 07 Feb 2006 19:56:45 +0100 wenzelm renamed gen_duplicates to duplicates;
Mon, 06 Feb 2006 20:59:52 +0100 wenzelm TableFun: renamed xxx_multi to xxx_list;
Fri, 03 Feb 2006 11:47:57 +0100 haftmann refined signature of locale module
Thu, 02 Feb 2006 16:31:35 +0100 wenzelm Proof.refine_insert;
Thu, 02 Feb 2006 12:54:08 +0100 wenzelm theorem(_in_locale): Element.statement, Obtain.statement;
Thu, 02 Feb 2006 10:12:45 +0100 ballarin *_asms_of fixed.
Sat, 28 Jan 2006 17:29:49 +0100 wenzelm LocalDefs;
Fri, 27 Jan 2006 19:03:12 +0100 wenzelm init: include view;
Fri, 27 Jan 2006 16:05:23 +0100 ballarin Interface to access the specification of a named locale.
Wed, 25 Jan 2006 00:21:40 +0100 wenzelm turned abstract_term into ProofContext.abs_def;
Tue, 24 Jan 2006 00:43:31 +0100 wenzelm removed the_params;
Sun, 22 Jan 2006 18:45:59 +0100 wenzelm added the_params;
Sat, 21 Jan 2006 23:02:14 +0100 wenzelm simplified type attribute;
Thu, 19 Jan 2006 21:22:08 +0100 wenzelm setup: theory -> theory;
Mon, 16 Jan 2006 21:55:15 +0100 wenzelm put_facts: do not pretend local thms were named;
Sat, 14 Jan 2006 17:14:06 +0100 wenzelm sane ERROR handling;
Fri, 13 Jan 2006 01:13:15 +0100 wenzelm uniform handling of fixes;
Sat, 07 Jan 2006 23:27:58 +0100 wenzelm added init;
less more (0) -100 -60 tip