src/Pure/Isar/local_theory.ML
changeset 78035 bd5f6cee8001
parent 74338 534b231ce041
child 78064 4e865c45458b
--- a/src/Pure/Isar/local_theory.ML	Thu May 11 14:17:24 2023 +0200
+++ b/src/Pure/Isar/local_theory.ML	Thu May 11 21:32:22 2023 +0200
@@ -43,6 +43,7 @@
   val target: (Proof.context -> Proof.context) -> local_theory -> local_theory
   val target_morphism: local_theory -> morphism
   val propagate_ml_env: generic_theory -> generic_theory
+  val touch_ml_env: generic_theory -> generic_theory
   val operations_of: local_theory -> operations
   val define: (binding * mixfix) * (Attrib.binding * term) -> local_theory ->
     (term * (string * thm)) * local_theory
@@ -253,6 +254,13 @@
       end
   | propagate_ml_env context = context;
 
+fun touch_ml_env context =
+  if Context.enabled_tracing () then
+    (case context of
+      Context.Theory _ => ML_Env.touch context
+    | Context.Proof _ => context)
+  else context;
+
 
 
 (** operations **)