coursework/cw05.tex
changeset 317 a61b50c5d57f
parent 298 bdf84605b6cd
child 328 bc03ff3d347c
equal deleted inserted replaced
316:76678ad5079d 317:a61b50c5d57f
   212   have "$\neg$ zeroable (STAR r)" "[] $\in$ L (r) ^ 0" by simp_all
   212   have "$\neg$ zeroable (STAR r)" "[] $\in$ L (r) ^ 0" by simp_all
   213   then show "zeroable (STAR r) $\longleftrightarrow$ (L (STAR r) = {})" 
   213   then show "zeroable (STAR r) $\longleftrightarrow$ (L (STAR r) = {})" 
   214     by (simp (no_asm) add: Star_def) blast
   214     by (simp (no_asm) add: Star_def) blast
   215 qed
   215 qed
   216 \end{lstlisting}
   216 \end{lstlisting}
   217 \caption{An Isabelle proof about the function \pcode{zeroable}.\label{proof}}
   217 \caption{An Isabelle proof about the function \texttt{zeroable}.\label{proof}}
   218 \end{figure}
   218 \end{figure}
   219 
   219 
   220 \end{document}
   220 \end{document}
   221 
   221 
   222 %%% Local Variables: 
   222 %%% Local Variables: