tuned signature;
authorwenzelm
Tue, 20 Feb 2018 16:20:36 +0100
changeset 67679 8fd84fe1d60b
parent 67678 b4db2e7e414e
child 67680 175a070e9dd8
tuned signature;
src/Pure/Isar/proof_context.ML
--- 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) ->