src/HOL/HOL.thy
changeset 52432 c03090937c3b
parent 52230 1105b3b5aa77
child 52435 6646bb548c6b
--- a/src/HOL/HOL.thy	Sun Jun 23 21:40:56 2013 +0200
+++ b/src/HOL/HOL.thy	Sun Jun 23 22:31:50 2013 +0200
@@ -7,8 +7,8 @@
 theory HOL
 imports Pure "~~/src/Tools/Code_Generator"
 keywords
-  "try" "solve_direct" "quickcheck"
-    "print_coercions" "print_coercion_maps" "print_claset" "print_induct_rules" :: diag and
+  "try" "solve_direct" "quickcheck" "print_coercions" "print_claset"
+    "print_induct_rules" :: diag and
   "quickcheck_params" :: thy_decl
 begin