removed obsolete ML_SUFFIX;
authorwenzelm
Sat, 14 Jun 2008 17:26:11 +0200
changeset 27203 9f02853e3f5b
parent 27202 1a604efd267d
child 27204 eed29f78dd9b
removed obsolete ML_SUFFIX; some reformatting;
src/FOL/IsaMakefile
src/ZF/IsaMakefile
--- a/src/FOL/IsaMakefile	Sat Jun 14 17:26:10 2008 +0200
+++ b/src/FOL/IsaMakefile	Sat Jun 14 17:26:11 2008 +0200
@@ -21,24 +21,23 @@
 
 ## FOL
 
-FOL: Pure $(OUT)/FOL$(ML_SUFFIX)
+FOL: Pure $(OUT)/FOL
 
 Pure:
 	@cd $(SRC)/Pure; $(ISATOOL) make Pure
 
-$(OUT)/Pure$(ML_SUFFIX): Pure
+$(OUT)/Pure: Pure
 
-$(OUT)/FOL$(ML_SUFFIX): $(OUT)/Pure$(ML_SUFFIX) $(SRC)/Provers/blast.ML	\
+$(OUT)/FOL: $(OUT)/Pure $(SRC)/Provers/blast.ML				\
   $(SRC)/Provers/clasimp.ML $(SRC)/Provers/classical.ML			\
-  $(SRC)/Tools/IsaPlanner/zipper.ML \
-  $(SRC)/Tools/IsaPlanner/isand.ML \
-  $(SRC)/Tools/IsaPlanner/rw_tools.ML	\
-  $(SRC)/Tools/IsaPlanner/rw_inst.ML \
-  $(SRC)/Provers/eqsubst.ML $(SRC)/Provers/hypsubst.ML			\
-  $(SRC)/Tools/induct.ML $(SRC)/Tools/atomize_elim.ML \
-  $(SRC)/Provers/project_rule.ML $(SRC)/Provers/quantifier1.ML		\
-  $(SRC)/Provers/splitter.ML FOL.thy IFOL.thy ROOT.ML blastdata.ML cladata.ML 		\
-  document/root.tex fologic.ML hypsubstdata.ML intprover.ML simpdata.ML
+  $(SRC)/Tools/IsaPlanner/zipper.ML $(SRC)/Tools/IsaPlanner/isand.ML	\
+  $(SRC)/Tools/IsaPlanner/rw_tools.ML					\
+  $(SRC)/Tools/IsaPlanner/rw_inst.ML $(SRC)/Provers/eqsubst.ML		\
+  $(SRC)/Provers/hypsubst.ML $(SRC)/Tools/induct.ML			\
+  $(SRC)/Tools/atomize_elim.ML $(SRC)/Provers/project_rule.ML		\
+  $(SRC)/Provers/quantifier1.ML $(SRC)/Provers/splitter.ML FOL.thy	\
+  IFOL.thy ROOT.ML blastdata.ML cladata.ML document/root.tex		\
+  fologic.ML hypsubstdata.ML intprover.ML simpdata.ML
 	@$(ISATOOL) usedir -p 2 -b $(OUT)/Pure FOL
 
 
@@ -46,12 +45,11 @@
 
 FOL-ex: FOL $(LOG)/FOL-ex.gz
 
-$(LOG)/FOL-ex.gz: $(OUT)/FOL$(ML_SUFFIX) ex/First_Order_Logic.thy \
-  ex/If.thy ex/IffOracle.thy ex/LocaleTest.thy \
-  ex/Nat.thy ex/Natural_Numbers.thy ex/Miniscope.thy \
-  ex/Prolog.thy ex/ROOT.ML ex/Classical.thy ex/document/root.tex \
-  ex/Foundation.thy ex/Intuitionistic.thy ex/Intro.thy \
-  ex/Propositional_Int.thy ex/Propositional_Cla.thy \
+$(LOG)/FOL-ex.gz: $(OUT)/FOL ex/First_Order_Logic.thy ex/If.thy		\
+  ex/IffOracle.thy ex/LocaleTest.thy ex/Nat.thy ex/Natural_Numbers.thy	\
+  ex/Miniscope.thy ex/Prolog.thy ex/ROOT.ML ex/Classical.thy		\
+  ex/document/root.tex ex/Foundation.thy ex/Intuitionistic.thy		\
+  ex/Intro.thy ex/Propositional_Int.thy ex/Propositional_Cla.thy	\
   ex/Quantifiers_Int.thy ex/Quantifiers_Cla.thy
 	@$(ISATOOL) usedir $(OUT)/FOL ex
 
@@ -59,4 +57,4 @@
 ## clean
 
 clean:
