Binary file coursework/cw01.pdf has changed
Binary file coursework/cw02.pdf has changed
Binary file coursework/cw03.pdf has changed
Binary file coursework/cw04.pdf has changed
Binary file coursework/cw05.pdf has changed
--- a/coursework/cw05.tex Wed Dec 03 00:23:54 2014 +0000
+++ b/coursework/cw05.tex Fri Dec 05 01:00:34 2014 +0000
@@ -214,7 +214,7 @@
by (simp (no_asm) add: Star_def) blast
qed
\end{lstlisting}
-\caption{An Isabelle proof about the function \pcode{zeroable}.\label{proof}}
+\caption{An Isabelle proof about the function \texttt{zeroable}.\label{proof}}
\end{figure}
\end{document}
Binary file handouts/ho01.pdf has changed
Binary file handouts/ho02.pdf has changed
Binary file handouts/ho03.pdf has changed
Binary file handouts/ho04.pdf has changed
Binary file handouts/ho05.pdf has changed
Binary file handouts/ho06.pdf has changed
Binary file handouts/notation.pdf has changed
Binary file handouts/scala-ho.pdf has changed
Binary file hws/hw01.pdf has changed
Binary file hws/hw02.pdf has changed
Binary file hws/hw03.pdf has changed
Binary file hws/hw04.pdf has changed
Binary file hws/hw05.pdf has changed
Binary file hws/hw06.pdf has changed
Binary file hws/hw07.pdf has changed
Binary file hws/hw08.pdf has changed
Binary file hws/hw09.pdf has changed
Binary file hws/proof.pdf has changed
--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/mk Fri Dec 05 01:00:34 2014 +0000
@@ -0,0 +1,11 @@
+#!/bin/sh
+
+subdirs="slides hws slides coursework handouts"
+
+for sd in $subdirs; do
+ cd $sd
+ for fl in *.tex; do
+ xelatex $fl
+ done
+ cd ..
+done
\ No newline at end of file
Binary file slides/slides01.pdf has changed
Binary file slides/slides02.pdf has changed
Binary file slides/slides03.pdf has changed
Binary file slides/slides04.pdf has changed
Binary file slides/slides05.pdf has changed
Binary file slides/slides06.pdf has changed
Binary file slides/slides07.pdf has changed
Binary file slides/slides08.pdf has changed
Binary file slides/slides09.pdf has changed
Binary file slides/slides10.pdf has changed