ProgTutorial/Base.thy
changeset 535 5734ab5dd86d
parent 517 d8c376662bb4
child 538 e9fd5eff62c1
--- a/ProgTutorial/Base.thy	Fri Jun 22 19:55:20 2012 +0100
+++ b/ProgTutorial/Base.thy	Mon Aug 27 10:24:10 2012 +0100
@@ -1,9 +1,10 @@
 theory Base
 imports Main 
         "~~/src/HOL/Library/LaTeXsugar"
-keywords "ML" "setup" "local_setup" :: thy_decl and
+(*keywords "ML" "setup" "local_setup" :: thy_decl and
          "ML_prf" :: prf_decl and
          "ML_val" :: diag
+*)
 uses
   ("output_tutorial.ML")
   ("antiquote_setup.ML")