Paper/Paper.thy
changeset 94 5b12cd0a3b3c
parent 93 2aa3756dcc9f
child 95 9540c2f2ea77
equal deleted inserted replaced
93:2aa3756dcc9f 94:5b12cd0a3b3c
     1 (*<*)
     1 (*<*)
     2 theory Paper
     2 theory Paper
     3 imports "../Myhill" "LaTeXsugar"
     3 imports "../Myhill" "LaTeXsugar" 
     4 begin
     4 begin
     5 
     5 
     6 declare [[show_question_marks = false]]
     6 declare [[show_question_marks = false]]
     7 
     7 
     8 consts
     8 consts
   497   \end{center}
   497   \end{center}
   498 
   498 
   499   \noindent
   499   \noindent
   500   which we also lift to entire right-hand sides of equations, written as
   500   which we also lift to entire right-hand sides of equations, written as
   501   @{thm (lhs) append_rhs_rexp_def[where rexp="r"]}. With this we can define
   501   @{thm (lhs) append_rhs_rexp_def[where rexp="r"]}. With this we can define
   502   the \emph{arden-operation}, which takes an equivalence class @{text X} and
   502   the \emph{arden-operation} for an equation of the form @{text "X = rhs"}:
   503   a rhs of an equation.
   503   
   504 
   504   \begin{center}
   505   \begin{center}
   505   \begin{tabular}{rc@ {\hspace{2mm}}r@ {\hspace{1mm}}l}
   506   @{thm arden_op_def}
   506   @{thm (lhs) Arden_def} & @{text "\<equiv>"}~~\mbox{} & \multicolumn{2}{@ {\hspace{-2mm}}l}{@{text "let"}}\\ 
   507   \end{center}
   507    & & @{text "rhs' ="} & @{term "rhs - {Trn X r | r. Trn X r \<in> rhs}"} \\
   508 
   508    & & @{text "r' ="}   & @{term "STAR (\<Uplus> {r. Trn X r \<in> rhs})"}\\
   509   \noindent
   509    & &  \multicolumn{2}{@ {\hspace{-2mm}}l}{@{text "in"}~~@{term "append_rhs_rexp rhs' r'"}}\\ 
   510   The term left of $\triangleright$ deletes all terms of the form @{text "(X, r)"};
   510   \end{tabular}
   511   the term on the right calculates first the combinded regular expressions for all
   511   \end{center}
   512   @{text r} in the @{text "(X, r)"}, forms the star and appends it to the remaining
   512 
   513   terms in the @{text rhs}. It can be easily seen that this operation mimics Arden's
   513   \noindent
   514   lemma on the level of equations.
   514   We first delete all terms of the form @{text "(X, r)"} from @{text rhs};
   515   
   515   then we calculate the combinded regular expressions for all @{text r} coming 
       
   516   from the deleted @{text "(X, r)"}, and take the @{const STAR} of it;
       
   517   finally we append this regular expression to @{text rhs'}. It can be easily seen 
       
   518   that this operation mimics Arden's lemma on the level of equations.
       
   519   
       
   520 
       
   521   \begin{center}
       
   522   @{thm Subst_def}
       
   523   \end{center}
   516 *}
   524 *}
   517 
   525 
   518 section {* Regular Expressions Generate Finitely Many Partitions *}
   526 section {* Regular Expressions Generate Finitely Many Partitions *}
   519 
   527 
   520 text {*
   528 text {*