-	@rm -f $(OUT)/FOL$(ML_SUFFIX) $(LOG)/FOL.gz $(LOG)/FOL-ex.gz
+	@rm -f $(OUT)/FOL $(LOG)/FOL.gz $(LOG)/FOL-ex.gz
--- a/src/ZF/IsaMakefile	Sat Jun 14 17:26:10 2008 +0200
+++ b/src/ZF/IsaMakefile	Sat Jun 14 17:26:11 2008 +0200
@@ -23,23 +23,23 @@
 
 ## ZF
 
-ZF: FOL $(OUT)/ZF$(ML_SUFFIX)
+ZF: FOL $(OUT)/ZF
 
 FOL:
 	@cd $(SRC)/FOL; $(ISATOOL) make FOL
 
-$(OUT)/ZF$(ML_SUFFIX): $(OUT)/FOL$(ML_SUFFIX) AC.thy Arith.thy		\
-  ArithSimp.thy Bin.thy Bool.thy Cardinal.thy CardinalArith.thy		\
-  Cardinal_AC.thy Datatype_ZF.thy Epsilon.thy EquivClass.thy Finite.thy	\
-  Fixedpt.thy Inductive_ZF.thy InfDatatype.thy Int_ZF.thy IntArith.thy	\
-  IntDiv_ZF.thy List_ZF.thy Main.thy Main_ZF.thy Main_ZFC.thy Nat_ZF.thy OrdQuant.thy	\
-  Order.thy OrderArith.thy OrderType.thy Ordinal.thy Perm.thy QPair.thy	\
-  QUniv.thy ROOT.ML Sum.thy Tools/cartprod.ML Tools/datatype_package.ML	\
-  Tools/ind_cases.ML Tools/induct_tacs.ML Tools/inductive_package.ML	\
-  Tools/numeral_syntax.ML Tools/primrec_package.ML Tools/typechk.ML	\
-  Trancl.thy Univ.thy WF.thy ZF.thy Zorn.thy arith_data.ML		\
-  equalities.thy func.thy ind_syntax.ML int_arith.ML pair.thy		\
-  simpdata.ML upair.thy
+$(OUT)/ZF: $(OUT)/FOL AC.thy Arith.thy ArithSimp.thy Bin.thy Bool.thy	\
+  Cardinal.thy CardinalArith.thy Cardinal_AC.thy Datatype_ZF.thy	\
+  Epsilon.thy EquivClass.thy Finite.thy Fixedpt.thy Inductive_ZF.thy	\
+  InfDatatype.thy Int_ZF.thy IntArith.thy IntDiv_ZF.thy List_ZF.thy	\
+  Main.thy Main_ZF.thy Main_ZFC.thy Nat_ZF.thy OrdQuant.thy Order.thy	\
+  OrderArith.thy OrderType.thy Ordinal.thy Perm.thy QPair.thy		\
+  QUniv.thy ROOT.ML Sum.thy Tools/cartprod.ML				\
+  Tools/datatype_package.ML Tools/ind_cases.ML Tools/induct_tacs.ML	\
+  Tools/inductive_package.ML Tools/numeral_syntax.ML			\
+  Tools/primrec_package.ML Tools/typechk.ML Trancl.thy Univ.thy WF.thy	\
+  ZF.thy Zorn.thy arith_data.ML equalities.thy func.thy ind_syntax.ML	\
+  int_arith.ML pair.thy simpdata.ML upair.thy
 	@$(ISATOOL) usedir -b -r $(OUT)/FOL ZF
 
 
@@ -47,12 +47,11 @@
 
 ZF-AC: ZF $(LOG)/ZF-AC.gz
 
-$(LOG)/ZF-AC.gz: $(OUT)/ZF$(ML_SUFFIX) \
-  AC/ROOT.ML  AC/AC15_WO6.thy AC/AC16_WO4.thy \
-  AC/AC16_lemmas.thy AC/AC17_AC1.thy AC/AC18_AC19.thy AC/AC7_AC9.thy \
-  AC/AC_Equiv.thy AC/Cardinal_aux.thy \
-  AC/DC.thy AC/HH.thy AC/Hartog.thy AC/WO1_AC.thy AC/WO1_WO7.thy \
-  AC/WO2_AC16.thy AC/WO6_WO1.thy AC/document/root.bib AC/document/root.tex
+$(LOG)/ZF-AC.gz: $(OUT)/ZF AC/ROOT.ML AC/AC15_WO6.thy AC/AC16_WO4.thy	\
+  AC/AC16_lemmas.thy AC/AC17_AC1.thy AC/AC18_AC19.thy AC/AC7_AC9.thy	\
+  AC/AC_Equiv.thy AC/Cardinal_aux.thy AC/DC.thy AC/HH.thy		\
+  AC/Hartog.thy AC/WO1_AC.thy AC/WO1_WO7.thy AC/WO2_AC16.thy		\
+  AC/WO6_WO1.thy AC/document/root.bib AC/document/root.tex
 	@$(ISATOOL) usedir -g true $(OUT)/ZF AC
 
 
