Matcher.thy
changeset 24 f72c82bf59e5
parent 5 074d9a4b2bc9
child 102 5fed809d0fc1
equal deleted inserted replaced
23:e31b733ace44 24:f72c82bf59e5
    19 where
    19 where
    20   start[intro]: "[] \<in> L\<star>"
    20   start[intro]: "[] \<in> L\<star>"
    21 | step[intro]:  "\<lbrakk>s1 \<in> L; s2 \<in> L\<star>\<rbrakk> \<Longrightarrow> s1 @ s2 \<in> L\<star>"
    21 | step[intro]:  "\<lbrakk>s1 \<in> L; s2 \<in> L\<star>\<rbrakk> \<Longrightarrow> s1 @ s2 \<in> L\<star>"
    22 
    22 
    23 
    23 
    24 text {* A standard property of star *}
    24 text {* A standard property of Star *}
    25 
    25 
    26 lemma lang_star_cases:
    26 lemma lang_star_cases:
    27   shows "L\<star> =  {[]} \<union> L ; L\<star>"
    27   shows "L\<star> =  {[]} \<union> L ; L\<star>"
    28 by (auto) (metis Star.simps)
    28 by (auto) (metis Star.simps)
    29 
    29