ProgTutorial/Package/Simple_Inductive_Package.thy
changeset 514 7e25716c3744
parent 442 7e33ba6190de
child 538 e9fd5eff62c1
--- a/ProgTutorial/Package/Simple_Inductive_Package.thy	Sun Feb 19 01:33:47 2012 +0000
+++ b/ProgTutorial/Package/Simple_Inductive_Package.thy	Tue Mar 20 09:39:44 2012 +0000
@@ -1,5 +1,6 @@
 theory Simple_Inductive_Package
 imports Main "../Base"
+keywords "simple_inductive" :: thy_decl
 uses "simple_inductive_package.ML"
 begin