src/Pure/goal.ML
changeset 78048 ec817f4486b3
parent 78046 78deba4fdf27
child 78084 f0aca0506531
--- a/src/Pure/goal.ML	Mon May 15 12:14:47 2023 +0200
+++ b/src/Pure/goal.ML	Mon May 15 14:09:45 2023 +0200
@@ -22,6 +22,7 @@
   val check_finished: Proof.context -> thm -> thm
   val finish: Proof.context -> thm -> thm
   val norm_result: Proof.context -> thm -> thm
+  val norm_result_without_context: thm -> thm
   val skip_proofs_enabled: unit -> bool
   val future_result: Proof.context -> thm future -> term -> thm
   val prove_internal: Proof.context -> cterm list -> cterm -> (thm list -> tactic) -> thm
@@ -96,6 +97,9 @@
   #> Thm.strip_shyps
   #> Drule.zero_var_indexes;
 
+fun norm_result_without_context th =
+  norm_result (Proof_Context.init_global (Thm.theory_of_thm th)) th;
+
 
 (* scheduling parameters *)