big_lemma.tex
author Chengsong
Mon, 22 Jul 2019 22:30:47 +0100
changeset 78 a67aff8fb06a
permissions -rw-r--r--
proof of big lemma
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
78
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     1
\documentclass{article}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     2
\usepackage[utf8]{inputenc}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     3
\usepackage[english]{babel}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     4
\usepackage{listings}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     5
 \usepackage{amsthm}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     6
 \usepackage{hyperref}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     7
 \usepackage[margin=1in]{geometry}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     8
\usepackage{pmboxdraw}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
     9
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    10
\theoremstyle{theorem}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    11
\newtheorem{theorem}{Theorem}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    12
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    13
\theoremstyle{lemma}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    14
\newtheorem{lemma}{Lemma}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    15
\usepackage{amsmath}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    16
\newcommand{\lemmaautorefname}{Lemma}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    17
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    18
\theoremstyle{definition}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    19
 \newtheorem{definition}{Definition}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    20
\begin{document}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    21
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    22
\section{BIG lemma} \begin{equation}\label{bg} \textit{ bsimp}( \textit{ ALTS}(
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    23
	bs, \textit{ ALTS}( bs_1, as_1),\textit{ ALTS}( bs2, as_2)))) =
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    24
	\textit{ bsimp}(\textit{ALTS}( bs, \textit{ map} \; ( \textit{fuse} \;
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    25
	bs_1) \; as_1 ++  \textit{ map} \; (\textit{fuse} \;  bs_2) \; as_2))
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    26
\end{equation}	We want to show the $ \textit{ LHS}$ of \eqref{bg} is equal to
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    27
the $ \textit{ RHS}$ of \eqref{bg}.  We can first write it in a shorter and
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    28
more readable form. And that is \begin{equation}\label{sm} s (A ( bs, A ( bs_1,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    29
as_1), A ( bs_2, as_2)))=s(A(bs, (bs_1 \rightarrow as_1) @ (bs_2 \rightarrow
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    30
as_2))) \end{equation} Where $s$ means $\textit{bsimp}$ and $A$ stands for
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    31
$\textit{ALTS}$. The right arrow denotes the $\textit{map \; fuse}$ operation.
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    32
We want to transform both sides into function application of $\textit{bsimp}$
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    33
with its arguments involving regexes of the form $s(as_1)$ and $s(as_2)$, which
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    34
can then be expanded by a case-by-case analysis. Each case can then be shown
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    35
with ease.  We have the following:\\ $\textit{LHS}=\textit{s}(A(bs, A(bs_1,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    36
as_1),A(bs_2, as_2)))=s(A(bs, s(A(bs_1,as_1)), s(A(bs_2,as_2)))).$ \\This is by
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    37
a previous lemma. We get "free" $\textit{bsimp}$ on the inner 2
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    38
$\textit{ALTS}$s out of nowhere.  And by application of the inner
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    39
$\textit{bsimp}$ in the above expression, we have that\\ $s(A(bs,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    40
s(A(bs_1,as_1)), s(A(bs_2,as_2)))) = s(A(bs, Li(A(bs_1,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    41
\textit{flts}(s(as_1)))),Li(A(bs_2, \textit{flts}(s(as_2))) ) )).$\\ Now we
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    42
have successfully added $s$ to $as_1$ and $as_2$.  Let us transform the
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    43
$\textit{RHS}$ of equation \eqref{bg}.  \\ $\textit{RHS}=s(s(A(bs, (bs_1
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    44
\rightarrow as_1)@(bs_2 \rightarrow as_2))))=s(Li(A(bs,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    45
\textit{flts}(s(as_1'@as_2'))))).$ \\where the $as_i'$ corresponds to $bs_i
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    46
\rightarrow as_i$.  \\The right hand side of the above equation can again be
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    47
transformed into $s(Li(A(bs, \textit{flts}(s(as_1')@s(as_2'))))).$ \\You might
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    48
want to have a lemma for $s(as_1'@as_2')= s(as_1')@s(as_2')$, which is
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    49
basically a linearity property of the $\textit{map}$ function.  The above
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    50
expression can then again be transformed into $s(Li(A(bs,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    51
\textit{flts}(s(as_1'))@\textit{flts}(s(as_2')))).$ You might again want to
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    52
have a lemma for this linearity property of $\textit{flats}.$\\
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    53
%The above can be then again transformed into $\$
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    54
We now want to equate $s(Li(A(bs,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    55
\textit{flts}(s(as_1'))@\textit{flts}(s(as_2'))))$ with $s(A(bs, Li(A(bs_1,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    56
\textit{flts}(s(as_1)))),Li(A(bs_2, \textit{flts}(s(as_2))) ) ))$ \\ We just
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    57
need to equate the contents inside $\textit{bsimp}$, namely we want to prove\\
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    58
$Li(A(bs, \textit{flts}(s(as_1'))@\textit{flts}(s(as_2'))))$ with $A(bs,
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    59
Li(A(bs_1, \textit{flts}(s(as_1)))),Li(A(bs_2, \textit{flts}(s(as_2))) ) ).$ \\
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    60
This shouldn't be surprising, we have added redundant $\textit{bsimp}$, now we
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    61
are just removing it.  This is where we need a case-by-case analysis.  We need
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    62
to assume the conditions when $s(as_i')$ is empty list, single element list and
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    63
list with 2 or more elements.  They are all trivial and therefore ommitted.
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    64
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    65
\end{document}
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    66
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    67
%The second part might still need some more development.
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    68
%When s is not in the set L(ar), we have that s = s1@s2 s.t. s1 $\in$ L(ar), and any longer string that is a prefix of s does not belong to L(ar).\\
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    69
%By first part of proof, we have ders(ar, s1) $\sim_{m\epsilon}$ ders\_simp(ar, s1)
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    70
%.....somehow show that by correctness, der(c, ders\_simp(ar, s1)) must be not nullable. But this will need that L(ders(ar, s1)) == L(ders\_simp(ar, s1)). By part 1 of proof we only have that for any string s1c s.t. s1c $\in$ L(ar) (which is equivalent to s $\in$ L(ders(ar, s1))), s is also in L(ders\_simp(ar, s1)). That is an inclusion, not an equality. c not in L(ders(ar, s1)) does not imply c not in L(ders\_simp(ar, s1))
a67aff8fb06a proof of big lemma
Chengsong
parents:
diff changeset
    71
%So this path stuck here.