src/Doc/Prog_Prove/Isar.thy
changeset 67299 ba52a058942f
parent 67039 690b4b334889
child 67406 23307fd33906
equal deleted inserted replaced
67298:fee3ed06a281 67299:ba52a058942f
   503 and after the second \isakeyword{also}, \<open>calculation\<close> is \<open>"t\<^sub>1 < t\<^sub>3"\<close>.
   503 and after the second \isakeyword{also}, \<open>calculation\<close> is \<open>"t\<^sub>1 < t\<^sub>3"\<close>.
   504 The command \isakeyword{finally} is short for \isakeyword{also from} \<open>calculation\<close>.
   504 The command \isakeyword{finally} is short for \isakeyword{also from} \<open>calculation\<close>.
   505 Therefore the \isakeyword{also} hidden in \isakeyword{finally} sets \<open>calculation\<close>
   505 Therefore the \isakeyword{also} hidden in \isakeyword{finally} sets \<open>calculation\<close>
   506 to \<open>t\<^sub>1 < t\<^sub>4\<close> and the final ``\texttt{.}'' succeeds.
   506 to \<open>t\<^sub>1 < t\<^sub>4\<close> and the final ``\texttt{.}'' succeeds.
   507 
   507 
   508 For more information on this style of proof see \cite{BauerW-TPHOLs01}.
   508 For more information on this style of proof see @{cite "BauerW-TPHOLs01"}.
   509 \fi
   509 \fi
   510 
   510 
   511 \section{Streamlining Proofs}
   511 \section{Streamlining Proofs}
   512 
   512 
   513 \subsection{Pattern Matching and Quotations}
   513 \subsection{Pattern Matching and Quotations}