src/HOL/List.thy
changeset 29927 ae8f42c245b2
parent 29856 984191be0357
child 30008 20c194b71bb7
child 30240 5b25fee0362c
equal deleted inserted replaced
29926:7dac794eec91 29927:ae8f42c245b2
   255 @{lemma "listsum [1,2,3::nat] = 6" by simp}
   255 @{lemma "listsum [1,2,3::nat] = 6" by simp}
   256 \end{tabular}}
   256 \end{tabular}}
   257 \caption{Characteristic examples}
   257 \caption{Characteristic examples}
   258 \label{fig:Characteristic}
   258 \label{fig:Characteristic}
   259 \end{figure}
   259 \end{figure}
   260 Figure~\ref{fig:Characteristic} shows charachteristic examples
   260 Figure~\ref{fig:Characteristic} shows characteristic examples
   261 that should give an intuitive understanding of the above functions.
   261 that should give an intuitive understanding of the above functions.
   262 *}
   262 *}
   263 
   263 
   264 text{* The following simple sort functions are intended for proofs,
   264 text{* The following simple sort functions are intended for proofs,
   265 not for efficient implementations. *}
   265 not for efficient implementations. *}