build image for session HOL-Library; introduced distinct session HOL-Codegenerator_Test
authorhaftmann
Fri, 02 Jul 2010 14:23:16 +0200
changeset 37691 4915de09b4d3
parent 37681 6ec40bc934e1
child 37692 7b072f0c8bde
build image for session HOL-Library; introduced distinct session HOL-Codegenerator_Test
src/HOL/IsaMakefile
--- a/src/HOL/IsaMakefile	Fri Jul 02 10:47:50 2010 +0200
+++ b/src/HOL/IsaMakefile	Fri Jul 02 14:23:16 2010 +0200
@@ -10,27 +10,28 @@
 
 images: \
   HOL \
+  HOL-Library \
   HOL-Algebra \
-  HOL-Base \
   HOL-Boogie \
-  HOL-Main \
   HOL-Multivariate_Analysis \
   HOL-NSA \
   HOL-Nominal \
-  HOL-Plain \
   HOL-Probability \
   HOL-Proofs \
   HOL-Word \
   HOL4 \
-  TLA
+  TLA \
+  HOL-Base \
+  HOL-Main \
+  HOL-Plain
 
-#Note: keep targets sorted (except for HOL-Library and HOL-ex)
+#Note: keep targets sorted (except for HOL-ex)
 test: \
-  HOL-Library \
   HOL-ex \
   HOL-Auth \
   HOL-Bali \
   HOL-Boogie-Examples \
+  HOL-Codegenerator_Test \
   HOL-Decision_Procs \
   HOL-Hahn_Banach \
   HOL-Hoare \
@@ -392,10 +393,11 @@
 
 ## HOL-Library
 
-HOL-Library: HOL $(LOG)/HOL-Library.gz
+HOL-Library: HOL $(OUT)/HOL-Library
 
-$(LOG)/HOL-Library.gz: $(OUT)/HOL $(SRC)/HOL/Tools/float_arith.ML	\
-  $(SRC)/Tools/float.ML Library/Abstract_Rat.thy Library/AssocList.thy	\
+$(OUT)/HOL-Library: $(OUT)/HOL library.ML				\
+  $(SRC)/HOL/Tools/float_arith.ML $(SRC)/Tools/float.ML			\
+  Library/Abstract_Rat.thy Library/AssocList.thy			\
   Library/BigO.thy Library/Binomial.thy Library/Bit.thy			\
   Library/Boolean_Algebra.thy Library/Cardinality.thy			\
   Library/Char_nat.thy Library/Code_Char.thy Library/Code_Char_chr.thy	\
@@ -408,7 +410,7 @@
   Library/FuncSet.thy Library/Fundamental_Theorem_Algebra.thy		\
   Library/Glbs.thy Library/Indicator_Function.thy			\
   Library/Infinite_Set.thy Library/Inner_Product.thy			\
-  Library/HOL_Library_ROOT.ML Library/Kleene_Algebra.thy		\
+  Library/Kleene_Algebra.thy						\
   Library/LaTeXsugar.thy Library/Lattice_Algebras.thy			\
   Library/Lattice_Syntax.thy Library/Library.thy			\
   Library/List_Prefix.thy Library/List_lexord.thy Library/Mapping.thy	\
@@ -432,10 +434,10 @@
   Library/Sum_Of_Squares/sum_of_squares.ML				\
   Library/Transitive_Closure_Table.thy Library/Univ_Poly.thy		\
   Library/While_Combinator.thy Library/Zorn.thy				\
-  Library/document/root.bib Library/document/root.tex			\
   Library/positivstellensatz.ML Library/reflection.ML			\
-  Library/reify_data.ML
-	@$(ISABELLE_TOOL) usedir -f HOL_Library_ROOT.ML $(OUT)/HOL Library
+  Library/reify_data.ML							\
+  Library/document/root.bib Library/document/root.tex
+	@$(ISABELLE_TOOL) usedir -b -f library.ML $(OUT)/HOL HOL-Library
 
 
 ## HOL-Hahn_Banach
@@ -632,6 +634,18 @@
 	@$(ISABELLE_TOOL) usedir -g true $(OUT)/HOL Hoare_Parallel
 
 
+## HOL-Codegenerator_Test
+
+HOL-Codegenerator_Test: HOL-Library $(LOG)/HOL-Codegenerator_Test.gz
+
+$(LOG)/HOL-Codegenerator_Test.gz: $(OUT)/HOL-Library			\
+  Codegenerator_Test/ROOT.ML Codegenerator_Test/Candidates.thy		\
+  Codegenerator_Test/Candidates_Pretty.thy				\
+  Codegenerator_Test/Generate.thy					\
+  Codegenerator_Test/Generate_Pretty.thy
+	@$(ISABELLE_TOOL) usedir -d false -g false -i false $(OUT)/HOL-Library Codegenerator_Test
+
+
 ## HOL-Metis_Examples
 
 HOL-Metis_Examples: HOL $(LOG)/HOL-Metis_Examples.gz
@@ -976,9 +990,7 @@
   ex/Abstract_NAT.thy ex/Antiquote.thy ex/Arith_Examples.thy		\
   ex/Arithmetic_Series_Complex.thy ex/BT.thy ex/BinEx.thy		\
   ex/Binary.thy ex/CTL.thy ex/Chinese.thy ex/Classical.thy		\
-  ex/CodegenSML_Test.thy ex/Codegenerator_Candidates.thy		\
-  ex/Codegenerator_Pretty.thy ex/Codegenerator_Pretty_Test.thy		\
-  ex/Codegenerator_Test.thy ex/Coherent.thy ex/Dedekind_Real.thy	\
+  ex/CodegenSML_Test.thy ex/Coherent.thy ex/Dedekind_Real.thy		\
   ex/Efficient_Nat_examples.thy ex/Eval_Examples.thy ex/Fundefs.thy	\
   ex/Gauge_Integration.thy ex/Groebner_Examples.thy ex/Guess.thy	\
   ex/HarmonicSeries.thy ex/Hebrew.thy ex/Hex_Bin_Examples.thy		\