doc-src/IsarImplementation/IsaMakefile
changeset 39846 cb6634eb8926
parent 39822 0de42180febe
child 39884 a16b18fd6299
--- a/doc-src/IsarImplementation/IsaMakefile	Wed Oct 13 11:15:15 2010 +0100
+++ b/doc-src/IsarImplementation/IsaMakefile	Wed Oct 13 13:05:23 2010 +0100
@@ -19,13 +19,13 @@
 
 ## sessions
 
-Thy: $(LOG)/Pure-Thy.gz
+Thy: $(LOG)/HOL-Thy.gz
 
-$(LOG)/Pure-Thy.gz: Thy/ROOT.ML Thy/Base.thy Thy/Integration.thy	\
+$(LOG)/HOL-Thy.gz: Thy/ROOT.ML Thy/Base.thy Thy/Integration.thy	\
   Thy/Isar.thy Thy/Local_Theory.thy Thy/Logic.thy Thy/Prelim.thy	\
   Thy/Proof.thy Thy/Syntax.thy Thy/Tactic.thy Thy/ML.thy		\
   Thy/ML_old.thy ../antiquote_setup.ML
-	@$(USEDIR) Pure Thy
+	@$(USEDIR) HOL Thy
 	@rm -f Thy/document/isabelle.sty Thy/document/isabellesym.sty \
 	 Thy/document/pdfsetup.sty Thy/document/session.tex
 
@@ -33,4 +33,4 @@
 ## clean
 
 clean:
-	@rm -f $(LOG)/Pure-Thy.gz
+	@rm -f $(LOG)/HOL-Thy.gz