src/HOL/IsaMakefile
author oheimb
Wed, 12 Nov 1997 18:58:50 +0100
changeset 4223 f60e3d2c81d3
parent 4081 f759352f669f
child 4263 a434327aef8b
permissions -rw-r--r--
added thin_refl to hyp_subst_tac

#
# $Id$
#
# IsaMakefile for HOL
#

#### Base system

OUT = $(ISABELLE_OUTPUT)

NAMES = HOL Ord Set Fun subset equalities Prod Relation Trancl Sum WF WF_Rel \
	mono Lfp Gfp NatDef Nat intr_elim indrule Inductive Finite Arith \
	Divides Power Sexp Univ List RelPow Option Map

PROVERS = hypsubst.ML classical.ML blast.ML \
	simplifier.ML splitter.ML nat_transitive.ML 

TFL   = dcterm.sml post.sml rules.new.sml rules.sig \
	sys.sml tfl.sig tfl.sml thms.sig thms.sml thry.sig thry.sml   \
	usyntax.sig usyntax.sml utils.sig utils.sml

FILES = ROOT.ML add_ind_def.ML datatype.ML hologic.ML \
	ind_syntax.ML cladata.ML simpdata.ML \
	typedef.ML thy_syntax.ML thy_data.ML ../Pure/section_utils.ML \
	$(NAMES:%=%.thy) $(NAMES:%=%.ML) $(TFL:%=../TFL/%) \
	$(PROVERS:%=../Provers/%)

$(OUT)/HOL: $(OUT)/Pure $(FILES)
	@$(ISATOOL) usedir -b $(OUT)/Pure HOL

$(OUT)/Pure:
	@cd ../Pure; $(ISATOOL) make


#### 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
IMP_FILES = IMP/ROOT.ML $(IMP_NAMES:%=IMP/%.thy) $(IMP_NAMES:%=IMP/%.ML)

