clarified keywords;
authorwenzelm
Mon, 11 Jul 2016 11:15:10 +0200
changeset 63435 7743df69a6b4
parent 63434 c956d995bec6
child 63436 9974230f9574
clarified keywords;
src/Tools/Code_Generator.thy
src/ZF/Inductive_ZF.thy
--- a/src/Tools/Code_Generator.thy	Mon Jul 11 10:43:54 2016 +0200
+++ b/src/Tools/Code_Generator.thy	Mon Jul 11 11:15:10 2016 +0200
@@ -10,8 +10,10 @@
   "print_codeproc" "code_thms" "code_deps" :: diag and
   "export_code" "code_identifier" "code_printing" "code_reserved"
     "code_monad" "code_reflect" :: thy_decl and
-  "datatypes" "functions" "module_name" "file" "checking"
-  "constant" "type_constructor" "type_class" "class_relation" "class_instance" "code_module"
+  "checking" and
+  "datatypes" "functions" "module_name" "file"
+    "constant" "type_constructor" "type_class" "class_relation" "class_instance" "code_module"
+    :: quasi_command
 begin
 
 ML_file "~~/src/Tools/cache_io.ML"
--- a/src/ZF/Inductive_ZF.thy	Mon Jul 11 10:43:54 2016 +0200
+++ b/src/ZF/Inductive_ZF.thy	Mon Jul 11 11:15:10 2016 +0200
@@ -16,7 +16,7 @@
 keywords
   "inductive" "coinductive" "inductive_cases" "rep_datatype" "primrec" :: thy_decl and
   "domains" "intros" "monos" "con_defs" "type_intros" "type_elims"
-  "elimination" "induction" "case_eqns" "recursor_eqns"
+    "elimination" "induction" "case_eqns" "recursor_eqns" :: quasi_command
 begin
 
 lemma def_swap_iff: "a == b ==> a = c \<longleftrightarrow> c = b"