src/Pure/Pure.thy
changeset 52437 c88354589b43
parent 52430 289e36c2870a
child 52438 7b5a5116f3af
--- a/src/Pure/Pure.thy	Mon Jun 24 13:54:57 2013 +0200
+++ b/src/Pure/Pure.thy	Mon Jun 24 17:03:53 2013 +0200
@@ -93,6 +93,9 @@
   and "end" :: thy_end % "theory"
   and "realizers" "realizability" "extract_type" "extract" :: thy_decl
   and "find_theorems" "find_consts" :: diag
+  and "ProofGeneral.process_pgip" "ProofGeneral.pr" "ProofGeneral.undo"
+    "ProofGeneral.restart" "ProofGeneral.kill_proof" "ProofGeneral.inform_file_processed"
+    "ProofGeneral.inform_file_retracted" :: control
 begin
 
 ML_file "Isar/isar_syn.ML"