@@ -60,9 +59,9 @@
 
 ZF-Coind: ZF $(LOG)/ZF-Coind.gz
 
-$(LOG)/ZF-Coind.gz: $(OUT)/ZF$(ML_SUFFIX) Coind/Dynamic.thy \
-  Coind/ECR.thy Coind/Language.thy Coind/Map.thy Coind/ROOT.ML \
-  Coind/Static.thy Coind/Types.thy Coind/Values.thy
+$(LOG)/ZF-Coind.gz: $(OUT)/ZF Coind/Dynamic.thy Coind/ECR.thy		\
+  Coind/Language.thy Coind/Map.thy Coind/ROOT.ML Coind/Static.thy	\
+  Coind/Types.thy Coind/Values.thy
 	@$(ISATOOL) usedir $(OUT)/ZF Coind
 
 
@@ -70,16 +69,16 @@
 
 ZF-Constructible: ZF $(LOG)/ZF-Constructible.gz
 
-$(LOG)/ZF-Constructible.gz: $(OUT)/ZF$(ML_SUFFIX)  Constructible/ROOT.ML \
-  Constructible/Datatype_absolute.thy Constructible/DPow_absolute.thy\
-  Constructible/Formula.thy Constructible/Internalize.thy \
-  Constructible/AC_in_L.thy Constructible/Relative.thy \
-  Constructible/L_axioms.thy    Constructible/Wellorderings.thy \
-  Constructible/MetaExists.thy  Constructible/Normal.thy \
-  Constructible/Rank.thy Constructible/Rank_Separation.thy \
-  Constructible/Rec_Separation.thy Constructible/Separation.thy \
-  Constructible/Satisfies_absolute.thy Constructible/WF_absolute.thy \
-  Constructible/Reflection.thy  Constructible/WFrec.thy \
+$(LOG)/ZF-Constructible.gz: $(OUT)/ZF Constructible/ROOT.ML		\
+  Constructible/Datatype_absolute.thy Constructible/DPow_absolute.thy	\
+  Constructible/Formula.thy Constructible/Internalize.thy		\
+  Constructible/AC_in_L.thy Constructible/Relative.thy			\
+  Constructible/L_axioms.thy Constructible/Wellorderings.thy		\
+  Constructible/MetaExists.thy Constructible/Normal.thy			\
+  Constructible/Rank.thy Constructible/Rank_Separation.thy		\
+  Constructible/Rec_Separation.thy Constructible/Separation.thy		\
+  Constructible/Satisfies_absolute.thy Constructible/WF_absolute.thy	\
+  Constructible/Reflection.thy Constructible/WFrec.thy			\
   Constructible/document/root.bib Constructible/document/root.tex
 	@$(ISATOOL) usedir -g true $(OUT)/ZF Constructible
 
@@ -88,8 +87,9 @@
 
 ZF-IMP: ZF $(LOG)/ZF-IMP.gz
 
-$(LOG)/ZF-IMP.gz: $(OUT)/ZF$(ML_SUFFIX) IMP/Com.thy IMP/Denotation.thy IMP/Equiv.thy \
-  IMP/ROOT.ML IMP/document/root.bib IMP/document/root.tex
+$(LOG)/ZF-IMP.gz: $(OUT)/ZF IMP/Com.thy IMP/Denotation.thy	\
+  IMP/Equiv.thy IMP/ROOT.ML IMP/document/root.bib		\
+  IMP/document/root.tex
 	@$(ISATOOL) usedir $(OUT)/ZF IMP
 
 
@@ -97,9 +97,9 @@
 
 ZF-Resid: ZF $(LOG)/ZF-Resid.gz
 
-$(LOG)/ZF-Resid.gz: $(OUT)/ZF$(ML_SUFFIX) Resid/ROOT.ML \
-  Resid/Confluence.thy  Resid/Redex.thy \
-  Resid/Reduction.thy Resid/Residuals.thy Resid/Substitution.thy 
+$(LOG)/ZF-Resid.gz: $(OUT)/ZF Resid/ROOT.ML Resid/Confluence.thy	\
+  Resid/Redex.thy Resid/Reduction.thy Resid/Residuals.thy		\
+  Resid/Substitution.thy
 	@$(ISATOOL) usedir $(OUT)/ZF Resid
 
 
@@ -107,14 +107,13 @@
 
 ZF-UNITY: ZF $(LOG)/ZF-UNITY.gz
 
