doc-src/Exercises/exercises.bib
changeset 13739 f5d0a66c8124
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/doc-src/Exercises/exercises.bib	Thu Dec 05 17:12:07 2002 +0100
@@ -0,0 +1,85 @@
+@string{LNCS="Lect.\ Notes in Comp.\ Sci."}
+@string{FAC="Formal Aspects of Computing"}
+
+@Book{Tanenbaum,
+  author = {Andrew S. Tanenbaum},
+  title = {Modern Operating Systems},
+  publisher = {Prentice-Hall},
+  year = 1992
+}
+
+@Misc{Unix-heritage,
+  key = {Unix},
+  title = {The {Unix} Heritage Society},
+  note = {\\ \url{http://www.tuhs.org/}}
+}
+
+@Book{Broy-PartI,
+  author =	 {M. Broy},
+  title = 	 {Informatik --- Eine grundlegende Einf{\"u}hrung
+                  (Teil I)},
+  publisher = 	 {Springer},
+  year = 	 1992
+}
+
+@Book{Huth-Ryan:2000,
+  author = 	 {M. R. A Huth and M. D. Ryan},
+  title = 	 {Logic in Computer Science --- Modelling and
+                  reasoning about systems},
+  publisher = 	 {Cambridge University Press},
+  year = 	 2000,
+  note =	 {\\ \url{http://www.cs.bham.ac.uk/research/lics/}}
+}
+
+@Misc{Wenzel:2000:Hoare,
+  author =	 {Markus Wenzel},
+  title =	 {A formulation of {H}oare {L}ogic in {I}sabelle/{I}sar},
+  month =	 {June},
+  year =	 2000,
+  note =	 {\\ \url{http://www4.in.tum.de/~wenzelm/papers/Hoare-Isar.pdf}}
+}
+
+@Misc{Naraschewski-Wenzel:1998:HOOL,
+author={Wolfgang Naraschewski and Markus Wenzel},
+title=
+{Object-Oriented Verification based on Record Subtyping in Higher-Order Logic},
+booktitle={Theorem Proving in Higher Order Logics:
+11th International Conference, TPHOLs'98},
+publisher={Springer},volume=1479,series=LNCS,year=1998
+}
+
+@Misc{Nipkow:1998:Winskel,
+author={Tobias Nipkow},
+title={Winskel is (almost) Right: Towards a Mechanized Semantics Textbook},
+journal=FAC,volume=10,pages={171--186},year=1998}
+}
+
+@Book{Winskel:1993,
+  author = 	 {G. Winskel},
+  title = 	 {The Formal Semantics of Programming Languages},
+  publisher = 	 {MIT Press},
+  year = 	 1993
+} 
+
+
+@manual{isabelle-isar-ref,
+  author	= {Markus Wenzel},
+  title		= {The {Isabelle/Isar} Reference Manual},
+  institution	= {TU M{\"u}nchen},
+  year          = 2000,
+  note          = {\\ \url{http://isabelle.in.tum.de/doc/}}}
+
+@manual{isabelle-tutorial,
+  author        = {Tobias Nipkow and Lawrence C. Paulson and Markus Wenzel},
+  title         = {Isabelle/HOL --- A Proof Assistant for Higher-Order Logic},
+  publisher     = {Springer},
+  series        = {LNCS},
+  volume        = 2283,
+  year          = 2002,
+  note          = {\\ \url{http://www4.in.tum.de/~nipkow/LNCS2283/}}}
+
+@Misc{McMillan-LectureNotes,
+  author =	 {Ken McMillan},
+  title =	 {Lecture notes for {NATO} summer school on verification of digital and hybrid systems},
+  note =	 {\\ \url{http://www-cad.eecs.berkeley.edu/~kenmcmil/tutorial/toc.html}}
+}