tuned signature;
authorwenzelm
Mon, 04 Jul 2016 10:29:56 +0200
changeset 63368 e9e677b73011
parent 63367 6c731c8b7f03
child 63369 4698dd1106ae
tuned signature;
src/Pure/Isar/calculation.ML
src/Pure/Isar/proof.ML
--- a/src/Pure/Isar/calculation.ML	Sat Jul 02 20:22:25 2016 +0200
+++ b/src/Pure/Isar/calculation.ML	Mon Jul 04 10:29:56 2016 +0200
@@ -61,7 +61,7 @@
 fun put_calculation calc =
   `Proof.level #-> (fn lev => Proof.map_context (Context.proof_map
      (Data.map (apsnd (K (Option.map (rpair lev) calc))))))
-  #> Proof.put_thms false (calculationN, calc);
+  #> Proof.map_context (Proof_Context.put_thms false (calculationN, calc));
 
 
 
--- a/src/Pure/Isar/proof.ML	Sat Jul 02 20:22:25 2016 +0200
+++ b/src/Pure/Isar/proof.ML	Mon Jul 04 10:29:56 2016 +0200
@@ -19,7 +19,6 @@
   val map_context_result : (context -> 'a * context) -> state -> 'a * state
   val map_contexts: (context -> context) -> state -> state
   val propagate_ml_env: state -> state
-  val put_thms: bool -> string * thm list option -> state -> state
   val the_facts: state -> thm list
   val the_fact: state -> thm
   val set_facts: thm list -> state -> state
@@ -241,8 +240,6 @@
 fun propagate_ml_env state = map_contexts
   (Context.proof_map (ML_Env.inherit (Context.Proof (context_of state)))) state;
 
-val put_thms = map_context oo Proof_Context.put_thms;
-
 
 (* facts *)
 
@@ -260,7 +257,7 @@
 
 fun put_facts facts =
   map_top (fn (ctxt, _, mode, goal) => (ctxt, facts, mode, goal)) #>
-  put_thms true (Auto_Bind.thisN, facts);
+  map_context (Proof_Context.put_thms true (Auto_Bind.thisN, facts));
 
 val set_facts = put_facts o SOME;
 val reset_facts = put_facts NONE;