Paper/Paper.thy
author zhang
Sun, 30 Jan 2011 12:22:07 +0000
changeset 49 59936c012add
parent 39 a59473f0229d
child 50 32bff8310071
permissions -rw-r--r--
Illustration added together with renewed explainations for case STAR.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
24
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
     1
(*<*)
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
     2
theory Paper
39
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
     3
imports "../Myhill" "LaTeXsugar"
24
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
     4
begin
39
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
     5
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
     6
declare [[show_question_marks = false]]
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
     7
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
     8
notation (latex output)
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
     9
  str_eq_rel ("\<approx>\<^bsub>_\<^esub>")
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    10
24
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    11
(*>*)
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    12
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    13
section {* Introduction *}
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    14
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    15
text {*
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    16
  
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    17
*}
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    18
39
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    19
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    20
section {* Regular expressions have finitely many partitions *}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    21
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    22
text {*
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    23
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    24
  \begin{lemma}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    25
  Given @{text "r"} is a regular expressions, then @{thm rexp_imp_finite}.
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    26
  \end{lemma}  
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    27
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    28
  \begin{proof}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    29
  By induction on the structure of @{text r}. The cases for @{const NULL}, @{const EMPTY}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    30
  and @{const CHAR} are starightforward, because we can easily establish
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    31
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    32
  \begin{center}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    33
  \begin{tabular}{l}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    34
  @{thm quot_null_eq}\\
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    35
  @{thm quot_empty_subset}\\
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    36
  @{thm quot_char_subset}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    37
  \end{tabular}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    38
  \end{center}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    39
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    40
  
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    41
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    42
  \end{proof}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    43
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    44
*}
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    45
a59473f0229d tuned a little bit the section about finite partitions
urbanc
parents: 37
diff changeset
    46
24
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    47
(*<*)
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    48
end
f72c82bf59e5 added paper
urbanc
parents:
diff changeset
    49
(*>*)