Myhill_1.thy
changeset 60 fb08f41ca33d
parent 56 b3898315e687
child 66 828ea293b61f
equal deleted inserted replaced
59:fc35eb54fdc9 60:fb08f41ca33d
    30 
    30 
    31 text {* 
    31 text {* 
    32   Sequential composition of two languages @{text "L1"} and @{text "L2"} 
    32   Sequential composition of two languages @{text "L1"} and @{text "L2"} 
    33 *}
    33 *}
    34 
    34 
    35 definition Seq :: "lang \<Rightarrow> lang \<Rightarrow> lang" (infixr ";;" 100)
    35 definition 
       
    36   Seq :: "lang \<Rightarrow> lang \<Rightarrow> lang" (infixr ";;" 100)
    36 where 
    37 where 
    37   "A ;; B = {s\<^isub>1 @ s\<^isub>2 | s\<^isub>1 s\<^isub>2. s\<^isub>1 \<in> A \<and> s\<^isub>2 \<in> B}"
    38   "A ;; B = {s\<^isub>1 @ s\<^isub>2 | s\<^isub>1 s\<^isub>2. s\<^isub>1 \<in> A \<and> s\<^isub>2 \<in> B}"
    38 
    39 
    39 text {* Some properties of operator @{text ";;"}. *}
    40 text {* Some properties of operator @{text ";;"}. *}
    40 
    41