src/Pure/Pure.thy
changeset 60371 8a5cfdda1b98
parent 60317 9b7248379101
child 60448 78f3c67bc35e
--- a/src/Pure/Pure.thy	Fri Jun 05 13:26:12 2015 +0200
+++ b/src/Pure/Pure.thy	Fri Jun 05 13:41:06 2015 +0200
@@ -51,7 +51,9 @@
   and "show" :: prf_asm_goal % "proof"
   and "thus" :: prf_asm_goal % "proof" == "then show"
   and "then" "from" "with" :: prf_chain % "proof"
-  and "note" "using" "unfolding" :: prf_decl % "proof"
+  and "note" :: prf_decl % "proof"
+  and "supply" :: prf_script % "proof"
+  and "using" "unfolding" :: prf_decl % "proof"
   and "fix" "assume" "presume" "def" :: prf_asm % "proof"
   and "obtain" :: prf_asm_goal % "proof"
   and "guess" :: prf_asm_goal_script % "proof"