src/Pure/IsaMakefile
changeset 16032 bbc85a9748fc
parent 15823 d1001770af17
child 16108 cf468b93a02e
--- a/src/Pure/IsaMakefile	Sun May 22 16:51:19 2005 +0200
+++ b/src/Pure/IsaMakefile	Sun May 22 16:53:11 2005 +0200
@@ -23,8 +23,8 @@
 
 Pure: $(OUT)/Pure
 
-$(OUT)/Pure: General/ROOT.ML General/buffer.ML General/file.ML		\
-  General/graph.ML General/heap.ML General/history.ML			\
+$(OUT)/Pure: CPure.thy General/ROOT.ML General/buffer.ML		\
+  General/file.ML General/graph.ML General/heap.ML General/history.ML	\
   General/lazy_scan.ML General/lazy_seq.ML General/name_space.ML	\
   General/object.ML General/output.ML General/path.ML			\
   General/position.ML General/pretty.ML General/scan.ML General/seq.ML	\
@@ -34,31 +34,31 @@
   IsaPlanner/rw_inst.ML IsaPlanner/rw_tools.ML IsaPlanner/term_lib.ML	\
   IsaPlanner/upterm_lib.ML Isar/ROOT.ML Isar/antiquote.ML Isar/args.ML	\
   Isar/attrib.ML Isar/auto_bind.ML Isar/calculation.ML			\
-  Isar/constdefs.ML Isar/context_rules.ML Isar/induct_attrib.ML		\
-  Isar/isar_cmd.ML Isar/isar_output.ML Isar/isar_syn.ML			\
-  Isar/isar_thy.ML Isar/locale.ML Isar/method.ML Isar/net_rules.ML	\
-  Isar/object_logic.ML Isar/obtain.ML Isar/outer_lex.ML			\
-  Isar/outer_parse.ML Isar/outer_syntax.ML Isar/proof.ML		\
-  Isar/proof_context.ML Isar/proof_data.ML Isar/proof_history.ML	\
-  Isar/rule_cases.ML Isar/session.ML Isar/skip_proof.ML			\
-  Isar/thy_header.ML Isar/toplevel.ML ML-Systems/cpu-timer-basis.ML	\
-  ML-Systems/cpu-timer-gc.ML ML-Systems/polyml-time-limit.ML		\
-  ML-Systems/polyml.ML ML-Systems/smlnj-basis-compat.ML			\
-  ML-Systems/smlnj-compiler.ML ML-Systems/smlnj-pp-new.ML		\
-  ML-Systems/smlnj-pp-old.ML ML-Systems/smlnj.ML Proof/extraction.ML	\
-  Proof/proof_rewrite_rules.ML Proof/proof_syntax.ML			\
-  Proof/proofchecker.ML Proof/reconstruct.ML Pure.thy ROOT.ML		\
-  Syntax/ROOT.ML Syntax/ast.ML Syntax/lexicon.ML Syntax/mixfix.ML	\
-  Syntax/parser.ML Syntax/printer.ML Syntax/syn_ext.ML			\
-  Syntax/syn_trans.ML Syntax/syntax.ML Syntax/type_ext.ML Thy/html.ML	\
-  Thy/latex.ML Thy/present.ML Thy/thm_database.ML Thy/thm_deps.ML	\
-  Thy/thy_info.ML Thy/thy_load.ML Thy/thy_parse.ML Thy/thy_scan.ML	\
-  Thy/thy_syn.ML axclass.ML codegen.ML context.ML display.ML drule.ML	\
-  envir.ML fact_index.ML goals.ML install_pp.ML library.ML logic.ML	\
-  meta_simplifier.ML net.ML pattern.ML proof_general.ML proofterm.ML	\
-  pure_thy.ML search.ML sign.ML sorts.ML tactic.ML tctical.ML term.ML	\
-  theory.ML theory_data.ML thm.ML type.ML type_infer.ML unify.ML	\
-  CPure.thy
+  Isar/constdefs.ML Isar/context_rules.ML Isar/find_theorems.ML		\
+  Isar/induct_attrib.ML Isar/isar_cmd.ML Isar/isar_output.ML		\
+  Isar/isar_syn.ML Isar/isar_thy.ML Isar/locale.ML Isar/method.ML	\
+  Isar/net_rules.ML Isar/object_logic.ML Isar/obtain.ML			\
+  Isar/outer_lex.ML Isar/outer_parse.ML Isar/outer_syntax.ML		\
+  Isar/proof.ML Isar/proof_context.ML Isar/proof_data.ML		\
+  Isar/proof_history.ML Isar/rule_cases.ML Isar/session.ML		\
+  Isar/skip_proof.ML Isar/thy_header.ML Isar/toplevel.ML		\
+  ML-Systems/cpu-timer-basis.ML ML-Systems/cpu-timer-gc.ML		\
+  ML-Systems/polyml-time-limit.ML ML-Systems/polyml.ML			\
+  ML-Systems/smlnj-basis-compat.ML ML-Systems/smlnj-compiler.ML		\
+  ML-Systems/smlnj-pp-new.ML ML-Systems/smlnj-pp-old.ML			\
+  ML-Systems/smlnj.ML Proof/extraction.ML Proof/proof_rewrite_rules.ML	\
+  Proof/proof_syntax.ML Proof/proofchecker.ML Proof/reconstruct.ML	\
+  Pure.thy ROOT.ML Syntax/ROOT.ML Syntax/ast.ML Syntax/lexicon.ML	\
+  Syntax/mixfix.ML Syntax/parser.ML Syntax/printer.ML			\
+  Syntax/syn_ext.ML Syntax/syn_trans.ML Syntax/syntax.ML		\
+  Syntax/type_ext.ML Thy/html.ML Thy/latex.ML Thy/present.ML		\
+  Thy/thm_database.ML Thy/thm_deps.ML Thy/thy_info.ML Thy/thy_load.ML	\
+  Thy/thy_parse.ML Thy/thy_scan.ML Thy/thy_syn.ML axclass.ML		\
+  codegen.ML context.ML display.ML drule.ML envir.ML fact_index.ML	\
+  goals.ML install_pp.ML library.ML logic.ML meta_simplifier.ML net.ML	\
+  pattern.ML proof_general.ML proofterm.ML pure_thy.ML search.ML	\
+  sign.ML simplifier.ML sorts.ML tactic.ML tctical.ML term.ML		\
+  theory.ML theory_data.ML thm.ML type.ML type_infer.ML unify.ML
 	@./mk