src/HOLCF/IsaMakefile
author wenzelm
Sun, 29 Nov 1998 13:16:47 +0100
changeset 5989 9670dae0143d
parent 4566 23c01c724d7a
child 6010 fc58d3c1fd62
permissions -rw-r--r--
proof_general_trans (experimental);

#
# $Id$
#
# IsaMakefile for HOLCF
#

## targets

default: HOLCF
images: HOLCF IOA
test: HOLCF-IMP HOLCF-ex IOA-ABP IOA-NTP
all: images test


## global settings

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


## HOLCF

HOLCF: HOL $(OUT)/HOLCF

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

$(OUT)/HOLCF: $(OUT)/HOL Cfun1.ML Cfun1.thy Cfun2.ML Cfun2.thy \
  Cfun3.ML Cfun3.thy Cont.ML Cont.thy Cprod1.ML Cprod1.thy Cprod2.ML \
  Cprod2.thy Cprod3.ML Cprod3.thy Discrete.ML Discrete.thy Discrete0.ML \
  Discrete0.thy Discrete1.ML Discrete1.thy Fix.ML Fix.thy Fun1.ML \
  Fun1.thy Fun2.ML Fun2.thy Fun3.ML Fun3.thy HOLCF.ML HOLCF.thy Lift.ML \
  Lift.thy Lift1.ML Lift1.thy Lift2.ML Lift2.thy Lift3.ML Lift3.thy \
  One.ML One.thy Pcpo.ML Pcpo.thy Porder.ML Porder.thy Porder0.ML \
  Porder0.thy ROOT.ML Sprod0.ML Sprod0.thy Sprod1.ML Sprod1.thy \
  Sprod2.ML Sprod2.thy Sprod3.ML Sprod3.thy Ssum0.ML Ssum0.thy Ssum1.ML \
  Ssum1.thy Ssum2.ML Ssum2.thy Ssum3.ML Ssum3.thy Tr.ML Tr.thy Up1.ML \
  Up1.thy Up2.ML Up2.thy Up3.ML Up3.thy adm.ML cont_consts.ML \
  domain/axioms.ML domain/extender.ML domain/interface.ML \
  domain/library.ML domain/syntax.ML domain/theorems.ML holcf_logic.ML
	@$(ISATOOL) usedir -b $(OUT)/HOL HOLCF


## HOLCF-IMP

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

$(LOG)/HOLCF-IMP.gz: $(OUT)/HOLCF IMP/Denotational.ML \
  IMP/Denotational.thy IMP/ROOT.ML
	@$(ISATOOL) usedir $(OUT)/HOLCF IMP


## HOLCF-ex

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

$(LOG)/HOLCF-ex.gz: $(OUT)/HOLCF ex/Dagstuhl.ML ex/Dagstuhl.thy \
  ex/Dnat.ML ex/Dnat.thy ex/Fix2.ML ex/Fix2.thy ex/Focus_ex.ML \
  ex/Focus_ex.thy ex/Hoare.ML ex/Hoare.thy ex/Loop.ML ex/Loop.thy \
  ex/ROOT.ML ex/Stream.ML ex/Stream.thy ex/loeckx.ML
	@$(ISATOOL) usedir $(OUT)/HOLCF ex


## IOA

IOA: HOLCF $(OUT)/IOA

