thys/SpecExt.thy
author cu
Tue, 10 Oct 2017 10:40:44 +0100
changeset 278 424bdcd01016
parent 277 42268a284ea6
child 279 f754a10875c7
permissions -rw-r--r--
updated
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     1
   
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     2
theory SpecExt
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     3
  imports Main "~~/src/HOL/Library/Sublist"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     4
begin
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     5
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     6
section {* Sequential Composition of Languages *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     7
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     8
definition
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     9
  Sequ :: "string set \<Rightarrow> string set \<Rightarrow> string set" ("_ ;; _" [100,100] 100)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    10
where 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    11
  "A ;; B = {s1 @ s2 | s1 s2. s1 \<in> A \<and> s2 \<in> B}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    12
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    13
text {* Two Simple Properties about Sequential Composition *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    14
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    15
lemma Sequ_empty_string [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    16
  shows "A ;; {[]} = A"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    17
  and   "{[]} ;; A = A"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    18
by (simp_all add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    19
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    20
lemma Sequ_empty [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    21
  shows "A ;; {} = {}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    22
  and   "{} ;; A = {}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    23
by (simp_all add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    24
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    25
lemma Sequ_assoc:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    26
  shows "(A ;; B) ;; C = A ;; (B ;; C)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    27
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    28
apply blast
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    29
by (metis append_assoc)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    30
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    31
lemma Sequ_Union_in:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    32
  shows "(A ;; (\<Union>x\<in> B. C x)) = (\<Union>x\<in> B. A ;; C x)" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    33
by (auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    34
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    35
section {* Semantic Derivative (Left Quotient) of Languages *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    36
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    37
definition
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    38
  Der :: "char \<Rightarrow> string set \<Rightarrow> string set"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    39
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    40
  "Der c A \<equiv> {s. c # s \<in> A}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    41
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    42
definition
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    43
  Ders :: "string \<Rightarrow> string set \<Rightarrow> string set"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    44
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    45
  "Ders s A \<equiv> {s'. s @ s' \<in> A}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    46
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    47
lemma Der_null [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    48
  shows "Der c {} = {}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    49
unfolding Der_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    50
by auto
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    51
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    52
lemma Der_empty [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    53
  shows "Der c {[]} = {}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    54
unfolding Der_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    55
by auto
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    56
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    57
lemma Der_char [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    58
  shows "Der c {[d]} = (if c = d then {[]} else {})"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    59
unfolding Der_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    60
by auto
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    61
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    62
lemma Der_union [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    63
  shows "Der c (A \<union> B) = Der c A \<union> Der c B"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    64
unfolding Der_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    65
by auto
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    66
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    67
lemma Der_UNION [simp]: 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    68
  shows "Der c (\<Union>x\<in>A. B x) = (\<Union>x\<in>A. Der c (B x))"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    69
by (auto simp add: Der_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    70
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    71
lemma Der_Sequ [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    72
  shows "Der c (A ;; B) = (Der c A) ;; B \<union> (if [] \<in> A then Der c B else {})"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    73
unfolding Der_def Sequ_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    74
by (auto simp add: Cons_eq_append_conv)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    75
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    76
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    77
section {* Kleene Star for Languages *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    78
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    79
inductive_set
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    80
  Star :: "string set \<Rightarrow> string set" ("_\<star>" [101] 102)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    81
  for A :: "string set"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    82
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    83
  start[intro]: "[] \<in> A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    84
| step[intro]:  "\<lbrakk>s1 \<in> A; s2 \<in> A\<star>\<rbrakk> \<Longrightarrow> s1 @ s2 \<in> A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    85
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    86
(* Arden's lemma *)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    87
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    88
lemma Star_cases:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    89
  shows "A\<star> = {[]} \<union> A ;; A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    90
unfolding Sequ_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    91
by (auto) (metis Star.simps)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    92
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    93
lemma Star_decomp: 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    94
  assumes "c # x \<in> A\<star>" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    95
  shows "\<exists>s1 s2. x = s1 @ s2 \<and> c # s1 \<in> A \<and> s2 \<in> A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    96
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    97
by (induct x\<equiv>"c # x" rule: Star.induct) 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    98
   (auto simp add: append_eq_Cons_conv)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    99
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   100
lemma Star_Der_Sequ: 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   101
  shows "Der c (A\<star>) \<subseteq> (Der c A) ;; A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   102
unfolding Der_def Sequ_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   103
by(auto simp add: Star_decomp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   104
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   105
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   106
lemma Der_star [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   107
  shows "Der c (A\<star>) = (Der c A) ;; A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   108
proof -    
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   109
  have "Der c (A\<star>) = Der c ({[]} \<union> A ;; A\<star>)"  
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   110
    by (simp only: Star_cases[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   111
  also have "... = Der c (A ;; A\<star>)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   112
    by (simp only: Der_union Der_empty) (simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   113
  also have "... = (Der c A) ;; A\<star> \<union> (if [] \<in> A then Der c (A\<star>) else {})"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   114
    by simp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   115
  also have "... =  (Der c A) ;; A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   116
    using Star_Der_Sequ by auto
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   117
  finally show "Der c (A\<star>) = (Der c A) ;; A\<star>" .
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   118
qed
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   119
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   120
section {* Power operation for Sets *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   121
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   122
fun 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   123
  Pow :: "string set \<Rightarrow> nat \<Rightarrow> string set" ("_ \<up> _" [101, 102] 101)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   124
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   125
   "A \<up> 0 = {[]}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   126
|  "A \<up> (Suc n) = A ;; (A \<up> n)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   127
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   128
lemma Pow_empty [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   129
  shows "[] \<in> A \<up> n \<longleftrightarrow> (n = 0 \<or> [] \<in> A)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   130
by(induct n) (auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   131
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   132
lemma Pow_Suc_rev:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   133
  "A \<up> (Suc n) =  (A \<up> n) ;; A"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   134
apply(induct n arbitrary: A)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   135
apply(simp_all)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   136
by (metis Sequ_assoc)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   137
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   138
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   139
lemma Pow_decomp: 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   140
  assumes "c # x \<in> A \<up> n" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   141
  shows "\<exists>s1 s2. x = s1 @ s2 \<and> c # s1 \<in> A \<and> s2 \<in> A \<up> (n - 1)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   142
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   143
apply(induct n) 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   144
apply(auto simp add: Cons_eq_append_conv Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   145
apply(case_tac n)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   146
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   147
apply(blast)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   148
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   149
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   150
lemma Star_Pow:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   151
  assumes "s \<in> A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   152
  shows "\<exists>n. s \<in> A \<up> n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   153
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   154
apply(induct)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   155
apply(auto)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   156
apply(rule_tac x="Suc n" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   157
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   158
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   159
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   160
lemma Pow_Star:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   161
  assumes "s \<in> A \<up> n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   162
  shows "s \<in> A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   163
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   164
apply(induct n arbitrary: s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   165
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   166
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   167
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   168
lemma Der_Pow_0:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   169
  shows "Der c (A \<up> 0) = {}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   170
by(simp add: Der_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   171
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   172
lemma Der_Pow_Suc:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   173
  shows "Der c (A \<up> (Suc n)) = (Der c A) ;; (A \<up> n)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   174
unfolding Der_def Sequ_def 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   175
apply(auto simp add: Cons_eq_append_conv Sequ_def dest!: Pow_decomp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   176
apply(case_tac n)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   177
apply(force simp add: Sequ_def)+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   178
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   179
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   180
lemma Der_Pow [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   181
  shows "Der c (A \<up> n) = (if n = 0 then {} else (Der c A) ;; (A \<up> (n - 1)))"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   182
apply(case_tac n)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   183
apply(simp_all del: Pow.simps add: Der_Pow_0 Der_Pow_Suc)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   184
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   185
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   186
lemma Der_Pow_Sequ [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   187
  shows "Der c (A ;; A \<up> n) = (Der c A) ;; (A \<up> n)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   188
by (simp only: Pow.simps[symmetric] Der_Pow) (simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   189
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   190
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   191
lemma Pow_Sequ_Un:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   192
  assumes "0 < x"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   193
  shows "(\<Union>n \<in> {..x}. (A \<up> n)) = ({[]} \<union> (\<Union>n \<in> {..x - Suc 0}. A ;; (A \<up> n)))"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   194
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   195
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   196
apply(smt Pow.elims Sequ_def Suc_le_mono Suc_pred atMost_iff empty_iff insert_iff mem_Collect_eq)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   197
apply(rule_tac x="Suc xa" in bexI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   198
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   199
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   200
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   201
lemma Pow_Sequ_Un2:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   202
  assumes "0 < x"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   203
  shows "(\<Union>n \<in> {x..}. (A \<up> n)) = (\<Union>n \<in> {x - Suc 0..}. A ;; (A \<up> n))"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   204
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   205
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   206
apply(case_tac n)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   207
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   208
apply fastforce
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   209
apply(case_tac x)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   210
apply(auto)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   211
apply(rule_tac x="Suc xa" in bexI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   212
apply(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   213
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   214
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   215
section {* Regular Expressions *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   216
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   217
datatype rexp =
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   218
  ZERO
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   219
| ONE
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   220
| CHAR char
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   221
| SEQ rexp rexp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   222
| ALT rexp rexp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   223
| STAR rexp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   224
| UPNTIMES rexp nat
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   225
| NTIMES rexp nat
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   226
| FROMNTIMES rexp nat
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   227
| NMTIMES rexp nat nat
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   228
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   229
section {* Semantics of Regular Expressions *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   230
 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   231
fun
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   232
  L :: "rexp \<Rightarrow> string set"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   233
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   234
  "L (ZERO) = {}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   235
| "L (ONE) = {[]}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   236
| "L (CHAR c) = {[c]}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   237
| "L (SEQ r1 r2) = (L r1) ;; (L r2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   238
| "L (ALT r1 r2) = (L r1) \<union> (L r2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   239
| "L (STAR r) = (L r)\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   240
| "L (UPNTIMES r n) = (\<Union>i\<in> {..n} . (L r) \<up> i)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   241
| "L (NTIMES r n) = (L r) \<up> n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   242
| "L (FROMNTIMES r n) = (\<Union>i\<in> {n..} . (L r) \<up> i)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   243
| "L (NMTIMES r n m) = (\<Union>i\<in>{n..m} . (L r) \<up> i)" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   244
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   245
section {* Nullable, Derivatives *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   246
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   247
fun
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   248
 nullable :: "rexp \<Rightarrow> bool"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   249
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   250
  "nullable (ZERO) = False"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   251
| "nullable (ONE) = True"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   252
| "nullable (CHAR c) = False"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   253
| "nullable (ALT r1 r2) = (nullable r1 \<or> nullable r2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   254
| "nullable (SEQ r1 r2) = (nullable r1 \<and> nullable r2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   255
| "nullable (STAR r) = True"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   256
| "nullable (UPNTIMES r n) = True"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   257
| "nullable (NTIMES r n) = (if n = 0 then True else nullable r)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   258
| "nullable (FROMNTIMES r n) = (if n = 0 then True else nullable r)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   259
| "nullable (NMTIMES r n m) = (if m < n then False else (if n = 0 then True else nullable r))"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   260
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   261
fun
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   262
 der :: "char \<Rightarrow> rexp \<Rightarrow> rexp"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   263
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   264
  "der c (ZERO) = ZERO"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   265
| "der c (ONE) = ZERO"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   266
| "der c (CHAR d) = (if c = d then ONE else ZERO)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   267
| "der c (ALT r1 r2) = ALT (der c r1) (der c r2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   268
| "der c (SEQ r1 r2) = 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   269
     (if nullable r1
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   270
      then ALT (SEQ (der c r1) r2) (der c r2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   271
      else SEQ (der c r1) r2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   272
| "der c (STAR r) = SEQ (der c r) (STAR r)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   273
| "der c (UPNTIMES r n) = (if n = 0 then ZERO else SEQ (der c r) (UPNTIMES r (n - 1)))"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   274
| "der c (NTIMES r n) = (if n = 0 then ZERO else SEQ (der c r) (NTIMES r (n - 1)))"
277
42268a284ea6 updated
cu
parents: 276
diff changeset
   275
| "der c (FROMNTIMES r n) = 
42268a284ea6 updated
cu
parents: 276
diff changeset
   276
     (if n = 0 
42268a284ea6 updated
cu
parents: 276
diff changeset
   277
      then SEQ (der c r) (STAR r)
42268a284ea6 updated
cu
parents: 276
diff changeset
   278
      else SEQ (der c r) (FROMNTIMES r (n - 1)))"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   279
| "der c (NMTIMES r n m) = 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   280
     (if m < n then ZERO 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   281
      else (if n = 0 then (if m = 0 then ZERO else 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   282
                           SEQ (der c r) (UPNTIMES r (m - 1))) else 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   283
                           SEQ (der c r) (NMTIMES r (n - 1) (m - 1))))" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   284
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   285
fun 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   286
 ders :: "string \<Rightarrow> rexp \<Rightarrow> rexp"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   287
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   288
  "ders [] r = r"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   289
| "ders (c # s) r = ders s (der c r)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   290
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   291
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   292
lemma nullable_correctness:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   293
  shows "nullable r  \<longleftrightarrow> [] \<in> (L r)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   294
by(induct r) (auto simp add: Sequ_def) 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   295
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   296
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   297
lemma der_correctness:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   298
  shows "L (der c r) = Der c (L r)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   299
apply(induct r) 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   300
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   301
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   302
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   303
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   304
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   305
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   306
prefer 2
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   307
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   308
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   309
apply(rule impI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   310
apply(subst Sequ_Union_in)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   311
apply(subst Der_Pow_Sequ[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   312
apply(subst Pow.simps[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   313
apply(subst Der_UNION[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   314
apply(subst Pow_Sequ_Un)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   315
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   316
apply(simp only: Der_union Der_empty)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   317
    apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
   318
(* FROMNTIMES *)    
a3134f7de065 updated
cu
parents: 275
diff changeset
   319
   apply(simp add: nullable_correctness del: Der_UNION)
277
42268a284ea6 updated
cu
parents: 276
diff changeset
   320
  apply(rule conjI)
42268a284ea6 updated
cu
parents: 276
diff changeset
   321
prefer 2    
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   322
apply(subst Sequ_Union_in)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   323
apply(subst Der_Pow_Sequ[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   324
apply(subst Pow.simps[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   325
apply(case_tac x2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   326
prefer 2
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   327
apply(subst Pow_Sequ_Un2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   328
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   329
apply(simp)
277
42268a284ea6 updated
cu
parents: 276
diff changeset
   330
    apply(auto simp add: Sequ_def Der_def)[1]
42268a284ea6 updated
cu
parents: 276
diff changeset
   331
   apply(auto simp add: Sequ_def split: if_splits)[1]
42268a284ea6 updated
cu
parents: 276
diff changeset
   332
  using Star_Pow apply fastforce
42268a284ea6 updated
cu
parents: 276
diff changeset
   333
  using Pow_Star apply blast
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   334
(* NMTIMES *)    
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   335
apply(simp add: nullable_correctness del: Der_UNION)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   336
apply(rule impI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   337
apply(rule conjI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   338
apply(rule impI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   339
apply(subst Sequ_Union_in)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   340
apply(subst Der_Pow_Sequ[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   341
apply(subst Pow.simps[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   342
apply(subst Der_UNION[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   343
apply(case_tac x3a)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   344
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   345
apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   346
apply(auto simp add: Sequ_def Der_def Cons_eq_append_conv)[1]
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   347
apply(rule_tac x="Suc xa" in bexI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   348
apply(auto simp add: Sequ_def)[2]
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   349
apply (metis append_Cons)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   350
apply (metis (no_types, hide_lams) Pow_decomp atMost_iff diff_Suc_eq_diff_pred diff_is_0_eq)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   351
apply(rule impI)+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   352
apply(subst Sequ_Union_in)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   353
apply(subst Der_Pow_Sequ[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   354
apply(subst Pow.simps[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   355
apply(subst Der_UNION[symmetric])
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   356
apply(case_tac x2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   357
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   358
apply(simp del: Pow.simps)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   359
apply(auto simp add: Sequ_def Der_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   360
apply (metis One_nat_def Suc_le_D Suc_le_mono atLeastAtMost_iff diff_Suc_1 not_le)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   361
by fastforce
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   362
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   363
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   364
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   365
lemma ders_correctness:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   366
  shows "L (ders s r) = Ders s (L r)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   367
by (induct s arbitrary: r)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   368
   (simp_all add: Ders_def der_correctness Der_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   369
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   370
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   371
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   372
section {* Values *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   373
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   374
datatype val = 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   375
  Void
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   376
| Char char
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   377
| Seq val val
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   378
| Right val
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   379
| Left val
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   380
| Stars "val list"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   381
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   382
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   383
section {* The string behind a value *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   384
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   385
fun 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   386
  flat :: "val \<Rightarrow> string"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   387
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   388
  "flat (Void) = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   389
| "flat (Char c) = [c]"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   390
| "flat (Left v) = flat v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   391
| "flat (Right v) = flat v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   392
| "flat (Seq v1 v2) = (flat v1) @ (flat v2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   393
| "flat (Stars []) = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   394
| "flat (Stars (v#vs)) = (flat v) @ (flat (Stars vs))" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   395
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   396
abbreviation
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   397
  "flats vs \<equiv> concat (map flat vs)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   398
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   399
lemma flat_Stars [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   400
 "flat (Stars vs) = flats vs"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   401
by (induct vs) (auto)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   402
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   403
lemma Star_concat:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   404
  assumes "\<forall>s \<in> set ss. s \<in> A"  
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   405
  shows "concat ss \<in> A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   406
using assms by (induct ss) (auto)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   407
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   408
lemma Star_cstring:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   409
  assumes "s \<in> A\<star>"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   410
  shows "\<exists>ss. concat ss = s \<and> (\<forall>s \<in> set ss. s \<in> A \<and> s \<noteq> [])"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   411
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   412
apply(induct rule: Star.induct)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   413
apply(auto)[1]
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   414
apply(rule_tac x="[]" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   415
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   416
apply(erule exE)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   417
apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   418
apply(case_tac "s1 = []")
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   419
apply(rule_tac x="ss" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   420
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   421
apply(rule_tac x="s1#ss" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   422
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   423
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   424
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   425
lemma Aux:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   426
  assumes "\<forall>s\<in>set ss. s = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   427
  shows "concat ss = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   428
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   429
by (induct ss) (auto)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   430
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   431
lemma Pow_cstring_nonempty:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   432
  assumes "s \<in> A \<up> n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   433
  shows "\<exists>ss. concat ss = s \<and> length ss \<le> n \<and> (\<forall>s \<in> set ss. s \<in> A \<and> s \<noteq> [])"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   434
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   435
apply(induct n arbitrary: s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   436
apply(auto)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   437
apply(simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   438
apply(erule exE)+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   439
apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   440
apply(drule_tac x="s2" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   441
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   442
apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   443
apply(case_tac "s1 = []")
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   444
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   445
apply(rule_tac x="ss" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   446
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   447
apply(rule_tac x="s1 # ss" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   448
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   449
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   450
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   451
lemma Pow_cstring:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   452
  assumes "s \<in> A \<up> n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   453
  shows "\<exists>ss1 ss2. concat (ss1 @ ss2) = s \<and> length (ss1 @ ss2) = n \<and> 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   454
         (\<forall>s \<in> set ss1. s \<in> A \<and> s \<noteq> []) \<and> (\<forall>s \<in> set ss2. s \<in> A \<and> s = [])"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   455
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   456
apply(induct n arbitrary: s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   457
apply(auto)[1]
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   458
apply(simp only: Pow_Suc_rev)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   459
apply(simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   460
apply(erule exE)+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   461
apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   462
apply(drule_tac x="s1" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   463
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   464
apply(erule exE)+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   465
apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   466
apply(case_tac "s2 = []")
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   467
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   468
apply(rule_tac x="ss1" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   469
apply(rule_tac x="s2#ss2" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   470
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   471
apply(rule_tac x="ss1 @ [s2]" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   472
apply(rule_tac x="ss2" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   473
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   474
apply(subst Aux)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   475
apply(auto)[1]
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   476
apply(subst Aux)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   477
apply(auto)[1]
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   478
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   479
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   480
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   481
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   482
section {* Lexical Values *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   483
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   484
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   485
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   486
inductive 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   487
  Prf :: "val \<Rightarrow> rexp \<Rightarrow> bool" ("\<Turnstile> _ : _" [100, 100] 100)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   488
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   489
 "\<lbrakk>\<Turnstile> v1 : r1; \<Turnstile> v2 : r2\<rbrakk> \<Longrightarrow> \<Turnstile>  Seq v1 v2 : SEQ r1 r2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   490
| "\<Turnstile> v1 : r1 \<Longrightarrow> \<Turnstile> Left v1 : ALT r1 r2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   491
| "\<Turnstile> v2 : r2 \<Longrightarrow> \<Turnstile> Right v2 : ALT r1 r2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   492
| "\<Turnstile> Void : ONE"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   493
| "\<Turnstile> Char c : CHAR c"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   494
| "\<lbrakk>\<forall>v \<in> set vs. \<Turnstile> v : r \<and> flat v \<noteq> []\<rbrakk> \<Longrightarrow> \<Turnstile> Stars vs : STAR r"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   495
| "\<lbrakk>\<forall>v \<in> set vs. \<Turnstile> v : r \<and> flat v \<noteq> []; length vs \<le> n\<rbrakk> \<Longrightarrow> \<Turnstile> Stars vs : UPNTIMES r n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   496
| "\<lbrakk>\<forall>v \<in> set vs1. \<Turnstile> v : r \<and> flat v \<noteq> []; 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   497
    \<forall>v \<in> set vs2. \<Turnstile> v : r \<and> flat v = []; 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   498
    length (vs1 @ vs2) = n\<rbrakk> \<Longrightarrow> \<Turnstile> Stars (vs1 @ vs2) : NTIMES r n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   499
| "\<lbrakk>\<forall>v \<in> set vs1. \<Turnstile> v : r  \<and> flat v \<noteq> []; 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   500
    \<forall>v \<in> set vs2. \<Turnstile> v : r \<and> flat v = []; 
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   501
    length (vs1 @ vs2) = n\<rbrakk> \<Longrightarrow> \<Turnstile> Stars (vs1 @ vs2) : FROMNTIMES r n"
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   502
| "\<lbrakk>\<forall>v \<in> set vs. \<Turnstile> v : r  \<and> flat v \<noteq> []; length vs > n\<rbrakk> \<Longrightarrow> \<Turnstile> Stars vs : FROMNTIMES r n"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   503
| "\<lbrakk>\<forall>v \<in> set vs1. \<Turnstile> v : r \<and> flat v \<noteq> [];
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   504
    \<forall>v \<in> set vs2. \<Turnstile> v : r \<and> flat v = []; 
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   505
    length (vs1 @ vs2) = n; length (vs1 @ vs2) \<le> m\<rbrakk> \<Longrightarrow> \<Turnstile> Stars (vs1 @ vs2) : NMTIMES r n m"
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   506
| "\<lbrakk>\<forall>v \<in> set vs. \<Turnstile> v : r \<and> flat v \<noteq> [];
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   507
    length vs > n; length vs \<le> m\<rbrakk> \<Longrightarrow> \<Turnstile> Stars vs : NMTIMES r n m"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   508
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   509
  
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   510
inductive_cases Prf_elims:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   511
  "\<Turnstile> v : ZERO"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   512
  "\<Turnstile> v : SEQ r1 r2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   513
  "\<Turnstile> v : ALT r1 r2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   514
  "\<Turnstile> v : ONE"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   515
  "\<Turnstile> v : CHAR c"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   516
  "\<Turnstile> vs : STAR r"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   517
  "\<Turnstile> vs : UPNTIMES r n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   518
  "\<Turnstile> vs : NTIMES r n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   519
  "\<Turnstile> vs : FROMNTIMES r n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   520
  "\<Turnstile> vs : NMTIMES r n m"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   521
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   522
lemma Prf_Stars_appendE:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   523
  assumes "\<Turnstile> Stars (vs1 @ vs2) : STAR r"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   524
  shows "\<Turnstile> Stars vs1 : STAR r \<and> \<Turnstile> Stars vs2 : STAR r" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   525
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   526
by (auto intro: Prf.intros elim!: Prf_elims)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   527
274
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   528
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   529
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   530
lemma flats_empty:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   531
  assumes "(\<forall>v\<in>set vs. flat v = [])"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   532
  shows "flats vs = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   533
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   534
by(induct vs) (simp_all)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   535
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   536
lemma Star_cval:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   537
  assumes "\<forall>s\<in>set ss. \<exists>v. s = flat v \<and> \<Turnstile> v : r"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   538
  shows "\<exists>vs. flats vs = concat ss \<and> (\<forall>v\<in>set vs. \<Turnstile> v : r \<and> flat v \<noteq> [])"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   539
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   540
apply(induct ss)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   541
apply(auto)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   542
apply(rule_tac x="[]" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   543
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   544
apply(case_tac "flat v = []")
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   545
apply(rule_tac x="vs" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   546
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   547
apply(rule_tac x="v#vs" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   548
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   549
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   550
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   551
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   552
lemma flats_cval:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   553
  assumes "\<forall>s\<in>set ss. \<exists>v. s = flat v \<and> \<Turnstile> v : r"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   554
  shows "\<exists>vs1 vs2. flats (vs1 @ vs2) = concat ss \<and> length (vs1 @ vs2) = length ss \<and> 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   555
          (\<forall>v\<in>set vs1. \<Turnstile> v : r \<and> flat v \<noteq> []) \<and>
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   556
          (\<forall>v\<in>set vs2. \<Turnstile> v : r \<and> flat v = [])"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   557
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   558
apply(induct ss rule: rev_induct)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   559
apply(rule_tac x="[]" in exI)+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   560
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   561
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   562
apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   563
apply(case_tac "flat v = []")
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   564
apply(rule_tac x="vs1" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   565
apply(rule_tac x="v#vs2" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   566
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   567
apply(rule_tac x="vs1 @ [v]" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   568
apply(rule_tac x="vs2" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   569
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   570
apply(subst (asm) (2) flats_empty)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   571
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   572
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   573
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   574
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   575
lemma flats_cval_nonempty:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   576
  assumes "\<forall>s\<in>set ss. \<exists>v. s = flat v \<and> \<Turnstile> v : r"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   577
  shows "\<exists>vs. flats vs = concat ss \<and> length vs \<le> length ss \<and> 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   578
          (\<forall>v\<in>set vs. \<Turnstile> v : r \<and> flat v \<noteq> [])" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   579
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   580
apply(induct ss)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   581
apply(rule_tac x="[]" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   582
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   583
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   584
apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   585
apply(case_tac "flat v = []")
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   586
apply(rule_tac x="vs" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   587
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   588
apply(rule_tac x="v # vs" in exI)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   589
apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   590
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   591
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   592
lemma Pow_flats:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   593
  assumes "\<forall>v \<in> set vs. flat v \<in> A"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   594
  shows "flats vs \<in> A \<up> length vs"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   595
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   596
by(induct vs)(auto simp add: Sequ_def)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   597
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   598
lemma Pow_flats_appends:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   599
  assumes "\<forall>v \<in> set vs1. flat v \<in> A" "\<forall>v \<in> set vs2. flat v \<in> A"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   600
  shows "flats vs1 @ flats vs2 \<in> A \<up> (length vs1 + length vs2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   601
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   602
apply(induct vs1)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   603
apply(auto simp add: Sequ_def Pow_flats)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   604
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   605
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   606
lemma L_flat_Prf1:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   607
  assumes "\<Turnstile> v : r" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   608
  shows "flat v \<in> L r"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   609
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   610
apply(induct) 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   611
apply(auto simp add: Sequ_def Star_concat Pow_flats)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   612
apply(meson Pow_flats atMost_iff)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   613
using Pow_flats_appends apply blast
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   614
using Pow_flats_appends apply blast
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   615
apply (meson Pow_flats atLeast_iff less_imp_le)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   616
apply(rule_tac x="length vs1 + length vs2" in  bexI)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   617
apply(meson Pow_flats_appends atLeastAtMost_iff)
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   618
apply(simp)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   619
apply(meson Pow_flats atLeastAtMost_iff less_or_eq_imp_le)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   620
done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   621
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   622
lemma L_flat_Prf2:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   623
  assumes "s \<in> L r" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   624
  shows "\<exists>v. \<Turnstile> v : r \<and> flat v = s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   625
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   626
proof(induct r arbitrary: s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   627
  case (STAR r s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   628
  have IH: "\<And>s. s \<in> L r \<Longrightarrow> \<exists>v. \<Turnstile> v : r \<and> flat v = s" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   629
  have "s \<in> L (STAR r)" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   630
  then obtain ss where "concat ss = s" "\<forall>s \<in> set ss. s \<in> L r \<and> s \<noteq> []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   631
  using Star_cstring by auto  
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   632
  then obtain vs where "flats vs = s" "\<forall>v\<in>set vs. \<Turnstile> v : r \<and> flat v \<noteq> []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   633
  using IH Star_cval by metis 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   634
  then show "\<exists>v. \<Turnstile> v : STAR r \<and> flat v = s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   635
  using Prf.intros(6) flat_Stars by blast
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   636
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   637
  case (SEQ r1 r2 s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   638
  then show "\<exists>v. \<Turnstile> v : SEQ r1 r2 \<and> flat v = s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   639
  unfolding Sequ_def L.simps by (fastforce intro: Prf.intros)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   640
next
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   641
  case (ALT r1 r2 s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   642
  then show "\<exists>v. \<Turnstile> v : ALT r1 r2 \<and> flat v = s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   643
  unfolding L.simps by (fastforce intro: Prf.intros)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   644
next
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   645
  case (NTIMES r n)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   646
  have IH: "\<And>s. s \<in> L r \<Longrightarrow> \<exists>v. \<Turnstile> v : r \<and> flat v = s" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   647
  have "s \<in> L (NTIMES r n)" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   648
  then obtain ss1 ss2 where "concat (ss1 @ ss2) = s" "length (ss1 @ ss2) = n" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   649
    "\<forall>s \<in> set ss1. s \<in> L r \<and> s \<noteq> []" "\<forall>s \<in> set ss2. s \<in> L r \<and> s = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   650
  using Pow_cstring by force
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   651
  then obtain vs1 vs2 where "flats (vs1 @ vs2) = s" "length (vs1 @ vs2) = n" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   652
      "\<forall>v\<in>set vs1. \<Turnstile> v : r \<and> flat v \<noteq> []" "\<forall>v\<in>set vs2. \<Turnstile> v : r \<and> flat v = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   653
  using IH flats_cval 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   654
  apply -
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   655
  apply(drule_tac x="ss1 @ ss2" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   656
  apply(drule_tac x="r" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   657
  apply(drule meta_mp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   658
  apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   659
  apply (metis Un_iff)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   660
  apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   661
  apply(drule_tac x="vs1" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   662
  apply(drule_tac x="vs2" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   663
  apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   664
  done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   665
  then show "\<exists>v. \<Turnstile> v : NTIMES r n \<and> flat v = s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   666
  using Prf.intros(8) flat_Stars by blast
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   667
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   668
  case (FROMNTIMES r n)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   669
  have IH: "\<And>s. s \<in> L r \<Longrightarrow> \<exists>v. \<Turnstile> v : r \<and> flat v = s" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   670
  have "s \<in> L (FROMNTIMES r n)" by fact 
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   671
  then obtain ss1 ss2 k where "concat (ss1 @ ss2) = s" "length (ss1 @ ss2) = k"  "n \<le> k"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   672
    "\<forall>s \<in> set ss1. s \<in> L r \<and> s \<noteq> []" "\<forall>s \<in> set ss2. s \<in> L r \<and> s = []"
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   673
    using Pow_cstring by force 
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   674
  then obtain vs1 vs2 where "flats (vs1 @ vs2) = s" "length (vs1 @ vs2) = k" "n \<le> k"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   675
      "\<forall>v\<in>set vs1. \<Turnstile> v : r \<and> flat v \<noteq> []" "\<forall>v\<in>set vs2. \<Turnstile> v : r \<and> flat v = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   676
  using IH flats_cval 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   677
  apply -
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   678
  apply(drule_tac x="ss1 @ ss2" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   679
  apply(drule_tac x="r" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   680
  apply(drule meta_mp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   681
  apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   682
  apply (metis Un_iff)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   683
  apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   684
  apply(drule_tac x="vs1" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   685
  apply(drule_tac x="vs2" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   686
  apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   687
  done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   688
  then show "\<exists>v. \<Turnstile> v : FROMNTIMES r n \<and> flat v = s"
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   689
  apply(case_tac "length vs1 \<le> n")
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   690
  apply(rule_tac x="Stars (vs1 @ take (n - length vs1) vs2)" in exI)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   691
  apply(simp)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   692
  apply(subgoal_tac "flats (take (n - length vs1) vs2) = []")
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   693
  prefer 2
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   694
  apply (meson flats_empty in_set_takeD)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   695
  apply(clarify)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   696
    apply(rule conjI)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   697
      apply(rule Prf.intros)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   698
        apply(simp)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   699
       apply (meson in_set_takeD)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   700
      apply(simp)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   701
     apply(simp)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   702
     apply (simp add: flats_empty)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   703
      apply(rule_tac x="Stars vs1" in exI)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   704
  apply(simp)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   705
    apply(rule conjI)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   706
     apply(rule Prf.intros(10))
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   707
      apply(auto)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   708
  done    
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   709
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   710
  case (NMTIMES r n m)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   711
  have IH: "\<And>s. s \<in> L r \<Longrightarrow> \<exists>v. \<Turnstile> v : r \<and> flat v = s" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   712
  have "s \<in> L (NMTIMES r n m)" by fact 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   713
  then obtain ss1 ss2 k where "concat (ss1 @ ss2) = s" "length (ss1 @ ss2) = k" "n \<le> k" "k \<le> m" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   714
    "\<forall>s \<in> set ss1. s \<in> L r \<and> s \<noteq> []" "\<forall>s \<in> set ss2. s \<in> L r \<and> s = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   715
  using Pow_cstring by (auto, blast)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   716
  then obtain vs1 vs2 where "flats (vs1 @ vs2) = s" "length (vs1 @ vs2) = k" "n \<le> k" "k \<le> m"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   717
      "\<forall>v\<in>set vs1. \<Turnstile> v : r \<and> flat v \<noteq> []" "\<forall>v\<in>set vs2. \<Turnstile> v : r \<and> flat v = []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   718
  using IH flats_cval 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   719
  apply -
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   720
  apply(drule_tac x="ss1 @ ss2" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   721
  apply(drule_tac x="r" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   722
  apply(drule meta_mp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   723
  apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   724
  apply (metis Un_iff)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   725
  apply(clarify)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   726
  apply(drule_tac x="vs1" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   727
  apply(drule_tac x="vs2" in meta_spec)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   728
  apply(simp)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   729
  done
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   730
  then show "\<exists>v. \<Turnstile> v : NMTIMES r n m \<and> flat v = s"
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   731
    apply(case_tac "length vs1 \<le> n")
a3134f7de065 updated
cu
parents: 275
diff changeset
   732
  apply(rule_tac x="Stars (vs1 @ take (n - length vs1) vs2)" in exI)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   733
  apply(simp)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   734
  apply(subgoal_tac "flats (take (n - length vs1) vs2) = []")
a3134f7de065 updated
cu
parents: 275
diff changeset
   735
  prefer 2
a3134f7de065 updated
cu
parents: 275
diff changeset
   736
  apply (meson flats_empty in_set_takeD)
a3134f7de065 updated
cu
parents: 275
diff changeset
   737
  apply(clarify)
a3134f7de065 updated
cu
parents: 275
diff changeset
   738
    apply(rule conjI)
a3134f7de065 updated
cu
parents: 275
diff changeset
   739
      apply(rule Prf.intros)
a3134f7de065 updated
cu
parents: 275
diff changeset
   740
        apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
   741
       apply (meson in_set_takeD)
a3134f7de065 updated
cu
parents: 275
diff changeset
   742
      apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
   743
     apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
   744
     apply (simp add: flats_empty)
a3134f7de065 updated
cu
parents: 275
diff changeset
   745
      apply(rule_tac x="Stars vs1" in exI)
a3134f7de065 updated
cu
parents: 275
diff changeset
   746
  apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
   747
    apply(rule conjI)
a3134f7de065 updated
cu
parents: 275
diff changeset
   748
     apply(rule Prf.intros)
a3134f7de065 updated
cu
parents: 275
diff changeset
   749
      apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
   750
  done    
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   751
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   752
  case (UPNTIMES r n s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   753
  have IH: "\<And>s. s \<in> L r \<Longrightarrow> \<exists>v. \<Turnstile> v : r \<and> flat v = s" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   754
  have "s \<in> L (UPNTIMES r n)" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   755
  then obtain ss where "concat ss = s" "\<forall>s \<in> set ss. s \<in> L r \<and> s \<noteq> []" "length ss \<le> n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   756
  using Pow_cstring_nonempty by force
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   757
  then obtain vs where "flats vs = s" "\<forall>v\<in>set vs. \<Turnstile> v : r \<and> flat v \<noteq> []" "length vs \<le> n"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   758
  using IH flats_cval_nonempty by (smt order.trans) 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   759
  then show "\<exists>v. \<Turnstile> v : UPNTIMES r n \<and> flat v = s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   760
  using Prf.intros(7) flat_Stars by blast
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   761
qed (auto intro: Prf.intros)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   762
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   763
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   764
lemma L_flat_Prf:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   765
  shows "L(r) = {flat v | v. \<Turnstile> v : r}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   766
using L_flat_Prf1 L_flat_Prf2 by blast
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   767
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   768
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   769
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   770
section {* Sets of Lexical Values *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   771
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   772
text {*
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   773
  Shows that lexical values are finite for a given regex and string.
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   774
*}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   775
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   776
definition
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   777
  LV :: "rexp \<Rightarrow> string \<Rightarrow> val set"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   778
where  "LV r s \<equiv> {v. \<Turnstile> v : r \<and> flat v = s}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   779
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   780
lemma LV_simps:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   781
  shows "LV ZERO s = {}"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   782
  and   "LV ONE s = (if s = [] then {Void} else {})"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   783
  and   "LV (CHAR c) s = (if s = [c] then {Char c} else {})"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   784
  and   "LV (ALT r1 r2) s = Left ` LV r1 s \<union> Right ` LV r2 s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   785
unfolding LV_def
274
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   786
apply(auto intro: Prf.intros elim: Prf.cases)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   787
done
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   788
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   789
abbreviation
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   790
  "Prefixes s \<equiv> {s'. prefix s' s}"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   791
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   792
abbreviation
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   793
  "Suffixes s \<equiv> {s'. suffix s' s}"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   794
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   795
abbreviation
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   796
  "SSuffixes s \<equiv> {s'. strict_suffix s' s}"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   797
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   798
lemma Suffixes_cons [simp]:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   799
  shows "Suffixes (c # s) = Suffixes s \<union> {c # s}"
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   800
by (auto simp add: suffix_def Cons_eq_append_conv)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   801
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   802
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   803
lemma finite_Suffixes: 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   804
  shows "finite (Suffixes s)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   805
by (induct s) (simp_all)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   806
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   807
lemma finite_SSuffixes: 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   808
  shows "finite (SSuffixes s)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   809
proof -
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   810
  have "SSuffixes s \<subseteq> Suffixes s"
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   811
   unfolding suffix_def strict_suffix_def by auto
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   812
  then show "finite (SSuffixes s)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   813
   using finite_Suffixes finite_subset by blast
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   814
qed
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   815
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   816
lemma finite_Prefixes: 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   817
  shows "finite (Prefixes s)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   818
proof -
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   819
  have "finite (Suffixes (rev s))" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   820
    by (rule finite_Suffixes)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   821
  then have "finite (rev ` Suffixes (rev s))" by simp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   822
  moreover
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   823
  have "rev ` (Suffixes (rev s)) = Prefixes s"
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   824
  unfolding suffix_def prefix_def image_def
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   825
   by (auto)(metis rev_append rev_rev_ident)+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   826
  ultimately show "finite (Prefixes s)" by simp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   827
qed
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   828
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   829
definition
a3134f7de065 updated
cu
parents: 275
diff changeset
   830
  "Stars_Cons V Vs \<equiv> {Stars (v # vs) | v vs. v \<in> V \<and> Stars vs \<in> Vs}"
a3134f7de065 updated
cu
parents: 275
diff changeset
   831
  
a3134f7de065 updated
cu
parents: 275
diff changeset
   832
definition
a3134f7de065 updated
cu
parents: 275
diff changeset
   833
  "Stars_Append Vs1 Vs2 \<equiv> {Stars (vs1 @ vs2) | vs1 vs2. Stars vs1 \<in> Vs1 \<and> Stars vs2 \<in> Vs2}"
a3134f7de065 updated
cu
parents: 275
diff changeset
   834
a3134f7de065 updated
cu
parents: 275
diff changeset
   835
fun Stars_Pow :: "val set \<Rightarrow> nat \<Rightarrow> val set"
a3134f7de065 updated
cu
parents: 275
diff changeset
   836
where  
a3134f7de065 updated
cu
parents: 275
diff changeset
   837
  "Stars_Pow Vs 0 = {Stars []}"
a3134f7de065 updated
cu
parents: 275
diff changeset
   838
| "Stars_Pow Vs (Suc n) = Stars_Cons Vs (Stars_Pow Vs n)"
a3134f7de065 updated
cu
parents: 275
diff changeset
   839
  
a3134f7de065 updated
cu
parents: 275
diff changeset
   840
lemma finite_Stars_Cons:
a3134f7de065 updated
cu
parents: 275
diff changeset
   841
  assumes "finite V" "finite Vs"
a3134f7de065 updated
cu
parents: 275
diff changeset
   842
  shows "finite (Stars_Cons V Vs)"
a3134f7de065 updated
cu
parents: 275
diff changeset
   843
  using assms  
a3134f7de065 updated
cu
parents: 275
diff changeset
   844
proof -
a3134f7de065 updated
cu
parents: 275
diff changeset
   845
  from assms(2) have "finite (Stars -` Vs)"
a3134f7de065 updated
cu
parents: 275
diff changeset
   846
    by(simp add: finite_vimageI inj_on_def) 
a3134f7de065 updated
cu
parents: 275
diff changeset
   847
  with assms(1) have "finite (V \<times> (Stars -` Vs))"
a3134f7de065 updated
cu
parents: 275
diff changeset
   848
    by(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
   849
  then have "finite ((\<lambda>(v, vs). Stars (v # vs)) ` (V \<times> (Stars -` Vs)))"
a3134f7de065 updated
cu
parents: 275
diff changeset
   850
    by simp
a3134f7de065 updated
cu
parents: 275
diff changeset
   851
  moreover have "Stars_Cons V Vs = (\<lambda>(v, vs). Stars (v # vs)) ` (V \<times> (Stars -` Vs))"
a3134f7de065 updated
cu
parents: 275
diff changeset
   852
    unfolding Stars_Cons_def by auto    
a3134f7de065 updated
cu
parents: 275
diff changeset
   853
  ultimately show "finite (Stars_Cons V Vs)"   
a3134f7de065 updated
cu
parents: 275
diff changeset
   854
    by simp
a3134f7de065 updated
cu
parents: 275
diff changeset
   855
qed
a3134f7de065 updated
cu
parents: 275
diff changeset
   856
a3134f7de065 updated
cu
parents: 275
diff changeset
   857
lemma finite_Stars_Append:
a3134f7de065 updated
cu
parents: 275
diff changeset
   858
  assumes "finite Vs1" "finite Vs2"
a3134f7de065 updated
cu
parents: 275
diff changeset
   859
  shows "finite (Stars_Append Vs1 Vs2)"
a3134f7de065 updated
cu
parents: 275
diff changeset
   860
  using assms  
a3134f7de065 updated
cu
parents: 275
diff changeset
   861
proof -
a3134f7de065 updated
cu
parents: 275
diff changeset
   862
  define UVs1 where "UVs1 \<equiv> Stars -` Vs1"
a3134f7de065 updated
cu
parents: 275
diff changeset
   863
  define UVs2 where "UVs2 \<equiv> Stars -` Vs2"  
a3134f7de065 updated
cu
parents: 275
diff changeset
   864
  from assms have "finite UVs1" "finite UVs2"
a3134f7de065 updated
cu
parents: 275
diff changeset
   865
    unfolding UVs1_def UVs2_def
a3134f7de065 updated
cu
parents: 275
diff changeset
   866
    by(simp_all add: finite_vimageI inj_on_def) 
a3134f7de065 updated
cu
parents: 275
diff changeset
   867
  then have "finite ((\<lambda>(vs1, vs2). Stars (vs1 @ vs2)) ` (UVs1 \<times> UVs2))"
a3134f7de065 updated
cu
parents: 275
diff changeset
   868
    by simp
a3134f7de065 updated
cu
parents: 275
diff changeset
   869
  moreover 
a3134f7de065 updated
cu
parents: 275
diff changeset
   870
    have "Stars_Append Vs1 Vs2 = (\<lambda>(vs1, vs2). Stars (vs1 @ vs2)) ` (UVs1 \<times> UVs2)"
a3134f7de065 updated
cu
parents: 275
diff changeset
   871
    unfolding Stars_Append_def UVs1_def UVs2_def by auto    
a3134f7de065 updated
cu
parents: 275
diff changeset
   872
  ultimately show "finite (Stars_Append Vs1 Vs2)"   
a3134f7de065 updated
cu
parents: 275
diff changeset
   873
    by simp
a3134f7de065 updated
cu
parents: 275
diff changeset
   874
qed 
a3134f7de065 updated
cu
parents: 275
diff changeset
   875
 
a3134f7de065 updated
cu
parents: 275
diff changeset
   876
lemma finite_Stars_Pow:
a3134f7de065 updated
cu
parents: 275
diff changeset
   877
  assumes "finite Vs"
a3134f7de065 updated
cu
parents: 275
diff changeset
   878
  shows "finite (Stars_Pow Vs n)"    
a3134f7de065 updated
cu
parents: 275
diff changeset
   879
by (induct n) (simp_all add: finite_Stars_Cons assms)
a3134f7de065 updated
cu
parents: 275
diff changeset
   880
    
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   881
lemma LV_STAR_finite:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   882
  assumes "\<forall>s. finite (LV r s)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   883
  shows "finite (LV (STAR r) s)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   884
proof(induct s rule: length_induct)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   885
  fix s::"char list"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   886
  assume "\<forall>s'. length s' < length s \<longrightarrow> finite (LV (STAR r) s')"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   887
  then have IH: "\<forall>s' \<in> SSuffixes s. finite (LV (STAR r) s')"
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   888
    by (auto simp add: strict_suffix_def) 
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   889
  define f where "f \<equiv> \<lambda>(v, vs). Stars (v # vs)"
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   890
  define S1 where "S1 \<equiv> \<Union>s' \<in> Prefixes s. LV r s'"
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   891
  define S2 where "S2 \<equiv> \<Union>s2 \<in> SSuffixes s. LV (STAR r) s2"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   892
  have "finite S1" using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   893
    unfolding S1_def by (simp_all add: finite_Prefixes)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   894
  moreover 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   895
  with IH have "finite S2" unfolding S2_def
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   896
    by (auto simp add: finite_SSuffixes)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   897
  ultimately 
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   898
  have "finite ({Stars []} \<union> Stars_Cons S1 S2)" 
a3134f7de065 updated
cu
parents: 275
diff changeset
   899
    by (simp add: finite_Stars_Cons)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   900
  moreover 
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   901
  have "LV (STAR r) s \<subseteq> {Stars []} \<union> (Stars_Cons S1 S2)" 
a3134f7de065 updated
cu
parents: 275
diff changeset
   902
  unfolding S1_def S2_def f_def LV_def Stars_Cons_def
a3134f7de065 updated
cu
parents: 275
diff changeset
   903
  unfolding prefix_def strict_suffix_def 
a3134f7de065 updated
cu
parents: 275
diff changeset
   904
  unfolding image_def
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   905
  apply(auto)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   906
  apply(case_tac x)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   907
  apply(auto elim: Prf_elims)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   908
  apply(erule Prf_elims)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   909
  apply(auto)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   910
  apply(case_tac vs)
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   911
  apply(auto intro: Prf.intros)  
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   912
  apply(rule exI)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   913
  apply(rule conjI)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   914
  apply(rule_tac x="flats list" in exI)
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   915
  apply(rule conjI)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   916
  apply(rule_tac x="flat a" in exI)
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   917
  apply(simp)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   918
  apply(blast)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   919
  using Prf.intros(6) flat_Stars by blast  
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   920
  ultimately
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   921
  show "finite (LV (STAR r) s)" by (simp add: finite_subset)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   922
qed  
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   923
    
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   924
lemma LV_UPNTIMES_STAR:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   925
  "LV (UPNTIMES r n) s \<subseteq> LV (STAR r) s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   926
by(auto simp add: LV_def intro: Prf.intros elim: Prf_elims)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   927
274
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   928
lemma LV_NTIMES_3:
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   929
  shows "LV (NTIMES r (Suc n)) [] = (\<lambda>(v,vs). Stars (v#vs)) ` (LV r [] \<times> (Stars -` (LV (NTIMES r n) [])))"
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   930
unfolding LV_def
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   931
apply(auto elim!: Prf_elims simp add: image_def)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   932
apply(case_tac vs1)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   933
apply(auto)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   934
apply(case_tac vs2)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   935
apply(auto)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   936
apply(subst append.simps(1)[symmetric])
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   937
apply(rule Prf.intros)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   938
apply(auto)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   939
apply(subst append.simps(1)[symmetric])
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   940
apply(rule Prf.intros)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   941
apply(auto)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   942
  done 
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   943
    
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   944
lemma LV_FROMNTIMES_3:
a3134f7de065 updated
cu
parents: 275
diff changeset
   945
  shows "LV (FROMNTIMES r (Suc n)) [] = 
a3134f7de065 updated
cu
parents: 275
diff changeset
   946
    (\<lambda>(v,vs). Stars (v#vs)) ` (LV r [] \<times> (Stars -` (LV (FROMNTIMES r n) [])))"
a3134f7de065 updated
cu
parents: 275
diff changeset
   947
unfolding LV_def
a3134f7de065 updated
cu
parents: 275
diff changeset
   948
apply(auto elim!: Prf_elims simp add: image_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
   949
apply(case_tac vs1)
a3134f7de065 updated
cu
parents: 275
diff changeset
   950
apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
   951
apply(case_tac vs2)
a3134f7de065 updated
cu
parents: 275
diff changeset
   952
apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
   953
apply(subst append.simps(1)[symmetric])
a3134f7de065 updated
cu
parents: 275
diff changeset
   954
apply(rule Prf.intros)
a3134f7de065 updated
cu
parents: 275
diff changeset
   955
     apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
   956
  apply (metis le_imp_less_Suc length_greater_0_conv less_antisym list.exhaust list.set_intros(1) not_less_eq zero_le)
a3134f7de065 updated
cu
parents: 275
diff changeset
   957
  prefer 2
a3134f7de065 updated
cu
parents: 275
diff changeset
   958
  using nth_mem apply blast
a3134f7de065 updated
cu
parents: 275
diff changeset
   959
  apply(case_tac vs1)
a3134f7de065 updated
cu
parents: 275
diff changeset
   960
  apply (smt Groups.add_ac(2) Prf.intros(9) add.right_neutral add_Suc_right append.simps(1) insert_iff length_append list.set(2) list.size(3) list.size(4))
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
   961
    apply(auto)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   962
done     
a3134f7de065 updated
cu
parents: 275
diff changeset
   963
  
a3134f7de065 updated
cu
parents: 275
diff changeset
   964
lemma LV_NTIMES_4:
a3134f7de065 updated
cu
parents: 275
diff changeset
   965
 "LV (NTIMES r n) [] = Stars_Pow (LV r []) n" 
a3134f7de065 updated
cu
parents: 275
diff changeset
   966
  apply(induct n)
a3134f7de065 updated
cu
parents: 275
diff changeset
   967
   apply(simp add: LV_def)    
a3134f7de065 updated
cu
parents: 275
diff changeset
   968
   apply(auto elim!: Prf_elims simp add: image_def)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
   969
   apply(subst append.simps[symmetric])
a3134f7de065 updated
cu
parents: 275
diff changeset
   970
    apply(rule Prf.intros)
a3134f7de065 updated
cu
parents: 275
diff changeset
   971
      apply(simp_all)
a3134f7de065 updated
cu
parents: 275
diff changeset
   972
    apply(simp add: LV_NTIMES_3 image_def Stars_Cons_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
   973
  apply blast
a3134f7de065 updated
cu
parents: 275
diff changeset
   974
 done   
274
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
   975
276
a3134f7de065 updated
cu
parents: 275
diff changeset
   976
lemma LV_NTIMES_5:
a3134f7de065 updated
cu
parents: 275
diff changeset
   977
  "LV (NTIMES r n) s \<subseteq> Stars_Append (LV (STAR r) s) (\<Union>i\<le>n. LV (NTIMES r i) [])"
a3134f7de065 updated
cu
parents: 275
diff changeset
   978
apply(auto simp add: LV_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
   979
apply(auto elim!: Prf_elims)
a3134f7de065 updated
cu
parents: 275
diff changeset
   980
  apply(auto simp add: Stars_Append_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
   981
  apply(rule_tac x="vs1" in exI)
a3134f7de065 updated
cu
parents: 275
diff changeset
   982
  apply(rule_tac x="vs2" in exI)  
a3134f7de065 updated
cu
parents: 275
diff changeset
   983
  apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
   984
    using Prf.intros(6) apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
   985
      apply(rule_tac x="length vs2" in bexI)
a3134f7de065 updated
cu
parents: 275
diff changeset
   986
    thm Prf.intros
a3134f7de065 updated
cu
parents: 275
diff changeset
   987
      apply(subst append.simps(1)[symmetric])
a3134f7de065 updated
cu
parents: 275
diff changeset
   988
    apply(rule Prf.intros)
a3134f7de065 updated
cu
parents: 275
diff changeset
   989
      apply(auto)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
   990
      apply(auto)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
   991
     apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
   992
    apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
   993
      done
a3134f7de065 updated
cu
parents: 275
diff changeset
   994
      
a3134f7de065 updated
cu
parents: 275
diff changeset
   995
lemma ttty:
a3134f7de065 updated
cu
parents: 275
diff changeset
   996
 "LV (FROMNTIMES r n) [] = Stars_Pow (LV r []) n" 
a3134f7de065 updated
cu
parents: 275
diff changeset
   997
  apply(induct n)
a3134f7de065 updated
cu
parents: 275
diff changeset
   998
   apply(simp add: LV_def)    
a3134f7de065 updated
cu
parents: 275
diff changeset
   999
   apply(auto elim: Prf_elims simp add: image_def)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1000
   prefer 2
a3134f7de065 updated
cu
parents: 275
diff changeset
  1001
    apply(subst append.simps[symmetric])
a3134f7de065 updated
cu
parents: 275
diff changeset
  1002
    apply(rule Prf.intros)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1003
      apply(simp_all)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1004
   apply(erule Prf_elims) 
a3134f7de065 updated
cu
parents: 275
diff changeset
  1005
    apply(case_tac vs1)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1006
     apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1007
    apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1008
   apply(case_tac x)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1009
    apply(simp_all)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1010
    apply(simp add: LV_FROMNTIMES_3 image_def Stars_Cons_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1011
  apply blast
a3134f7de065 updated
cu
parents: 275
diff changeset
  1012
 done     
a3134f7de065 updated
cu
parents: 275
diff changeset
  1013
a3134f7de065 updated
cu
parents: 275
diff changeset
  1014
lemma LV_FROMNTIMES_5:
a3134f7de065 updated
cu
parents: 275
diff changeset
  1015
  "LV (FROMNTIMES r n) s \<subseteq> Stars_Append (LV (STAR r) s) (\<Union>i\<le>n. LV (FROMNTIMES r i) [])"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1016
apply(auto simp add: LV_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1017
apply(auto elim!: Prf_elims)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1018
  apply(auto simp add: Stars_Append_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1019
  apply(rule_tac x="vs1" in exI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1020
  apply(rule_tac x="vs2" in exI)  
a3134f7de065 updated
cu
parents: 275
diff changeset
  1021
  apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1022
    using Prf.intros(6) apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1023
      apply(rule_tac x="length vs2" in bexI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1024
    thm Prf.intros
a3134f7de065 updated
cu
parents: 275
diff changeset
  1025
      apply(subst append.simps(1)[symmetric])
a3134f7de065 updated
cu
parents: 275
diff changeset
  1026
    apply(rule Prf.intros)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1027
      apply(auto)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1028
      apply(auto)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1029
     apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1030
     apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1031
      apply(rule_tac x="vs" in exI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1032
    apply(rule_tac x="[]" in exI) 
a3134f7de065 updated
cu
parents: 275
diff changeset
  1033
    apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1034
    by (metis Prf.intros(9) append_Nil atMost_iff empty_iff le_imp_less_Suc less_antisym list.set(1) nth_mem zero_le)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1035
a3134f7de065 updated
cu
parents: 275
diff changeset
  1036
lemma LV_FROMNTIMES_6:
a3134f7de065 updated
cu
parents: 275
diff changeset
  1037
  assumes "\<forall>s. finite (LV r s)"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1038
  shows "finite (LV (FROMNTIMES r n) s)"
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
  1039
  apply(rule finite_subset)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1040
   apply(rule LV_FROMNTIMES_5)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1041
  apply(rule finite_Stars_Append)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1042
    apply(rule LV_STAR_finite)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1043
   apply(rule assms)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1044
  apply(rule finite_UN_I)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1045
   apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1046
  by (simp add: assms finite_Stars_Pow ttty)
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
  1047
    
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1048
lemma LV_NMTIMES_5:
a3134f7de065 updated
cu
parents: 275
diff changeset
  1049
  "LV (NMTIMES r n m) s \<subseteq> Stars_Append (LV (STAR r) s) (\<Union>i\<le>n. LV (FROMNTIMES r i) [])"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1050
apply(auto simp add: LV_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1051
apply(auto elim!: Prf_elims)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1052
  apply(auto simp add: Stars_Append_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1053
  apply(rule_tac x="vs1" in exI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1054
  apply(rule_tac x="vs2" in exI)  
a3134f7de065 updated
cu
parents: 275
diff changeset
  1055
  apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1056
    using Prf.intros(6) apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1057
      apply(rule_tac x="length vs2" in bexI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1058
    thm Prf.intros
a3134f7de065 updated
cu
parents: 275
diff changeset
  1059
      apply(subst append.simps(1)[symmetric])
a3134f7de065 updated
cu
parents: 275
diff changeset
  1060
    apply(rule Prf.intros)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1061
      apply(auto)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1062
      apply(auto)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1063
     apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1064
     apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1065
      apply(rule_tac x="vs" in exI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1066
    apply(rule_tac x="[]" in exI) 
a3134f7de065 updated
cu
parents: 275
diff changeset
  1067
    apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1068
    by (metis Prf.intros(9) append_Nil atMost_iff empty_iff le_imp_less_Suc less_antisym list.set(1) nth_mem zero_le)
274
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
  1069
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1070
lemma LV_NMTIMES_6:
a3134f7de065 updated
cu
parents: 275
diff changeset
  1071
  assumes "\<forall>s. finite (LV r s)"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1072
  shows "finite (LV (NMTIMES r n m) s)"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1073
  apply(rule finite_subset)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1074
   apply(rule LV_NMTIMES_5)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1075
  apply(rule finite_Stars_Append)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1076
    apply(rule LV_STAR_finite)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1077
   apply(rule assms)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1078
  apply(rule finite_UN_I)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1079
   apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1080
  by (simp add: assms finite_Stars_Pow ttty)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1081
        
a3134f7de065 updated
cu
parents: 275
diff changeset
  1082
    
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1083
lemma LV_finite:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1084
  shows "finite (LV r s)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1085
proof(induct r arbitrary: s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1086
  case (ZERO s) 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1087
  show "finite (LV ZERO s)" by (simp add: LV_simps)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1088
next
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1089
  case (ONE s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1090
  show "finite (LV ONE s)" by (simp add: LV_simps)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1091
next
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1092
  case (CHAR c s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1093
  show "finite (LV (CHAR c) s)" by (simp add: LV_simps)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1094
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1095
  case (ALT r1 r2 s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1096
  then show "finite (LV (ALT r1 r2) s)" by (simp add: LV_simps)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1097
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1098
  case (SEQ r1 r2 s)
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
  1099
  define f where "f \<equiv> \<lambda>(v1, v2). Seq v1 v2"
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
  1100
  define S1 where "S1 \<equiv> \<Union>s' \<in> Prefixes s. LV r1 s'"
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
  1101
  define S2 where "S2 \<equiv> \<Union>s' \<in> Suffixes s. LV r2 s'"
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1102
  have IHs: "\<And>s. finite (LV r1 s)" "\<And>s. finite (LV r2 s)" by fact+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1103
  then have "finite S1" "finite S2" unfolding S1_def S2_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1104
    by (simp_all add: finite_Prefixes finite_Suffixes)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1105
  moreover
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1106
  have "LV (SEQ r1 r2) s \<subseteq> f ` (S1 \<times> S2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1107
    unfolding f_def S1_def S2_def 
275
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
  1108
    unfolding LV_def image_def prefix_def suffix_def
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
  1109
    apply (auto elim!: Prf_elims)
deea42c83c9e updated
Christian Urban <urbanc@in.tum.de>
parents: 274
diff changeset
  1110
    by (metis (mono_tags, lifting) mem_Collect_eq)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1111
  ultimately 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1112
  show "finite (LV (SEQ r1 r2) s)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1113
    by (simp add: finite_subset)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1114
next
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1115
  case (STAR r s)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1116
  then show "finite (LV (STAR r) s)" by (simp add: LV_STAR_finite)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1117
next 
274
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
  1118
  case (UPNTIMES r n s)
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1119
  have "\<And>s. finite (LV r s)" by fact
274
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
  1120
  then show "finite (LV (UPNTIMES r n) s)"
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
  1121
  by (meson LV_STAR_finite LV_UPNTIMES_STAR rev_finite_subset)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
  1122
next 
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
  1123
  case (FROMNTIMES r n s)
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
  1124
  have "\<And>s. finite (LV r s)" by fact
692b62426677 updated
Christian Urban <urbanc@in.tum.de>
parents: 273
diff changeset
  1125
  then show "finite (LV (FROMNTIMES r n) s)"
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1126
    by (simp add: LV_FROMNTIMES_6)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1127
next 
a3134f7de065 updated
cu
parents: 275
diff changeset
  1128
  case (NTIMES r n s)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1129
  have "\<And>s. finite (LV r s)" by fact
a3134f7de065 updated
cu
parents: 275
diff changeset
  1130
  then show "finite (LV (NTIMES r n) s)"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1131
    by (metis (no_types, lifting) LV_NTIMES_4 LV_NTIMES_5 LV_STAR_finite finite_Stars_Append finite_Stars_Pow finite_UN_I finite_atMost finite_subset)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1132
next
a3134f7de065 updated
cu
parents: 275
diff changeset
  1133
  case (NMTIMES r n m s)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1134
  have "\<And>s. finite (LV r s)" by fact
a3134f7de065 updated
cu
parents: 275
diff changeset
  1135
  then show "finite (LV (NMTIMES r n m) s)"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1136
    by (simp add: LV_NMTIMES_6)         
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1137
qed
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1138
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1139
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1140
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1141
section {* Our POSIX Definition *}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1142
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1143
inductive 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1144
  Posix :: "string \<Rightarrow> rexp \<Rightarrow> val \<Rightarrow> bool" ("_ \<in> _ \<rightarrow> _" [100, 100, 100] 100)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1145
where
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1146
  Posix_ONE: "[] \<in> ONE \<rightarrow> Void"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1147
| Posix_CHAR: "[c] \<in> (CHAR c) \<rightarrow> (Char c)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1148
| Posix_ALT1: "s \<in> r1 \<rightarrow> v \<Longrightarrow> s \<in> (ALT r1 r2) \<rightarrow> (Left v)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1149
| Posix_ALT2: "\<lbrakk>s \<in> r2 \<rightarrow> v; s \<notin> L(r1)\<rbrakk> \<Longrightarrow> s \<in> (ALT r1 r2) \<rightarrow> (Right v)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1150
| Posix_SEQ: "\<lbrakk>s1 \<in> r1 \<rightarrow> v1; s2 \<in> r2 \<rightarrow> v2;
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1151
    \<not>(\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> (s1 @ s\<^sub>3) \<in> L r1 \<and> s\<^sub>4 \<in> L r2)\<rbrakk> \<Longrightarrow> 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1152
    (s1 @ s2) \<in> (SEQ r1 r2) \<rightarrow> (Seq v1 v2)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1153
| Posix_STAR1: "\<lbrakk>s1 \<in> r \<rightarrow> v; s2 \<in> STAR r \<rightarrow> Stars vs; flat v \<noteq> [];
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1154
    \<not>(\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> (s1 @ s\<^sub>3) \<in> L r \<and> s\<^sub>4 \<in> L (STAR r))\<rbrakk>
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1155
    \<Longrightarrow> (s1 @ s2) \<in> STAR r \<rightarrow> Stars (v # vs)"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1156
| Posix_STAR2: "[] \<in> STAR r \<rightarrow> Stars []"
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1157
| Posix_NTIMES1: "\<lbrakk>s1 \<in> r \<rightarrow> v; s2 \<in> NTIMES r (n - 1) \<rightarrow> Stars vs; flat v \<noteq> []; 0 < n;
a3134f7de065 updated
cu
parents: 275
diff changeset
  1158
    \<not>(\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> (s1 @ s\<^sub>3) \<in> L r \<and> s\<^sub>4 \<in> L (NTIMES r (n - 1)))\<rbrakk>
a3134f7de065 updated
cu
parents: 275
diff changeset
  1159
    \<Longrightarrow> (s1 @ s2) \<in> NTIMES r n \<rightarrow> Stars (v # vs)"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1160
| Posix_NTIMES2: "\<lbrakk>\<forall>v \<in> set vs. [] \<in> r \<rightarrow> v; length vs = n\<rbrakk>
a3134f7de065 updated
cu
parents: 275
diff changeset
  1161
    \<Longrightarrow> [] \<in> NTIMES r n \<rightarrow> Stars vs"  
a3134f7de065 updated
cu
parents: 275
diff changeset
  1162
| Posix_UPNTIMES1: "\<lbrakk>s1 \<in> r \<rightarrow> v; s2 \<in> UPNTIMES r (n - 1) \<rightarrow> Stars vs; flat v \<noteq> []; 0 < n;
a3134f7de065 updated
cu
parents: 275
diff changeset
  1163
    \<not>(\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> (s1 @ s\<^sub>3) \<in> L r \<and> s\<^sub>4 \<in> L (UPNTIMES r (n - 1)))\<rbrakk>
a3134f7de065 updated
cu
parents: 275
diff changeset
  1164
    \<Longrightarrow> (s1 @ s2) \<in> UPNTIMES r n \<rightarrow> Stars (v # vs)"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1165
| Posix_UPNTIMES2: "[] \<in> UPNTIMES r n \<rightarrow> Stars []"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1166
| Posix_FROMNTIMES2: "\<lbrakk>\<forall>v \<in> set vs. [] \<in> r \<rightarrow> v; length vs = n\<rbrakk>
a3134f7de065 updated
cu
parents: 275
diff changeset
  1167
    \<Longrightarrow> [] \<in> FROMNTIMES r n \<rightarrow> Stars vs"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1168
| Posix_FROMNTIMES1: "\<lbrakk>s1 \<in> r \<rightarrow> v; s2 \<in> FROMNTIMES r (n - 1) \<rightarrow> Stars vs; flat v \<noteq> []; 0 < n;
a3134f7de065 updated
cu
parents: 275
diff changeset
  1169
    \<not>(\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> (s1 @ s\<^sub>3) \<in> L r \<and> s\<^sub>4 \<in> L (FROMNTIMES r (n - 1)))\<rbrakk>
a3134f7de065 updated
cu
parents: 275
diff changeset
  1170
    \<Longrightarrow> (s1 @ s2) \<in> FROMNTIMES r n \<rightarrow> Stars (v # vs)"  
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1171
| Posix_FROMNTIMES3: "\<lbrakk>s1 \<in> r \<rightarrow> v; s2 \<in> STAR r \<rightarrow> Stars vs; flat v \<noteq> [];
42268a284ea6 updated
cu
parents: 276
diff changeset
  1172
    \<not>(\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> (s1 @ s\<^sub>3) \<in> L r \<and> s\<^sub>4 \<in> L (STAR r))\<rbrakk>
42268a284ea6 updated
cu
parents: 276
diff changeset
  1173
    \<Longrightarrow> (s1 @ s2) \<in> FROMNTIMES r 0 \<rightarrow> Stars (v # vs)"  
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1174
| Posix_NMTIMES2: "\<lbrakk>\<forall>v \<in> set vs. [] \<in> r \<rightarrow> v; length vs = n; n \<le> m\<rbrakk>
a3134f7de065 updated
cu
parents: 275
diff changeset
  1175
    \<Longrightarrow> [] \<in> NMTIMES r n m \<rightarrow> Stars vs"  
278
424bdcd01016 updated
cu
parents: 277
diff changeset
  1176
| Posix_NMTIMES1: "\<lbrakk>s1 \<in> r \<rightarrow> v; s2 \<in> NMTIMES r (n - 1) (m - 1) \<rightarrow> Stars vs; flat v \<noteq> []; 0 < n; n \<le> m;
424bdcd01016 updated
cu
parents: 277
diff changeset
  1177
    \<not>(\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> (s1 @ s\<^sub>3) \<in> L r \<and> s\<^sub>4 \<in> L (NMTIMES r (n - 1) (m - 1)))\<rbrakk>
424bdcd01016 updated
cu
parents: 277
diff changeset
  1178
    \<Longrightarrow> (s1 @ s2) \<in> NMTIMES r n m \<rightarrow> Stars (v # vs)"  
424bdcd01016 updated
cu
parents: 277
diff changeset
  1179
| Posix_NMTIMES3: "\<lbrakk>s1 \<in> r \<rightarrow> v; s2 \<in> UPNTIMES r (m - 1) \<rightarrow> Stars vs; flat v \<noteq> []; 0 < m;
424bdcd01016 updated
cu
parents: 277
diff changeset
  1180
    \<not>(\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> (s1 @ s\<^sub>3) \<in> L r \<and> s\<^sub>4 \<in> L (UPNTIMES r (m - 1)))\<rbrakk>
424bdcd01016 updated
cu
parents: 277
diff changeset
  1181
    \<Longrightarrow> (s1 @ s2) \<in> NMTIMES r 0 m \<rightarrow> Stars (v # vs)"    
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1182
  
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1183
inductive_cases Posix_elims:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1184
  "s \<in> ZERO \<rightarrow> v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1185
  "s \<in> ONE \<rightarrow> v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1186
  "s \<in> CHAR c \<rightarrow> v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1187
  "s \<in> ALT r1 r2 \<rightarrow> v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1188
  "s \<in> SEQ r1 r2 \<rightarrow> v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1189
  "s \<in> STAR r \<rightarrow> v"
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1190
  "s \<in> NTIMES r n \<rightarrow> v"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1191
  "s \<in> UPNTIMES r n \<rightarrow> v"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1192
  "s \<in> FROMNTIMES r n \<rightarrow> v"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1193
  "s \<in> NMTIMES r n m \<rightarrow> v"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1194
  
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1195
lemma Posix1:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1196
  assumes "s \<in> r \<rightarrow> v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1197
  shows "s \<in> L r" "flat v = s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1198
using assms
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1199
  apply(induct s r v rule: Posix.induct)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1200
                    apply(auto simp add: Sequ_def)[18]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1201
            apply(case_tac n)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1202
             apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1203
  apply(simp add: Sequ_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1204
            apply(auto)[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1205
           apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1206
  apply(clarify)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1207
  apply(rule_tac x="Suc x" in bexI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1208
  apply(simp add: Sequ_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1209
            apply(auto)[5]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1210
  using nth_mem nullable.simps(9) nullable_correctness apply auto[1]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1211
  apply simp
a3134f7de065 updated
cu
parents: 275
diff changeset
  1212
       apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1213
       apply(clarify)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1214
       apply(rule_tac x="Suc x" in bexI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1215
        apply(simp add: Sequ_def)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1216
          apply(auto)[3]
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1217
    defer
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1218
     apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1219
  apply fastforce
a3134f7de065 updated
cu
parents: 275
diff changeset
  1220
    apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1221
   apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1222
    apply(clarify)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1223
   apply(rule_tac x="Suc x" in bexI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1224
    apply(auto simp add: Sequ_def)[2]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1225
   apply(simp)
278
424bdcd01016 updated
cu
parents: 277
diff changeset
  1226
    apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1227
    apply(clarify)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1228
     apply(rule_tac x="Suc x" in bexI)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1229
    apply(auto simp add: Sequ_def)[2]
424bdcd01016 updated
cu
parents: 277
diff changeset
  1230
   apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1231
  apply(simp add: Star.step Star_Pow)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1232
done  
424bdcd01016 updated
cu
parents: 277
diff changeset
  1233
    
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1234
text {*
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1235
  Our Posix definition determines a unique value.
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1236
*}
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1237
  
a3134f7de065 updated
cu
parents: 275
diff changeset
  1238
lemma List_eq_zipI:
a3134f7de065 updated
cu
parents: 275
diff changeset
  1239
  assumes "\<forall>(v1, v2) \<in> set (zip vs1 vs2). v1 = v2" 
a3134f7de065 updated
cu
parents: 275
diff changeset
  1240
  and "length vs1 = length vs2"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1241
  shows "vs1 = vs2"  
a3134f7de065 updated
cu
parents: 275
diff changeset
  1242
 using assms
a3134f7de065 updated
cu
parents: 275
diff changeset
  1243
  apply(induct vs1 arbitrary: vs2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1244
   apply(case_tac vs2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1245
   apply(simp)    
a3134f7de065 updated
cu
parents: 275
diff changeset
  1246
   apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1247
   apply(case_tac vs2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1248
   apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1249
  apply(simp)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1250
done    
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1251
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1252
lemma Posix_determ:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1253
  assumes "s \<in> r \<rightarrow> v1" "s \<in> r \<rightarrow> v2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1254
  shows "v1 = v2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1255
using assms
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1256
proof (induct s r v1 arbitrary: v2 rule: Posix.induct)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1257
  case (Posix_ONE v2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1258
  have "[] \<in> ONE \<rightarrow> v2" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1259
  then show "Void = v2" by cases auto
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1260
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1261
  case (Posix_CHAR c v2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1262
  have "[c] \<in> CHAR c \<rightarrow> v2" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1263
  then show "Char c = v2" by cases auto
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1264
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1265
  case (Posix_ALT1 s r1 v r2 v2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1266
  have "s \<in> ALT r1 r2 \<rightarrow> v2" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1267
  moreover
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1268
  have "s \<in> r1 \<rightarrow> v" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1269
  then have "s \<in> L r1" by (simp add: Posix1)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1270
  ultimately obtain v' where eq: "v2 = Left v'" "s \<in> r1 \<rightarrow> v'" by cases auto 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1271
  moreover
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1272
  have IH: "\<And>v2. s \<in> r1 \<rightarrow> v2 \<Longrightarrow> v = v2" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1273
  ultimately have "v = v'" by simp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1274
  then show "Left v = v2" using eq by simp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1275
next 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1276
  case (Posix_ALT2 s r2 v r1 v2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1277
  have "s \<in> ALT r1 r2 \<rightarrow> v2" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1278
  moreover
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1279
  have "s \<notin> L r1" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1280
  ultimately obtain v' where eq: "v2 = Right v'" "s \<in> r2 \<rightarrow> v'" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1281
    by cases (auto simp add: Posix1) 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1282
  moreover
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1283
  have IH: "\<And>v2. s \<in> r2 \<rightarrow> v2 \<Longrightarrow> v = v2" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1284
  ultimately have "v = v'" by simp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1285
  then show "Right v = v2" using eq by simp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1286
next
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1287
  case (Posix_SEQ s1 r1 v1 s2 r2 v2 v')
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1288
  have "(s1 @ s2) \<in> SEQ r1 r2 \<rightarrow> v'" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1289
       "s1 \<in> r1 \<rightarrow> v1" "s2 \<in> r2 \<rightarrow> v2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1290
       "\<not> (\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> s1 @ s\<^sub>3 \<in> L r1 \<and> s\<^sub>4 \<in> L r2)" by fact+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1291
  then obtain v1' v2' where "v' = Seq v1' v2'" "s1 \<in> r1 \<rightarrow> v1'" "s2 \<in> r2 \<rightarrow> v2'"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1292
  apply(cases) apply (auto simp add: append_eq_append_conv2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1293
  using Posix1(1) by fastforce+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1294
  moreover
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1295
  have IHs: "\<And>v1'. s1 \<in> r1 \<rightarrow> v1' \<Longrightarrow> v1 = v1'"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1296
            "\<And>v2'. s2 \<in> r2 \<rightarrow> v2' \<Longrightarrow> v2 = v2'" by fact+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1297
  ultimately show "Seq v1 v2 = v'" by simp
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1298
next
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1299
  case (Posix_STAR1 s1 r v s2 vs v2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1300
  have "(s1 @ s2) \<in> STAR r \<rightarrow> v2" 
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1301
       "s1 \<in> r \<rightarrow> v" "s2 \<in> STAR r \<rightarrow> Stars vs" "flat v \<noteq> []"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1302
       "\<not> (\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> s1 @ s\<^sub>3 \<in> L r \<and> s\<^sub>4 \<in> L (STAR r))" by fact+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1303
  then obtain v' vs' where "v2 = Stars (v' # vs')" "s1 \<in> r \<rightarrow> v'" "s2 \<in> (STAR r) \<rightarrow> (Stars vs')"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1304
  apply(cases) apply (auto simp add: append_eq_append_conv2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1305
  using Posix1(1) apply fastforce
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1306
  apply (metis Posix1(1) Posix_STAR1.hyps(6) append_Nil append_Nil2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1307
  using Posix1(2) by blast
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1308
  moreover
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1309
  have IHs: "\<And>v2. s1 \<in> r \<rightarrow> v2 \<Longrightarrow> v = v2"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1310
            "\<And>v2. s2 \<in> STAR r \<rightarrow> v2 \<Longrightarrow> Stars vs = v2" by fact+
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1311
  ultimately show "Stars (v # vs) = v2" by auto
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1312
next
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1313
  case (Posix_STAR2 r v2)
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1314
  have "[] \<in> STAR r \<rightarrow> v2" by fact
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1315
  then show "Stars [] = v2" by cases (auto simp add: Posix1)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1316
next
a3134f7de065 updated
cu
parents: 275
diff changeset
  1317
  case (Posix_NTIMES2 vs r n v2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1318
  then show "Stars vs = v2"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1319
    apply(erule_tac Posix_elims)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1320
     apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1321
     apply (simp add: Posix1(2))
a3134f7de065 updated
cu
parents: 275
diff changeset
  1322
    apply(rule List_eq_zipI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1323
     apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1324
    by (meson in_set_zipE)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1325
next
a3134f7de065 updated
cu
parents: 275
diff changeset
  1326
  case (Posix_NTIMES1 s1 r v s2 n vs v2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1327
  have "(s1 @ s2) \<in> NTIMES r n \<rightarrow> v2" 
a3134f7de065 updated
cu
parents: 275
diff changeset
  1328
       "s1 \<in> r \<rightarrow> v" "s2 \<in> NTIMES r (n - 1) \<rightarrow> Stars vs" "flat v \<noteq> []"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1329
       "\<not> (\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> s1 @ s\<^sub>3 \<in> L r \<and> s\<^sub>4 \<in> L (NTIMES r (n - 1 )))" by fact+
a3134f7de065 updated
cu
parents: 275
diff changeset
  1330
  then obtain v' vs' where "v2 = Stars (v' # vs')" "s1 \<in> r \<rightarrow> v'" "s2 \<in> (NTIMES r (n - 1)) \<rightarrow> (Stars vs')"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1331
  apply(cases) apply (auto simp add: append_eq_append_conv2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1332
    using Posix1(1) apply fastforce
a3134f7de065 updated
cu
parents: 275
diff changeset
  1333
    apply (metis One_nat_def Posix1(1) Posix_NTIMES1.hyps(7) append.right_neutral append_self_conv2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1334
  using Posix1(2) by blast
a3134f7de065 updated
cu
parents: 275
diff changeset
  1335
  moreover
a3134f7de065 updated
cu
parents: 275
diff changeset
  1336
  have IHs: "\<And>v2. s1 \<in> r \<rightarrow> v2 \<Longrightarrow> v = v2"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1337
            "\<And>v2. s2 \<in> NTIMES r (n - 1) \<rightarrow> v2 \<Longrightarrow> Stars vs = v2" by fact+
a3134f7de065 updated
cu
parents: 275
diff changeset
  1338
  ultimately show "Stars (v # vs) = v2" by auto
a3134f7de065 updated
cu
parents: 275
diff changeset
  1339
next
a3134f7de065 updated
cu
parents: 275
diff changeset
  1340
  case (Posix_UPNTIMES1 s1 r v s2 n vs v2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1341
  have "(s1 @ s2) \<in> UPNTIMES r n \<rightarrow> v2" 
a3134f7de065 updated
cu
parents: 275
diff changeset
  1342
       "s1 \<in> r \<rightarrow> v" "s2 \<in> UPNTIMES r (n - 1) \<rightarrow> Stars vs" "flat v \<noteq> []"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1343
       "\<not> (\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> s1 @ s\<^sub>3 \<in> L r \<and> s\<^sub>4 \<in> L (UPNTIMES r (n - 1 )))" by fact+
a3134f7de065 updated
cu
parents: 275
diff changeset
  1344
  then obtain v' vs' where "v2 = Stars (v' # vs')" "s1 \<in> r \<rightarrow> v'" "s2 \<in> (UPNTIMES r (n - 1)) \<rightarrow> (Stars vs')"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1345
  apply(cases) apply (auto simp add: append_eq_append_conv2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1346
    using Posix1(1) apply fastforce
a3134f7de065 updated
cu
parents: 275
diff changeset
  1347
    apply (metis One_nat_def Posix1(1) Posix_UPNTIMES1.hyps(7) append.right_neutral append_self_conv2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1348
  using Posix1(2) by blast
a3134f7de065 updated
cu
parents: 275
diff changeset
  1349
  moreover
a3134f7de065 updated
cu
parents: 275
diff changeset
  1350
  have IHs: "\<And>v2. s1 \<in> r \<rightarrow> v2 \<Longrightarrow> v = v2"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1351
            "\<And>v2. s2 \<in> UPNTIMES r (n - 1) \<rightarrow> v2 \<Longrightarrow> Stars vs = v2" by fact+
a3134f7de065 updated
cu
parents: 275
diff changeset
  1352
  ultimately show "Stars (v # vs) = v2" by auto
a3134f7de065 updated
cu
parents: 275
diff changeset
  1353
next
a3134f7de065 updated
cu
parents: 275
diff changeset
  1354
  case (Posix_UPNTIMES2 r n v2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1355
  then show "Stars [] = v2"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1356
    apply(erule_tac Posix_elims)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1357
     apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1358
    by (simp add: Posix1(2))
a3134f7de065 updated
cu
parents: 275
diff changeset
  1359
next
a3134f7de065 updated
cu
parents: 275
diff changeset
  1360
  case (Posix_FROMNTIMES1 s1 r v s2 n vs v2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1361
  have "(s1 @ s2) \<in> FROMNTIMES r n \<rightarrow> v2" 
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1362
       "s1 \<in> r \<rightarrow> v" "s2 \<in> FROMNTIMES r (n - 1) \<rightarrow> Stars vs" "flat v \<noteq> []" "0 < n"
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1363
       "\<not> (\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> s1 @ s\<^sub>3 \<in> L r \<and> s\<^sub>4 \<in> L (FROMNTIMES r (n - 1 )))" by fact+
a3134f7de065 updated
cu
parents: 275
diff changeset
  1364
  then obtain v' vs' where "v2 = Stars (v' # vs')" "s1 \<in> r \<rightarrow> v'" "s2 \<in> (FROMNTIMES r (n - 1)) \<rightarrow> (Stars vs')"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1365
  apply(cases) apply (auto simp add: append_eq_append_conv2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1366
    using Posix1(1) Posix1(2) apply blast 
a3134f7de065 updated
cu
parents: 275
diff changeset
  1367
     apply(case_tac n)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1368
      apply(simp)
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1369
      apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1370
    apply(drule_tac x="va" in meta_spec)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1371
    apply(drule_tac x="vs" in meta_spec)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1372
    apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1373
     apply(drule meta_mp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1374
    apply (metis L.simps(9) Posix1(1) UN_E append.right_neutral append_Nil diff_Suc_1 local.Posix_FROMNTIMES1(4) val.inject(5))
42268a284ea6 updated
cu
parents: 276
diff changeset
  1375
    apply (metis L.simps(9) Posix1(1) UN_E append.right_neutral append_Nil)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1376
    by (metis One_nat_def Posix1(1) Posix_FROMNTIMES1.hyps(7) self_append_conv self_append_conv2)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1377
  moreover
a3134f7de065 updated
cu
parents: 275
diff changeset
  1378
  have IHs: "\<And>v2. s1 \<in> r \<rightarrow> v2 \<Longrightarrow> v = v2"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1379
            "\<And>v2. s2 \<in> FROMNTIMES r (n - 1) \<rightarrow> v2 \<Longrightarrow> Stars vs = v2" by fact+
a3134f7de065 updated
cu
parents: 275
diff changeset
  1380
  ultimately show "Stars (v # vs) = v2" by auto    
a3134f7de065 updated
cu
parents: 275
diff changeset
  1381
next
a3134f7de065 updated
cu
parents: 275
diff changeset
  1382
  case (Posix_FROMNTIMES2 vs r n v2)  
a3134f7de065 updated
cu
parents: 275
diff changeset
  1383
  then show "Stars vs = v2"
a3134f7de065 updated
cu
parents: 275
diff changeset
  1384
    apply(erule_tac Posix_elims)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1385
     apply(auto)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1386
    apply(rule List_eq_zipI)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1387
     apply(auto)
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1388
      apply(meson in_set_zipE)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1389
     apply (simp add: Posix1(2))
42268a284ea6 updated
cu
parents: 276
diff changeset
  1390
    using Posix1(2) by blast
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1391
next
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1392
  case (Posix_FROMNTIMES3 s1 r v s2 vs v2)  
42268a284ea6 updated
cu
parents: 276
diff changeset
  1393
    have "(s1 @ s2) \<in> FROMNTIMES r 0 \<rightarrow> v2" 
42268a284ea6 updated
cu
parents: 276
diff changeset
  1394
       "s1 \<in> r \<rightarrow> v" "s2 \<in> STAR r \<rightarrow> Stars vs" "flat v \<noteq> []"
42268a284ea6 updated
cu
parents: 276
diff changeset
  1395
       "\<not> (\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> s1 @ s\<^sub>3 \<in> L r \<and> s\<^sub>4 \<in> L (STAR r))" by fact+
42268a284ea6 updated
cu
parents: 276
diff changeset
  1396
  then obtain v' vs' where "v2 = Stars (v' # vs')" "s1 \<in> r \<rightarrow> v'" "s2 \<in> (STAR r) \<rightarrow> (Stars vs')"
42268a284ea6 updated
cu
parents: 276
diff changeset
  1397
  apply(cases) apply (auto simp add: append_eq_append_conv2)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1398
    using Posix1(2) apply fastforce
42268a284ea6 updated
cu
parents: 276
diff changeset
  1399
    using Posix1(1) apply fastforce
42268a284ea6 updated
cu
parents: 276
diff changeset
  1400
    by (metis Posix1(1) Posix_FROMNTIMES3.hyps(6) append.right_neutral append_Nil)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1401
  moreover
42268a284ea6 updated
cu
parents: 276
diff changeset
  1402
  have IHs: "\<And>v2. s1 \<in> r \<rightarrow> v2 \<Longrightarrow> v = v2"
42268a284ea6 updated
cu
parents: 276
diff changeset
  1403
            "\<And>v2. s2 \<in> STAR r \<rightarrow> v2 \<Longrightarrow> Stars vs = v2" by fact+
42268a284ea6 updated
cu
parents: 276
diff changeset
  1404
  ultimately show "Stars (v # vs) = v2" by auto     
42268a284ea6 updated
cu
parents: 276
diff changeset
  1405
next    
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1406
  case (Posix_NMTIMES1 s1 r v s2 n m vs v2)
278
424bdcd01016 updated
cu
parents: 277
diff changeset
  1407
  have "(s1 @ s2) \<in> NMTIMES r n m \<rightarrow> v2" 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1408
       "s1 \<in> r \<rightarrow> v" "s2 \<in> NMTIMES r (n - 1) (m - 1) \<rightarrow> Stars vs" "flat v \<noteq> []" 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1409
       "0 < n" "n \<le> m"
424bdcd01016 updated
cu
parents: 277
diff changeset
  1410
       "\<not> (\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> s1 @ s\<^sub>3 \<in> L r \<and> s\<^sub>4 \<in> L (NMTIMES r (n - 1) (m - 1)))" by fact+
424bdcd01016 updated
cu
parents: 277
diff changeset
  1411
  then obtain v' vs' where "v2 = Stars (v' # vs')" "s1 \<in> r \<rightarrow> v'" 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1412
    "s2 \<in> (NMTIMES r (n - 1) (m - 1)) \<rightarrow> (Stars vs')"
424bdcd01016 updated
cu
parents: 277
diff changeset
  1413
  apply(cases) apply (auto simp add: append_eq_append_conv2)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1414
    using Posix1(1) Posix1(2) apply blast 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1415
     apply(case_tac n)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1416
      apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1417
     apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1418
       apply(case_tac m)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1419
      apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1420
     apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1421
    apply(drule_tac x="va" in meta_spec)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1422
    apply(drule_tac x="vs" in meta_spec)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1423
    apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1424
     apply(drule meta_mp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1425
      apply (smt L.simps(10) Posix1(1) Posix1(2) Posix_NMTIMES1.hyps(4) UN_E append.right_neutral
424bdcd01016 updated
cu
parents: 277
diff changeset
  1426
             append_eq_append_conv2 diff_Suc_1 val.inject(5))
424bdcd01016 updated
cu
parents: 277
diff changeset
  1427
     apply (metis L.simps(10) Posix1(1) UN_E append_Nil2 append_self_conv2)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1428
    by (metis One_nat_def Posix1(1) Posix_NMTIMES1.hyps(8) append.right_neutral append_Nil)      
424bdcd01016 updated
cu
parents: 277
diff changeset
  1429
  moreover
424bdcd01016 updated
cu
parents: 277
diff changeset
  1430
  have IHs: "\<And>v2. s1 \<in> r \<rightarrow> v2 \<Longrightarrow> v = v2"
424bdcd01016 updated
cu
parents: 277
diff changeset
  1431
            "\<And>v2. s2 \<in> NMTIMES r (n - 1) (m - 1) \<rightarrow> v2 \<Longrightarrow> Stars vs = v2" by fact+
424bdcd01016 updated
cu
parents: 277
diff changeset
  1432
  ultimately show "Stars (v # vs) = v2" by auto     
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1433
next
a3134f7de065 updated
cu
parents: 275
diff changeset
  1434
  case (Posix_NMTIMES2 vs r n m v2)
a3134f7de065 updated
cu
parents: 275
diff changeset
  1435
  then show "Stars vs = v2"
278
424bdcd01016 updated
cu
parents: 277
diff changeset
  1436
    apply(erule_tac Posix_elims)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1437
      apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1438
      apply(rule List_eq_zipI)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1439
       apply(auto)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1440
      apply (meson in_set_zipE)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1441
    apply (simp add: Posix1(2))
424bdcd01016 updated
cu
parents: 277
diff changeset
  1442
    apply(erule_tac Posix_elims)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1443
     apply(auto)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1444
    apply (simp add: Posix1(2))+
424bdcd01016 updated
cu
parents: 277
diff changeset
  1445
    done  
424bdcd01016 updated
cu
parents: 277
diff changeset
  1446
next
424bdcd01016 updated
cu
parents: 277
diff changeset
  1447
  case (Posix_NMTIMES3 s1 r v s2 m vs v2)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1448
   have "(s1 @ s2) \<in> NMTIMES r 0 m \<rightarrow> v2" 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1449
       "s1 \<in> r \<rightarrow> v" "s2 \<in> UPNTIMES r (m - 1) \<rightarrow> Stars vs" "flat v \<noteq> []" "0 < m"
424bdcd01016 updated
cu
parents: 277
diff changeset
  1450
       "\<not> (\<exists>s\<^sub>3 s\<^sub>4. s\<^sub>3 \<noteq> [] \<and> s\<^sub>3 @ s\<^sub>4 = s2 \<and> s1 @ s\<^sub>3 \<in> L r \<and> s\<^sub>4 \<in> L (UPNTIMES r (m - 1 )))" by fact+
424bdcd01016 updated
cu
parents: 277
diff changeset
  1451
  then obtain v' vs' where "v2 = Stars (v' # vs')" "s1 \<in> r \<rightarrow> v'" "s2 \<in> (UPNTIMES r (m - 1)) \<rightarrow> (Stars vs')"
424bdcd01016 updated
cu
parents: 277
diff changeset
  1452
    apply(cases) apply (auto simp add: append_eq_append_conv2)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1453
    using Posix1(2) apply blast
424bdcd01016 updated
cu
parents: 277
diff changeset
  1454
    apply (smt L.simps(7) Posix1(1) UN_E append_eq_append_conv2)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1455
    by (metis One_nat_def Posix1(1) Posix_NMTIMES3.hyps(7) append.right_neutral append_Nil)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1456
  moreover
424bdcd01016 updated
cu
parents: 277
diff changeset
  1457
  have IHs: "\<And>v2. s1 \<in> r \<rightarrow> v2 \<Longrightarrow> v = v2"
424bdcd01016 updated
cu
parents: 277
diff changeset
  1458
            "\<And>v2. s2 \<in> UPNTIMES r (m - 1) \<rightarrow> v2 \<Longrightarrow> Stars vs = v2" by fact+
424bdcd01016 updated
cu
parents: 277
diff changeset
  1459
  ultimately show "Stars (v # vs) = v2" by auto  
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1460
qed
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1461
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1462
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1463
text {*
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1464
  Our POSIX value is a lexical value.
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1465
*}
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1466
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1467
lemma Posix_LV:
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1468
  assumes "s \<in> r \<rightarrow> v"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1469
  shows "v \<in> LV r s"
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1470
using assms unfolding LV_def
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1471
apply(induct rule: Posix.induct)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1472
            apply(auto simp add: intro!: Prf.intros elim!: Prf_elims)[7]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1473
     defer
a3134f7de065 updated
cu
parents: 275
diff changeset
  1474
  defer
a3134f7de065 updated
cu
parents: 275
diff changeset
  1475
     apply(auto simp add: intro!: Prf.intros elim!: Prf_elims)[2]
a3134f7de065 updated
cu
parents: 275
diff changeset
  1476
  apply (metis (mono_tags, lifting) Prf.intros(9) append_Nil empty_iff flat_Stars flats_empty list.set(1) mem_Collect_eq)
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1477
     apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1478
     apply(clarify)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1479
     apply(case_tac n)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1480
      apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1481
     apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1482
     apply(erule Prf_elims)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1483
      apply(simp)
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1484
  apply(subst append.simps(2)[symmetric])
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1485
      apply(rule Prf.intros) 
42268a284ea6 updated
cu
parents: 276
diff changeset
  1486
        apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1487
       apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1488
      apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1489
     apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1490
     apply(rule Prf.intros)  
42268a284ea6 updated
cu
parents: 276
diff changeset
  1491
      apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1492
     apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1493
    apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1494
   apply(clarify)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1495
   apply(erule Prf_elims)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1496
      apply(simp)
42268a284ea6 updated
cu
parents: 276
diff changeset
  1497
  apply(rule Prf.intros)  
42268a284ea6 updated
cu
parents: 276
diff changeset
  1498
       apply(simp)
278
424bdcd01016 updated
cu
parents: 277
diff changeset
  1499
     apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1500
  (* NTIMES *)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1501
   prefer 4
424bdcd01016 updated
cu
parents: 277
diff changeset
  1502
   apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1503
   apply(case_tac n)
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1504
    apply(simp)
278
424bdcd01016 updated
cu
parents: 277
diff changeset
  1505
   apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1506
   apply(clarify)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1507
   apply(rotate_tac 5)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1508
   apply(erule Prf_elims)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1509
   apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1510
  apply(subst append.simps(2)[symmetric])
424bdcd01016 updated
cu
parents: 277
diff changeset
  1511
      apply(rule Prf.intros) 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1512
        apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1513
       apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1514
   apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1515
  prefer 4
424bdcd01016 updated
cu
parents: 277
diff changeset
  1516
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1517
  apply (metis Prf.intros(8) length_removeAll_less less_irrefl_nat removeAll.simps(1) self_append_conv2)
277
42268a284ea6 updated
cu
parents: 276
diff changeset
  1518
  (* NMTIMES *)
278
424bdcd01016 updated
cu
parents: 277
diff changeset
  1519
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1520
  apply (metis Prf.intros(11) append_Nil empty_iff list.set(1))
424bdcd01016 updated
cu
parents: 277
diff changeset
  1521
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1522
  apply(clarify)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1523
  apply(rotate_tac 6)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1524
  apply(erule Prf_elims)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1525
   apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1526
  apply(subst append.simps(2)[symmetric])
424bdcd01016 updated
cu
parents: 277
diff changeset
  1527
      apply(rule Prf.intros) 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1528
        apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1529
       apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1530
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1531
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1532
  apply(rule Prf.intros) 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1533
        apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1534
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1535
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1536
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1537
  apply(clarify)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1538
  apply(rotate_tac 6)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1539
  apply(erule Prf_elims)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1540
   apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1541
      apply(rule Prf.intros) 
424bdcd01016 updated
cu
parents: 277
diff changeset
  1542
        apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1543
       apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1544
  apply(simp)
424bdcd01016 updated
cu
parents: 277
diff changeset
  1545
done    
276
a3134f7de065 updated
cu
parents: 275
diff changeset
  1546
  
273
e85099ac4c6c updated
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
  1547
end