src/HOL/IsaMakefile
changeset 3125 3f0ab2c306f7
parent 3118 24dae6222579
child 3195 dcb458d38724
--- a/src/HOL/IsaMakefile	Wed May 07 13:50:52 1997 +0200
+++ b/src/HOL/IsaMakefile	Wed May 07 13:51:22 1997 +0200
@@ -41,6 +41,17 @@
 
 #### Tests and examples
 
+## Inductive definitions: simple examples
+
+INDUCT_FILES =  Perm Comb Mutil SList LList LFilter Acc PropLog Term Simult
+
+INDUCT_FILES = Induct/ROOT.ML \
+	    $(INDUCT_NAMES:%=Induct/%.thy) $(INDUCT_NAMES:%=Induct/%.ML)
+
+Induct:	$(OUT)/HOL $(INDUCT_FILES)
+	@$(ISATOOL) usedir $(OUT)/HOL Induct
+
+
 ## IMP-semantics example
 
 IMP_NAMES = Expr Com Natural Transition Denotation Hoare VC
@@ -185,8 +196,7 @@
 
 ## Miscellaneous examples
 
-EX_NAMES = String BT Perm Comb InSort Qsort LexProd Puzzle Mutil \
-	   Primes NatSum SList LList LFilter Acc PropLog Term Simult MT
+EX_NAMES = String BT InSort Qsort LexProd Puzzle Primes NatSum MT
 
 EX_FILES = ex/ROOT.ML ex/cla.ML ex/meson.ML ex/mesontest.ML ex/rel.ML \
 	   ex/set.ML $(EX_NAMES:%=ex/%.thy) $(EX_NAMES:%=ex/%.ML)
@@ -198,7 +208,8 @@
 ## Full test
 
 test:	$(OUT)/HOL \
-	TFL IMP Hoare Lex Integ Auth Subst Lambda W0 MiniML IOA AxClasses Quot ex
+		TFL Induct IMP Hoare Lex Integ Auth Subst Lambda  \
+		W0 MiniML IOA AxClasses Quot ex
 	echo 'Test examples ran successfully' > test