$(OUT)/IOA: $(OUT)/HOLCF IOA/ROOT.ML IOA/meta_theory/Traces.thy \
  IOA/meta_theory/Asig.ML IOA/meta_theory/Asig.thy \
  IOA/meta_theory/CompoScheds.thy IOA/meta_theory/CompoExecs.ML \
  IOA/meta_theory/CompoTraces.thy IOA/meta_theory/CompoScheds.ML \
  IOA/meta_theory/CompoTraces.ML IOA/meta_theory/Sequence.ML \
  IOA/meta_theory/Seq.thy IOA/meta_theory/RefCorrectness.thy \
  IOA/meta_theory/Automata.thy IOA/meta_theory/Traces.ML \
  IOA/meta_theory/Seq.ML IOA/meta_theory/RefMappings.ML \
  IOA/meta_theory/ShortExecutions.thy IOA/meta_theory/ShortExecutions.ML \
  IOA/meta_theory/IOA.thy IOA/meta_theory/IOA.ML \
  IOA/meta_theory/Sequence.thy IOA/meta_theory/Automata.ML \
  IOA/meta_theory/CompoExecs.thy IOA/meta_theory/RefMappings.thy \
  IOA/meta_theory/RefCorrectness.ML IOA/meta_theory/Compositionality.ML \
  IOA/meta_theory/Compositionality.thy \
  IOA/meta_theory/TL.thy IOA/meta_theory/TL.ML IOA/meta_theory/TLS.thy \
  IOA/meta_theory/TLS.ML IOA/meta_theory/LiveIOA.thy IOA/meta_theory/LiveIOA.ML \
  IOA/meta_theory/Pred.thy IOA/meta_theory/Abstraction.thy \
  IOA/meta_theory/Abstraction.ML IOA/meta_theory/TrivEx.thy IOA/meta_theory/TrivEx.ML \
  IOA/meta_theory/TrivEx2.thy IOA/meta_theory/TrivEx2.ML \
  IOA/meta_theory/Simulations.thy IOA/meta_theory/Simulations.ML \
  IOA/meta_theory/SimCorrectness.thy IOA/meta_theory/SimCorrectness.ML 
	@cd IOA; $(ISATOOL) usedir -b $(OUT)/HOLCF IOA


## IOA-ABP

IOA-ABP: IOA $(LOG)/IOA-ABP.gz

$(LOG)/IOA-ABP.gz: $(OUT)/IOA IOA/ABP/Abschannel.thy \
  IOA/ABP/Abschannel_finite.thy IOA/ABP/Action.ML IOA/ABP/Action.thy \
  IOA/ABP/Check.ML IOA/ABP/Correctness.ML IOA/ABP/Correctness.thy \
  IOA/ABP/Env.thy IOA/ABP/Impl.thy IOA/ABP/Impl_finite.thy \
  IOA/ABP/Lemmas.ML IOA/ABP/Lemmas.thy IOA/ABP/Packet.thy \
  IOA/ABP/ROOT.ML IOA/ABP/Receiver.thy IOA/ABP/Sender.thy \
  IOA/ABP/Spec.thy
	@cd IOA; $(ISATOOL) usedir $(OUT)/IOA ABP


## IOA-NTP

IOA-NTP: IOA $(LOG)/IOA-NTP.gz

$(LOG)/IOA-NTP.gz: $(OUT)/IOA IOA/NTP/Abschannel.ML \
  IOA/NTP/Abschannel.thy IOA/NTP/Action.ML IOA/NTP/Action.thy \
  IOA/NTP/Correctness.ML IOA/NTP/Correctness.thy IOA/NTP/Impl.ML \
  IOA/NTP/Impl.thy IOA/NTP/Lemmas.ML IOA/NTP/Lemmas.thy \
  IOA/NTP/Multiset.ML IOA/NTP/Multiset.thy IOA/NTP/Packet.ML \
  IOA/NTP/Packet.thy IOA/NTP/ROOT.ML IOA/NTP/Receiver.ML \
  IOA/NTP/Receiver.thy IOA/NTP/Sender.ML IOA/NTP/Sender.thy \
  IOA/NTP/Spec.thy
	@cd IOA; $(ISATOOL) usedir $(OUT)/IOA NTP


## clean

clean:
	@rm -f $(OUT)/HOLCF $(LOG)/HOLCF.gz $(LOG)/HOLCF-IMP.gz \
	  $(LOG)/HOLCF-ex.gz $(OUT)/IOA $(LOG)/IOA.gz $(LOG)/IOA-ABP.gz \
	  $(LOG)/IOA-NTP.gz