paulson [Mon, 23 Jan 2006 11:36:05 +0100] rev 18749
replacement of bool by a datatype (making problems first-order). More lemma names
mengj [Mon, 23 Jan 2006 10:34:38 +0100] rev 18748
Fixed a bug.
urbanc [Sun, 22 Jan 2006 22:16:34 +0100] rev 18747
no essential changes
urbanc [Sun, 22 Jan 2006 22:11:50 +0100] rev 18746
made the change for setup-functions not returning functions
anymore
urbanc [Sun, 22 Jan 2006 21:58:43 +0100] rev 18745
a fixme comments about abs_fun_if, which should be called perm_if
and moved to the "bool"-section
wenzelm [Sun, 22 Jan 2006 18:46:01 +0100] rev 18744
Local theory operations, with optional target locale.
wenzelm [Sun, 22 Jan 2006 18:46:00 +0100] rev 18743
added restore_body;
wenzelm [Sun, 22 Jan 2006 18:45:59 +0100] rev 18742
added the_params;
wenzelm [Sun, 22 Jan 2006 18:45:58 +0100] rev 18741
tuned order;
wenzelm [Sun, 22 Jan 2006 18:45:57 +0100] rev 18740
added Isar/local_theory.ML;
mengj [Sat, 21 Jan 2006 23:22:40 +0100] rev 18739
Ensure dereference is delayed.
wenzelm [Sat, 21 Jan 2006 23:07:26 +0100] rev 18738
tuned;
wenzelm [Sat, 21 Jan 2006 23:02:30 +0100] rev 18737
* ML: simplified type attribute;
wenzelm [Sat, 21 Jan 2006 23:02:29 +0100] rev 18736
simplified type attribute;
removed obsolete tcset operations -- clean data/attribute/method setup;
wenzelm [Sat, 21 Jan 2006 23:02:28 +0100] rev 18735
removed duplicate type_solver (cf. Tools/typechk.ML);
wenzelm [Sat, 21 Jan 2006 23:02:27 +0100] rev 18734
simplified type attribute;
removed rule/declaration (cf. thm.ML);
removed obsolete theory/proof/generic/common;
removed obsolete global/local/context_attribute(_i);
added attribute(_i);
renamed attribute to internal;
wenzelm [Sat, 21 Jan 2006 23:02:25 +0100] rev 18733
simplified type attribute;
added rule/declaration_attribute (from drule.ML);
added theory/proof_attributes;
removed apply(s)_attributes;
wenzelm [Sat, 21 Jan 2006 23:02:24 +0100] rev 18732
simplified type attribute;
moved rule/declaration_attribute to thm.ML;
wenzelm [Sat, 21 Jan 2006 23:02:23 +0100] rev 18731
rename map_theory/proof to theory/proof_map;
added separate map_theory/proof;
wenzelm [Sat, 21 Jan 2006 23:02:21 +0100] rev 18730
tuned proofs;
wenzelm [Sat, 21 Jan 2006 23:02:20 +0100] rev 18729
simplified type attribute;
tuned;
wenzelm [Sat, 21 Jan 2006 23:02:14 +0100] rev 18728
simplified type attribute;
mengj [Fri, 20 Jan 2006 04:53:59 +0100] rev 18727
type information is now also printed.
mengj [Fri, 20 Jan 2006 04:50:01 +0100] rev 18726
added some debugging code.
mengj [Fri, 20 Jan 2006 04:35:23 +0100] rev 18725
fixed a bug
wenzelm [Thu, 19 Jan 2006 21:22:30 +0100] rev 18724
quote "atom";
wenzelm [Thu, 19 Jan 2006 21:22:29 +0100] rev 18723
updated;
wenzelm [Thu, 19 Jan 2006 21:22:27 +0100] rev 18722
* ML/Isar: theory setup has type (theory -> theory);
wenzelm [Thu, 19 Jan 2006 21:22:26 +0100] rev 18721
use/use_thy: Output.toplevel_errors;
wenzelm [Thu, 19 Jan 2006 21:22:25 +0100] rev 18720
added basic syntax;
removed pure syntax;