IMP:	$(OUT)/HOL $(IMP_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL IMP


## Hoare logic

Hoare_NAMES = Hoare Arith2 Examples
Hoare_FILES = Hoare/ROOT.ML $(Hoare_NAMES:%=Hoare/%.thy) \
	      $(Hoare_NAMES:%=Hoare/%.ML)

Hoare:	$(OUT)/HOL $(Hoare_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL Hoare


## The integers in HOL

INTEG_NAMES = Equiv Integ Group Ring Lagrange IntRingDefs IntRing

INTEG_FILES = Integ/ROOT.ML \
	      $(INTEG_NAMES:%=Integ/%.thy) $(INTEG_NAMES:%=Integ/%.ML)

Integ:	$(OUT)/HOL $(INTEG_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL Integ


## TLA -- Temporal Logic of Actions

TLA_FILES = TLA/Action.ML TLA/Action.thy TLA/IntLemmas.ML \
	TLA/Intensional.ML TLA/Intensional.thy TLA/ROOT.ML TLA/Stfun.ML \
	TLA/Stfun.thy TLA/TLA.ML TLA/TLA.thy TLA/cladata.ML TLA/hypsubst.ML

TLA_INC_FILES = TLA/Inc/Inc.thy TLA/Inc/Inc.ML TLA/Inc/Pcount.thy

TLA_BUFFER_FILES = TLA/Buffer/Buffer.thy TLA/Buffer/Buffer.ML \
	TLA/Buffer/DBuffer.thy TLA/Buffer/DBuffer.ML

TLA_MEMORY_FILES = TLA/Memory/MIParameters.thy TLA/Memory/MIlive.ML \
	TLA/Memory/MIsafe.ML TLA/Memory/MemClerk.ML TLA/Memory/MemClerk.thy \
	TLA/Memory/MemClerkParameters.ML TLA/Memory/MemClerkParameters.thy \
	TLA/Memory/Memory.ML TLA/Memory/Memory.thy \
	TLA/Memory/MemoryImplementation.ML TLA/Memory/MemoryImplementation.thy \
	TLA/Memory/MemoryParameters.ML TLA/Memory/MemoryParameters.thy \
	TLA/Memory/ProcedureInterface.ML TLA/Memory/ProcedureInterface.thy \
	TLA/Memory/RPC.ML TLA/Memory/RPC.thy TLA/Memory/RPCMemoryParams.thy \
	TLA/Memory/RPCParameters.ML TLA/Memory/RPCParameters.thy


TLA: $(OUT)/HOL $(TLA_FILES)
	@cd TLA; $(ISATOOL) usedir -b $(OUT)/HOL TLA

TLA_Inc: $(OUT)/TLA $(TLA_INC_FILES)
	@cd TLA; $(ISATOOL) usedir $(OUT)/TLA Inc

TLA_Buffer: $(OUT)/TLA $(TLA_BUFFER_FILES)
	@cd TLA; $(ISATOOL) usedir $(OUT)/TLA Buffer

TLA_Memory: $(OUT)/TLA $(TLA_MEMORY_FILES)
	@cd TLA; $(ISATOOL) usedir $(OUT)/TLA Memory


## I/O Automata (meta theory only)

IOA_FILES = IOA/ROOT.ML IOA/Asig.thy IOA/Asig.ML IOA/IOA.thy \
  IOA/IOA.ML IOA/Solve.thy IOA/Solve.ML

IOA: $(OUT)/HOL $(IOA_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL IOA


## Authentication & Security Protocols

AUTH_NAMES = Message Event Shared NS_Shared \
	     OtwayRees OtwayRees_AN OtwayRees_Bad \
	     Recur WooLam Yahalom Yahalom2 \
	     Public NS_Public_Bad NS_Public TLS

AUTH_FILES = Auth/ROOT.ML $(AUTH_NAMES:%=Auth/%.thy) $(AUTH_NAMES:%=Auth/%.ML)

Auth:	$(OUT)/HOL $(AUTH_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL Auth


## Modelchecker invocation

MC_FILES = Modelcheck/CTL.thy Modelcheck/Example.ML \
  Modelcheck/Example.thy Modelcheck/MCSyn.ML Modelcheck/MCSyn.thy \
  Modelcheck/MuCalculus.ML Modelcheck/MuCalculus.thy Modelcheck/ROOT.ML

Modelcheck: $(OUT)/HOL $(MC_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL Modelcheck


## Properties of substitutions

SUBST_NAMES = AList Subst Unifier UTerm Unify

SUBST_FILES = Subst/ROOT.ML \
	      $(SUBST_NAMES:%=Subst/%.thy) $(SUBST_NAMES:%=Subst/%.ML)

Subst:	$(OUT)/HOL $(SUBST_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL Subst


## Confluence of Lambda-calculus

LAMBDA_NAMES = Lambda ParRed Commutation Eta

LAMBDA_FILES = Lambda/ROOT.ML \
	      $(LAMBDA_NAMES:%=Lambda/%.thy) $(LAMBDA_NAMES:%=Lambda/%.ML)

Lambda:	 $(OUT)/HOL $(LAMBDA_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL Lambda


## Type inference without let

W0_NAMES = I Maybe MiniML Type W

W0_FILES = W0/ROOT.ML \
	      $(W0_NAMES:%=W0/%.thy) $(W0_NAMES:%=W0/%.ML)

W0: $(OUT)/HOL $(W0_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL W0


## Type inference with let

MINIML_NAMES = Generalize Instance Maybe MiniML Type W

MINIML_FILES = MiniML/ROOT.ML \
	      $(MINIML_NAMES:%=MiniML/%.thy) $(MINIML_NAMES:%=MiniML/%.ML)

MiniML: $(OUT)/HOL $(MINIML_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL MiniML


## Lexical analysis

LEX_FILES = Auto AutoChopper Chopper Prefix

LEX_FILES = Lex/ROOT.ML \
	    $(LEX_NAMES:%=Lex/%.thy) $(LEX_NAMES:%=Lex/%.ML)

Lex:	$(OUT)/HOL $(LEX_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL Lex


## Axiomatic type classes examples

AXC_GROUP_FILES = Group.ML Group.thy GroupDefs.ML GroupDefs.thy \
	GroupInsts.thy Monoid.thy MonoidGroupInsts.thy ROOT.ML Sigs.thy

AXC_LATTICE_FILES = CLattice.ML CLattice.thy LatInsts.ML LatInsts.thy \
	LatMorph.ML LatMorph.thy LatPreInsts.ML LatPreInsts.thy \
	Lattice.ML Lattice.thy OrdDefs.ML OrdDefs.thy OrdInsts.thy \
	Order.ML Order.thy ROOT.ML tools.ML

AXC_TUTORIAL_FILES = BoolGroupInsts.thy Group.ML Group.thy Monoid.thy \
	MonoidGroupInsts.thy ProdGroupInsts.thy Product.thy \
	ProductInsts.thy ROOT.ML Semigroup.thy Semigroups.thy Sigs.thy \
	Xor.ML Xor.thy

AXCLASSES_FILES = AxClasses/ROOT.ML \
	$(AXC_GROUP_FILES:%=AxClasses/Group/%) \
	$(AXC_LATTICE_FILES:%=AxClasses/Lattice/%) \
	$(AXC_TUTORIAL_FILES:%=AxClasses/Tutorial/%)

AxClasses: $(OUT)/HOL $(AXCLASSES_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL AxClasses
	@$(ISATOOL) usedir -s AxClasses-Group $(OUT)/HOL AxClasses/Group
	@$(ISATOOL) usedir -s AxClasses-Lattice $(OUT)/HOL AxClasses/Lattice
	@$(ISATOOL) usedir -s AxClasses-Tutorial $(OUT)/HOL AxClasses/Tutorial


## Higher-order quotients and example fractionals

QUOT_FILES = Quot/ROOT.ML Quot/PER0.thy Quot/PER0.ML Quot/PER.thy Quot/PER.ML \
	Quot/HQUOT.thy Quot/HQUOT.ML Quot/NPAIR.thy Quot/NPAIR.ML \
	Quot/FRACT.thy Quot/FRACT.ML
Quot:	$(OUT)/HOL $(QUOT_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL Quot


## Miscellaneous examples

EX_NAMES = Recdef Fib Primes Primrec NatSum String BT InSort Qsort Puzzle 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)

ex:	$(OUT)/HOL $(EX_FILES)
	@$(ISATOOL) usedir $(OUT)/HOL ex


## Full test

test:	$(OUT)/HOL \
	  Subst Induct IMP Hoare Lex Integ Auth Modelcheck Lambda  \
	  W0 MiniML TLA TLA_Inc TLA_Buffer TLA_Memory IOA AxClasses Quot ex
	echo 'Test examples ran successfully' > test


.PRECIOUS: $(OUT)/Pure $(OUT)/HOL