src/Pure/Isar/proof_context.ML
changeset 67679 8fd84fe1d60b
parent 67671 857da80611ab
child 67713 041898537c19
--- a/src/Pure/Isar/proof_context.ML	Tue Feb 20 16:20:14 2018 +0100
+++ b/src/Pure/Isar/proof_context.ML	Tue Feb 20 16:20:36 2018 +0100
@@ -125,6 +125,7 @@
   val get_fact_single: Proof.context -> Facts.ref -> thm
   val get_thms: Proof.context -> xstring -> thm list
   val get_thm: Proof.context -> xstring -> thm
+  val is_stmt: Proof.context -> bool
   val set_stmt: bool -> Proof.context -> Proof.context
   val restore_stmt: Proof.context -> Proof.context -> Proof.context
   val add_thms_dynamic: binding * (Context.generic -> thm list) ->