src/Pure/Pure.thy
changeset 58842 22b87ab47d3b
parent 58800 bfed1c26caed
child 58845 8451eddc4d67
equal deleted inserted replaced
58840:f4bb3068d819 58842:22b87ab47d3b
    98   and "realizers" :: thy_decl == ""
    98   and "realizers" :: thy_decl == ""
    99   and "realizability" :: thy_decl == ""
    99   and "realizability" :: thy_decl == ""
   100   and "extract_type" "extract" :: thy_decl
   100   and "extract_type" "extract" :: thy_decl
   101   and "find_theorems" "find_consts" :: diag
   101   and "find_theorems" "find_consts" :: diag
   102   and "named_theorems" :: thy_decl
   102   and "named_theorems" :: thy_decl
   103   and "ProofGeneral.process_pgip" "ProofGeneral.pr" "ProofGeneral.undo"
       
   104     "ProofGeneral.restart" "ProofGeneral.kill_proof" "ProofGeneral.inform_file_processed"
       
   105     "ProofGeneral.inform_file_retracted" :: control
       
   106 begin
   103 begin
   107 
   104 
   108 ML_file "ML/ml_antiquotations.ML"
   105 ML_file "ML/ml_antiquotations.ML"
   109 ML_file "ML/ml_thms.ML"
   106 ML_file "ML/ml_thms.ML"
   110 ML_file "Tools/print_operation.ML"
   107 ML_file "Tools/print_operation.ML"
   115 ML_file "Tools/rule_insts.ML";
   112 ML_file "Tools/rule_insts.ML";
   116 ML_file "Tools/thm_deps.ML";
   113 ML_file "Tools/thm_deps.ML";
   117 ML_file "Tools/class_deps.ML"
   114 ML_file "Tools/class_deps.ML"
   118 ML_file "Tools/find_theorems.ML"
   115 ML_file "Tools/find_theorems.ML"
   119 ML_file "Tools/find_consts.ML"
   116 ML_file "Tools/find_consts.ML"
   120 ML_file "Tools/proof_general_pure.ML"
       
   121 ML_file "Tools/simplifier_trace.ML"
   117 ML_file "Tools/simplifier_trace.ML"
   122 ML_file "Tools/named_theorems.ML"
   118 ML_file "Tools/named_theorems.ML"
   123 
   119 
   124 
   120 
   125 section \<open>Basic attributes\<close>
   121 section \<open>Basic attributes\<close>