src/ZF/IsaMakefile
author paulson
Tue, 21 May 2002 13:06:36 +0200
changeset 13168 afcbca3498b0
parent 13165 31d020705aff
child 13169 394a6c649547
permissions -rw-r--r--
converted domrange to Isar and merged with equalities

#
# $Id$
#
# IsaMakefile for ZF
#

## targets

default: ZF
images: ZF

#Note: keep targets sorted
test: ZF-AC ZF-Coind ZF-IMP ZF-Induct ZF-Resid ZF-UNITY ZF-ex
all: images test


## global settings

SRC = $(ISABELLE_HOME)/src
OUT = $(ISABELLE_OUTPUT)
LOG = $(OUT)/log


## ZF

ZF: FOL $(OUT)/ZF

FOL:
	@cd $(SRC)/FOL; $(ISATOOL) make FOL

$(OUT)/ZF: $(OUT)/FOL AC.thy Arith.thy ArithSimp.ML	\
  ArithSimp.thy Bool.ML Bool.thy Cardinal.ML Cardinal.thy		\
  CardinalArith.ML CardinalArith.thy Cardinal_AC.thy \
  Datatype.ML Datatype.thy Epsilon.thy Finite.ML Finite.thy	\
  Fixedpt.ML Fixedpt.thy Inductive.ML Inductive.thy 	\
  InfDatatype.thy Integ/Bin.ML Integ/Bin.thy Integ/EquivClass.ML	\
  Integ/EquivClass.thy Integ/Int.ML Integ/Int.thy Integ/IntArith.thy	\
  Integ/IntDiv.ML Integ/IntDiv.thy Integ/int_arith.ML			\
  Integ/twos_compl.ML Let.ML Let.thy List.ML List.thy Main.ML Main.thy	\
  Main_ZFC.ML Main_ZFC.thy	\
  Nat.ML Nat.thy Order.thy OrderArith.thy	\
  OrderType.thy Ordinal.thy OrdQuant.ML OrdQuant.thy Perm.ML Perm.thy	\
  QPair.ML QPair.thy QUniv.ML QUniv.thy ROOT.ML Rel.ML Rel.thy Sum.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.ML Trancl.thy Univ.thy Update.ML Update.thy \
  WF.thy ZF.ML ZF.thy Zorn.thy arith_data.ML equalities.thy func.thy	\
  ind_syntax.ML mono.ML mono.thy pair.ML pair.thy simpdata.ML		\
  subset.ML subset.thy thy_syntax.ML upair.ML upair.thy
	@$(ISATOOL) usedir -b -r $(OUT)/FOL ZF


## ZF-AC

ZF-AC: ZF $(LOG)/ZF-AC.gz

$(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 
	@$(ISATOOL) usedir $(OUT)/ZF AC


## ZF-Coind

ZF-Coind: ZF $(LOG)/ZF-Coind.gz

$(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


## ZF-IMP

ZF-IMP: ZF $(LOG)/ZF-IMP.gz

$(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


## ZF-Resid

ZF-Resid: ZF $(LOG)/ZF-Resid.gz

$(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


## ZF-UNITY

ZF-UNITY: ZF $(LOG)/ZF-UNITY.gz

$(LOG)/ZF-UNITY.gz: $(OUT)/ZF UNITY/ROOT.ML \
  UNITY/Comp.ML UNITY/Comp.thy UNITY/Constrains.ML UNITY/Constrains.thy \
  UNITY/FP.ML UNITY/FP.thy UNITY/Guar.ML UNITY/Guar.thy \
  UNITY/Mutex.ML UNITY/Mutex.thy UNITY/State.ML UNITY/State.thy \
  UNITY/SubstAx.ML UNITY/SubstAx.thy UNITY/UNITY.ML UNITY/UNITY.thy \
  UNITY/UNITYMisc.ML UNITY/UNITYMisc.thy UNITY/Union.ML UNITY/Union.thy \
  UNITY/WFair.ML UNITY/WFair.thy
	@$(ISATOOL) usedir $(OUT)/ZF UNITY


## ZF-Induct

ZF-Induct: ZF $(LOG)/ZF-Induct.gz

$(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.ML Induct/FoldSet.thy \
  Induct/ListN.thy Induct/Multiset.ML 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


## ZF-ex

ZF-ex: ZF $(LOG)/ZF-ex.gz

$(LOG)/ZF-ex.gz: $(OUT)/ZF ex/ROOT.ML \
  ex/BinEx.thy ex/CoUnit.thy ex/Commutation.thy \
  ex/Limit.thy ex/LList.thy ex/Primes.thy \
  ex/NatSum.thy ex/Ramsey.thy ex/misc.thy
	@$(ISATOOL) usedir $(OUT)/ZF ex


## clean

clean:
	@rm -f $(OUT)/ZF $(LOG)/ZF.gz $(LOG)/ZF-AC.gz $(LOG)/ZF-Coind.gz \
	  $(LOG)/ZF-ex.gz $(LOG)/ZF-IMP.gz $(LOG)/ZF-Resid.gz \
	  $(LOG)/ZF-UNITY.gz