Paper/Paper.thy
changeset 39 a59473f0229d
parent 37 e4d0e6cdc3d2
child 50 32bff8310071
equal deleted inserted replaced
38:a1268fb0deea 39:a59473f0229d
     1 (*<*)
     1 (*<*)
     2 theory Paper
     2 theory Paper
     3 imports "../Myhill"
     3 imports "../Myhill" "LaTeXsugar"
     4 begin
     4 begin
       
     5 
       
     6 declare [[show_question_marks = false]]
       
     7 
       
     8 notation (latex output)
       
     9   str_eq_rel ("\<approx>\<^bsub>_\<^esub>")
       
    10 
     5 (*>*)
    11 (*>*)
     6 
    12 
     7 section {* Introduction *}
    13 section {* Introduction *}
     8 
    14 
     9 text {*
    15 text {*
    10   
    16   
    11 *}
    17 *}
    12 
    18 
       
    19 
       
    20 section {* Regular expressions have finitely many partitions *}
       
    21 
       
    22 text {*
       
    23 
       
    24   \begin{lemma}
       
    25   Given @{text "r"} is a regular expressions, then @{thm rexp_imp_finite}.
       
    26   \end{lemma}  
       
    27 
       
    28   \begin{proof}
       
    29   By induction on the structure of @{text r}. The cases for @{const NULL}, @{const EMPTY}
       
    30   and @{const CHAR} are starightforward, because we can easily establish
       
    31 
       
    32   \begin{center}
       
    33   \begin{tabular}{l}
       
    34   @{thm quot_null_eq}\\
       
    35   @{thm quot_empty_subset}\\
       
    36   @{thm quot_char_subset}
       
    37   \end{tabular}
       
    38   \end{center}
       
    39 
       
    40   
       
    41 
       
    42   \end{proof}
       
    43 
       
    44 *}
       
    45 
       
    46 
    13 (*<*)
    47 (*<*)
    14 end
    48 end
    15 (*>*)
    49 (*>*)