-$(LOG)/ZF-UNITY.gz: $(OUT)/ZF$(ML_SUFFIX) UNITY/ROOT.ML \
-  UNITY/Comp.thy UNITY/Constrains.thy UNITY/FP.thy\
-  UNITY/GenPrefix.thy UNITY/Guar.thy UNITY/Mutex.thy UNITY/State.thy \
-  UNITY/SubstAx.thy UNITY/UNITY.thy UNITY/Union.thy \
-  UNITY/AllocBase.thy UNITY/AllocImpl.thy\
-  UNITY/ClientImpl.thy UNITY/Distributor.thy\
-  UNITY/Follows.thy UNITY/Increasing.thy UNITY/Merge.thy\
-  UNITY/Monotonicity.thy UNITY/MultisetSum.thy UNITY/WFair.thy
+$(LOG)/ZF-UNITY.gz: $(OUT)/ZF UNITY/ROOT.ML UNITY/Comp.thy		\
+  UNITY/Constrains.thy UNITY/FP.thy UNITY/GenPrefix.thy UNITY/Guar.thy	\
+  UNITY/Mutex.thy UNITY/State.thy UNITY/SubstAx.thy UNITY/UNITY.thy	\
+  UNITY/Union.thy UNITY/AllocBase.thy UNITY/AllocImpl.thy		\
+  UNITY/ClientImpl.thy UNITY/Distributor.thy UNITY/Follows.thy		\
+  UNITY/Increasing.thy UNITY/Merge.thy UNITY/Monotonicity.thy		\
+  UNITY/MultisetSum.thy UNITY/WFair.thy
 	@$(ISATOOL) usedir $(OUT)/ZF UNITY
 
 
@@ -122,11 +121,11 @@
 
 ZF-Induct: ZF $(LOG)/ZF-Induct.gz
 
-$(LOG)/ZF-Induct.gz: $(OUT)/ZF$(ML_SUFFIX)  Induct/ROOT.ML Induct/Acc.thy \
-  Induct/Binary_Trees.thy Induct/Brouwer.thy Induct/Comb.thy \
-  Induct/Datatypes.thy Induct/FoldSet.thy \
-  Induct/ListN.thy Induct/Multiset.thy Induct/Mutil.thy \
-  Induct/Ntree.thy Induct/Primrec.thy Induct/PropLog.thy Induct/Rmap.thy \
+$(LOG)/ZF-Induct.gz: $(OUT)/ZF Induct/ROOT.ML Induct/Acc.thy		\
+  Induct/Binary_Trees.thy Induct/Brouwer.thy Induct/Comb.thy		\
+  Induct/Datatypes.thy Induct/FoldSet.thy Induct/ListN.thy		\
+  Induct/Multiset.thy Induct/Mutil.thy Induct/Ntree.thy			\
+  Induct/Primrec.thy Induct/PropLog.thy Induct/Rmap.thy			\
   Induct/Term.thy Induct/Tree_Forest.thy Induct/document/root.tex
 	@$(ISATOOL) usedir $(OUT)/ZF Induct
 
@@ -135,17 +134,16 @@
 
 ZF-ex: ZF $(LOG)/ZF-ex.gz
 
-$(LOG)/ZF-ex.gz: $(OUT)/ZF$(ML_SUFFIX) ex/ROOT.ML \
-  ex/BinEx.thy ex/CoUnit.thy ex/Commutation.thy ex/Group.thy\
-  ex/Limit.thy ex/LList.thy ex/Primes.thy \
-  ex/NatSum.thy ex/Ramsey.thy ex/Ring.thy ex/misc.thy
+$(LOG)/ZF-ex.gz: $(OUT)/ZF ex/ROOT.ML ex/BinEx.thy ex/CoUnit.thy	\
+  ex/Commutation.thy ex/Group.thy ex/Limit.thy ex/LList.thy		\
+  ex/Primes.thy ex/NatSum.thy ex/Ramsey.thy ex/Ring.thy ex/misc.thy
 	@$(ISATOOL) usedir $(OUT)/ZF ex
 
 
 ## clean
 
 clean:
-	@rm -f $(OUT)/ZF$(ML_SUFFIX) $(LOG)/ZF.gz $(LOG)/ZF-AC.gz $(LOG)/ZF-Coind.gz \
+	@rm -f $(OUT)/ZF $(LOG)/ZF.gz $(LOG)/ZF-AC.gz $(LOG)/ZF-Coind.gz \
 	  $(LOG)/ZF-Constructible.gz $(LOG)/ZF-ex.gz \
           $(LOG)/ZF-IMP.gz $(LOG)/ZF-Resid.gz \
 	  $(LOG)/ZF-UNITY.gz