fixed creation of bibliography
authorChristian Urban <urbanc@in.tum.de>
Thu, 02 Oct 2008 05:28:39 -0400
changeset 17 8afa1c990a14
parent 16 5045dec52d2b
child 18 b4c31af6af26
fixed creation of bibliography
CookBook/document/cookbook.bib
CookBook/document/root.bib
CookBook/document/root.tex
IsaMakefile
cookbook.pdf
--- 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