# HG changeset patch # User urbanc # Date 1297236450 0 # Node ID 42af13d194c918a96de36a9163ae310e1a577113 # Parent 1436fc451bb935c3c4f7ad3e4d3d31b050601ff7 a bit more on the paper diff -r 1436fc451bb9 -r 42af13d194c9 Myhill_1.thy --- a/Myhill_1.thy Wed Feb 09 06:09:46 2011 +0000 +++ b/Myhill_1.thy Wed Feb 09 07:27:30 2011 +0000 @@ -353,6 +353,9 @@ section {* Equational systems *} + +text {* The two kinds of terms in the rhs of equations. *} + datatype rhs_item = Lam "rexp" (* Lambda-marker *) | Trn "lang" "rexp" (* Transition *) diff -r 1436fc451bb9 -r 42af13d194c9 Paper/Paper.thy --- a/Paper/Paper.thy Wed Feb 09 06:09:46 2011 +0000 +++ b/Paper/Paper.thy Wed Feb 09 07:27:30 2011 +0000 @@ -24,7 +24,7 @@ UPLUS ("_ \<^raw:\ensuremath{\uplus}> _" [90, 90] 90) and L ("\<^raw:\ensuremath{\cal{L}}>'(_')" [0] 101) and Lam ("\'(_')" [100] 100) and - Trn ("_, _" [100, 100] 100) and + Trn ("'(_, _')" [100, 100] 100) and EClass ("\_\\<^bsub>_\<^esub>" [100, 100] 100) and transition ("_ \<^raw:\ensuremath{\stackrel{\text{>_\<^raw:}}{\Longmapsto}}> _" [100, 100, 100] 100) and Setalt ("\<^raw:\ensuremath{\bigplus}>_" [1000] 999) @@ -433,11 +433,24 @@ the other terms contain the empty string. - Our proof of Thm.~\ref{myhillnerodeone} - will be by transforming the equational system into a \emph{solved form} - maintaining the invariants \eqref{inv1} and \eqref{inv2}. From the solved - form we will be able to read off the regular expressions using our - variant of Arden's Lemma (Lem.~\ref{arden}). + Our proof of Thm.~\ref{myhillnerodeone} will be by transforming the + equational system into a \emph{solved form} maintaining the invariants + \eqref{inv1} and \eqref{inv2}. From the solved form we will be able to read + off the regular expressions. + + In order to transform an equational system into solved form, we have two main + operations: one that takes an equation of the form @{text "X = rhs"} and removes + the recursive occurences of @{text X} in @{text rhs} using our variant of Arden's + Lemma (Lem.~\ref{arden}). The other operation takes an equation @{text "X = rhs"} + and substitutes @{text X} throughout the rest of the equational system + adjusting the regular expressions approriately. To define them we need the + operation + + \begin{center} + @{thm attach_rexp.simps(2)[where X="Y" and r="r\<^isub>1" and rexp="r\<^isub>2", THEN eq_reflection]}\hspace{10mm} + @{thm attach_rexp.simps(1)[where r="r\<^isub>1" and rexp="r\<^isub>2", THEN eq_reflection]} + \end{center} + *}