removed old global get_claset/map_claset;
authorwenzelm
Wed, 29 Jul 2009 00:09:14 +0200
changeset 32261 05e687ddbcee
parent 32260 eb97888fa422
child 32262 73cd8f74cf2a
removed old global get_claset/map_claset; added local get_claset/put_claset;
src/FOL/FOL.thy
src/FOL/cladata.ML
src/Provers/classical.ML
--- a/src/FOL/FOL.thy	Tue Jul 28 20:03:58 2009 +0200
+++ b/src/FOL/FOL.thy	Wed Jul 29 00:09:14 2009 +0200
@@ -168,7 +168,7 @@
 
 use "cladata.ML"
 setup Cla.setup
-setup cla_setup
+ML {* Context.>> (Cla.map_cs (K FOL_cs)) *}
 
 ML {*
   structure Blast = Blast
--- a/src/FOL/cladata.ML	Tue Jul 28 20:03:58 2009 +0200
+++ b/src/FOL/cladata.ML	Wed Jul 29 00:09:14 2009 +0200
@@ -32,4 +32,3 @@
 val FOL_cs = prop_cs addSIs [@{thm allI}, @{thm ex_ex1I}] addIs [@{thm exI}]
                      addSEs [@{thm exE}, @{thm alt_ex1E}] addEs [@{thm allE}];
 
-val cla_setup = Cla.map_claset (K FOL_cs);
--- a/src/Provers/classical.ML	Tue Jul 28 20:03:58 2009 +0200
+++ b/src/Provers/classical.ML	Wed Jul 29 00:09:14 2009 +0200
@@ -113,8 +113,8 @@
   val del_context_safe_wrapper: string -> theory -> theory
   val add_context_unsafe_wrapper: string * (Proof.context -> wrapper) -> theory -> theory
   val del_context_unsafe_wrapper: string -> theory -> theory
-  val get_claset: theory -> claset
-  val map_claset: (claset -> claset) -> theory -> theory
+  val get_claset: Proof.context -> claset
+  val put_claset: claset -> Proof.context -> Proof.context
   val get_cs: Context.generic -> claset
   val map_cs: (claset -> claset) -> Context.generic -> Context.generic
   val safe_dest: int option -> attribute
@@ -845,8 +845,8 @@
     (merge_cs (cs1, cs2), merge_context_cs (ctxt_cs1, ctxt_cs2));
 );
 
-val get_claset = #1 o GlobalClaset.get;
-val map_claset = GlobalClaset.map o apfst;
+val get_global_claset = #1 o GlobalClaset.get;
+val map_global_claset = GlobalClaset.map o apfst;
 
 val get_context_cs = #2 o GlobalClaset.get o ProofContext.theory_of;
 fun map_context_cs f = GlobalClaset.map (apsnd
@@ -871,9 +871,12 @@
 structure LocalClaset = ProofDataFun
 (
   type T = claset;
-  val init = get_claset;
+  val init = get_global_claset;
 );
 
+val get_claset = LocalClaset.get;
+val put_claset = LocalClaset.put;
+
 fun claset_of ctxt =
   context_cs ctxt (LocalClaset.get ctxt) (get_context_cs ctxt);
 
@@ -881,13 +884,13 @@
 (* generic clasets *)
 
 val get_cs = Context.cases global_claset_of claset_of;
-fun map_cs f = Context.mapping (map_claset f) (LocalClaset.map f);
+fun map_cs f = Context.mapping (map_global_claset f) (LocalClaset.map f);
 
 
 (* attributes *)
 
 fun attrib f = Thm.declaration_attribute (fn th =>
-  Context.mapping (map_claset (f th)) (LocalClaset.map (f th)));
+  Context.mapping (map_global_claset (f th)) (LocalClaset.map (f th)));
 
 fun safe_dest w = attrib (addSE w o make_elim);
 val safe_elim = attrib o addSE;