changeset 24 | f72c82bf59e5 |
parent 5 | 074d9a4b2bc9 |
child 102 | 5fed809d0fc1 |
--- a/Matcher.thy Thu Nov 18 11:39:17 2010 +0000 +++ b/Matcher.thy Thu Nov 25 18:54:45 2010 +0000 @@ -21,7 +21,7 @@ | step[intro]: "\<lbrakk>s1 \<in> L; s2 \<in> L\<star>\<rbrakk> \<Longrightarrow> s1 @ s2 \<in> L\<star>" -text {* A standard property of star *} +text {* A standard property of Star *} lemma lang_star_cases: shows "L\<star> = {[]} \<union> L ; L\<star>"