doc-src/IsarRef/IsaMakefile
changeset 42651 e3fdb7c96be5
parent 41729 ae1a46cdb9cb
child 42915 f35aae36cad0
equal deleted inserted replaced
42650:552eae49f97d 42651:e3fdb7c96be5
    19 
    19 
    20 ## sessions
    20 ## sessions
    21 
    21 
    22 HOL-IsarRef: $(LOG)/HOL-IsarRef.gz
    22 HOL-IsarRef: $(LOG)/HOL-IsarRef.gz
    23 
    23 
    24 $(LOG)/HOL-IsarRef.gz: Thy/ROOT.ML ../antiquote_setup.ML		\
    24 $(LOG)/HOL-IsarRef.gz: Thy/ROOT.ML ../antiquote_setup.ML Thy/Base.thy	\
    25   Thy/First_Order_Logic.thy Thy/Framework.thy Thy/Inner_Syntax.thy	\
    25   Thy/First_Order_Logic.thy Thy/Framework.thy Thy/Inner_Syntax.thy	\
    26   Thy/Introduction.thy Thy/Outer_Syntax.thy Thy/Spec.thy Thy/Proof.thy	\
    26   Thy/Introduction.thy Thy/Outer_Syntax.thy Thy/Spec.thy Thy/Proof.thy	\
    27   Thy/Misc.thy Thy/Document_Preparation.thy Thy/Generic.thy		\
    27   Thy/Misc.thy Thy/Document_Preparation.thy Thy/Generic.thy		\
    28   Thy/HOL_Specific.thy Thy/Quick_Reference.thy Thy/Symbols.thy		\
    28   Thy/HOL_Specific.thy Thy/Quick_Reference.thy Thy/Symbols.thy		\
    29   Thy/ML_Tactic.thy
    29   Thy/ML_Tactic.thy
    33 
    33 
    34 
    34 
    35 HOLCF-IsarRef: $(LOG)/HOLCF-IsarRef.gz
    35 HOLCF-IsarRef: $(LOG)/HOLCF-IsarRef.gz
    36 
    36 
    37 $(LOG)/HOLCF-IsarRef.gz: Thy/ROOT-HOLCF.ML ../antiquote_setup.ML	\
    37 $(LOG)/HOLCF-IsarRef.gz: Thy/ROOT-HOLCF.ML ../antiquote_setup.ML	\
    38   Thy/HOLCF_Specific.thy
    38   Thy/Base.thy Thy/HOLCF_Specific.thy
    39 	@$(USEDIR) -s IsarRef -f ROOT-HOLCF.ML HOLCF Thy
    39 	@$(USEDIR) -s IsarRef -f ROOT-HOLCF.ML HOLCF Thy
    40 	@rm -f Thy/document/isabelle.sty Thy/document/isabellesym.sty \
    40 	@rm -f Thy/document/isabelle.sty Thy/document/isabellesym.sty \
    41 	 Thy/document/pdfsetup.sty Thy/document/session.tex
    41 	 Thy/document/pdfsetup.sty Thy/document/session.tex
    42 
    42 
    43 
    43 
    44 ZF-IsarRef: $(LOG)/ZF-IsarRef.gz
    44 ZF-IsarRef: $(LOG)/ZF-IsarRef.gz
    45 
    45 
    46 $(LOG)/ZF-IsarRef.gz: Thy/ROOT-ZF.ML ../antiquote_setup.ML 		\
    46 $(LOG)/ZF-IsarRef.gz: Thy/ROOT-ZF.ML ../antiquote_setup.ML	\
    47   Thy/ZF_Specific.thy
    47   Thy/Base.thy Thy/ZF_Specific.thy
    48 	@$(USEDIR) -s IsarRef -f ROOT-ZF.ML ZF Thy
    48 	@$(USEDIR) -s IsarRef -f ROOT-ZF.ML ZF Thy
    49 	@rm -f Thy/document/isabelle.sty Thy/document/isabellesym.sty \
    49 	@rm -f Thy/document/isabelle.sty Thy/document/isabellesym.sty \
    50 	 Thy/document/pdfsetup.sty Thy/document/session.tex
    50 	 Thy/document/pdfsetup.sty Thy/document/session.tex
    51 
    51 
    52 
    52