--- a/CookBook/document/cookbook.bib Thu Oct 02 05:18:49 2008 -0400
+++ /dev/null Thu Jan 01 00:00:00 1970 +0000
@@ -1,21 +0,0 @@
-
-@manual{isa-imp,
- author = {Makarius Wenzel},
- title = {The {Isabelle/Isar} Implementation},
- institution = {Technische Universit\"at M\"unchen},
- note = {\url{http://isabelle.in.tum.de/doc/implementation.pdf}}}
-
-
-@Book{isa-tutorial,
- author = {Tobias Nipkow and Lawrence C. Paulson and Markus Wenzel},
- title = {Isabelle/HOL: A Proof Assistant for Higher-Order Logic},
- publisher = {Springer},
- year = 2002,
- note = {LNCS Tutorial 2283}}
-
-@book{paulson-ml2,
- author = {Lawrence C. Paulson},
- title = {{ML} for the Working Programmer},
- year = 1996,
- edition = {2nd},
- publisher = {Cambridge University Press}}
\ No newline at end of file
--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/CookBook/document/root.bib Thu Oct 02 05:28:39 2008 -0400
@@ -0,0 +1,21 @@
+
+@manual{isa-imp,
+ author = {Makarius Wenzel},
+ title = {The {Isabelle/Isar} Implementation},
+ institution = {Technische Universit\"at M\"unchen},
+ note = {\url{http://isabelle.in.tum.de/doc/implementation.pdf}}}
+
+
+@Book{isa-tutorial,
+ author = {Tobias Nipkow and Lawrence C. Paulson and Markus Wenzel},
+ title = {Isabelle/HOL: A Proof Assistant for Higher-Order Logic},
+ publisher = {Springer},
+ year = 2002,
+ note = {LNCS Tutorial 2283}}
+
+@book{paulson-ml2,
+ author = {Lawrence C. Paulson},
+ title = {{ML} for the Working Programmer},
+ year = 1996,
+ edition = {2nd},
+ publisher = {Cambridge University Press}}
\ No newline at end of file
--- a/CookBook/document/root.tex Thu Oct 02 05:18:49 2008 -0400
+++ b/CookBook/document/root.tex Thu Oct 02 05:28:39 2008 -0400
@@ -54,7 +54,7 @@
\newpage
\bibliographystyle{abbrv}
-\bibliography{cookbook}
+\bibliography{root}
\end{document}
--- a/IsaMakefile Thu Oct 02 05:18:49 2008 -0400
+++ b/IsaMakefile Thu Oct 02 05:28:39 2008 -0400
@@ -23,7 +23,7 @@
CookBook/document/cookbook.bib \
CookBook/*.thy
$(USEDIR) HOL CookBook
- $(ISATOOL) document -o pdf CookBook/generated
+ $(ISATOOL) document CookBook/generated
@cp CookBook/document.pdf cookbook.pdf
## clean
Binary file cookbook.pdf has changed