diff -r 990c12ab1562 -r ea2e5acbfe4a Paper/Paper.thy --- a/Paper/Paper.thy Wed May 04 07:05:59 2011 +0000 +++ b/Paper/Paper.thy Mon May 09 07:25:37 2011 +0000 @@ -513,7 +513,7 @@ \end{equation} \noindent - The reason for adding the @{text \}-marker to our initial equational system is + holds. The reason for adding the @{text \}-marker to our initial equational system is to obtain this equation: it only holds with the marker, since none of the other terms contain the empty string. The point of the initial equational system is that solving it means we will be able to extract a regular expression for every equivalence class. @@ -721,7 +721,7 @@ \noindent The first two ensure that the equational system is always finite (number of equations - and number of terms in each equation); the second makes sure the `meaning' of the + and number of terms in each equation); the third makes sure the `meaning' of the equations is preserved under our transformations. The other properties are a bit more technical, but are needed to get our proof through. Distinctness states that every equation in the system is distinct. @{text Ardenable} ensures that we can always @@ -875,7 +875,7 @@ text {* We will prove in this section the second part of the Myhill-Nerode - theorem. It can be formulated in our setting as follows. + theorem. It can be formulated in our setting as follows: \begin{theorem} Given @{text "r"} is a regular expression, then @{thm Myhill_Nerode2}.