removed onsolete pure.thy (cf. Misc.thy);
--- a/doc-src/IsarRef/IsaMakefile Mon Jun 02 23:12:23 2008 +0200
+++ b/doc-src/IsarRef/IsaMakefile Mon Jun 02 23:38:22 2008 +0200
@@ -23,7 +23,7 @@
$(LOG)/HOL-IsarRef.gz: Thy/ROOT.ML ../antiquote_setup.ML \
Thy/Introduction.thy Thy/Outer_Syntax.thy Thy/Spec.thy Thy/Proof.thy \
- Thy/pure.thy Thy/Document_Preparation.thy Thy/Generic.thy \
+ Thy/Misc.thy Thy/Document_Preparation.thy Thy/Generic.thy \
Thy/HOL_Specific.thy Thy/Quick_Reference.thy Thy/ML_Tactic.thy
@$(USEDIR) -s IsarRef HOL Thy
--- a/doc-src/IsarRef/Makefile Mon Jun 02 23:12:23 2008 +0200
+++ b/doc-src/IsarRef/Makefile Mon Jun 02 23:38:22 2008 +0200
@@ -13,12 +13,12 @@
NAME = isar-ref
-FILES = isar-ref.tex style.sty basics.tex Thy/document/Generic.tex \
+FILES = isar-ref.tex style.sty Thy/document/Generic.tex \
Thy/document/HOLCF_Specific.tex Thy/document/HOL_Specific.tex \
Thy/document/ML_Tactic.tex Thy/document/Proof.tex \
Thy/document/Quick_Reference.tex Thy/document/Spec.tex \
Thy/document/ZF_Specific.tex Thy/document/Introduction.tex \
- Thy/document/Document_Preparation.tex Thy/document/pure.tex \
+ Thy/document/Document_Preparation.tex Thy/document/Misc.tex \
Thy/document/Outer_Syntax.tex ../isar.sty ../rail.sty \
../railsetup.sty ../proof.sty ../iman.sty ../extra.sty ../ttbox.sty \
../isabelle.sty ../isabellesym.sty ../pdfsetup.sty ../manual.bib
--- a/doc-src/IsarRef/Thy/ROOT.ML Mon Jun 02 23:12:23 2008 +0200
+++ b/doc-src/IsarRef/Thy/ROOT.ML Mon Jun 02 23:38:22 2008 +0200
@@ -9,7 +9,7 @@
use_thy "Spec";
use_thy "Proof";
use_thy "Document_Preparation";
-use_thy "pure";
+use_thy "Misc";
use_thy "Generic";
use_thy "HOL_Specific";
use_thy "Quick_Reference";
--- a/doc-src/IsarRef/isar-ref.tex Mon Jun 02 23:12:23 2008 +0200
+++ b/doc-src/IsarRef/isar-ref.tex Mon Jun 02 23:38:22 2008 +0200
@@ -78,8 +78,8 @@
\input{Thy/document/Outer_Syntax.tex}
\input{Thy/document/Spec.tex}
\input{Thy/document/Proof.tex}
-\input{Thy/document/pure.tex}
\input{Thy/document/Document_Preparation.tex}
+\input{Thy/document/Misc.tex}
\input{Thy/document/Generic.tex}
\input{Thy/document/HOL_Specific.tex}
\input{Thy/document/HOLCF_Specific.tex}