diff -r 60bcf13adb77 -r e5e32faa2446 Myhill_2.thy --- a/Myhill_2.thy Thu Jul 11 16:46:05 2013 +0100 +++ b/Myhill_2.thy Thu Sep 12 10:34:11 2013 +0200 @@ -207,7 +207,7 @@ subsection {* Case for @{text "Times"} *} definition - "Partitions x \ {(x\<^isub>p, x\<^isub>s). x\<^isub>p @ x\<^isub>s = x}" + "Partitions x \ {(x\<^sub>p, x\<^sub>s). x\<^sub>p @ x\<^sub>s = x}" lemma conc_partitions_elim: assumes "x \ A \ B" @@ -234,7 +234,7 @@ definition tag_Times :: "'a lang \ 'a lang \ 'a list \ 'a lang \ 'a lang set" where - "tag_Times A B \ \x. (\A `` {x}, {(\B `` {x\<^isub>s}) | x\<^isub>p x\<^isub>s. x\<^isub>p \ A \ (x\<^isub>p, x\<^isub>s) \ Partitions x})" + "tag_Times A B \ \x. (\A `` {x}, {(\B `` {x\<^sub>s}) | x\<^sub>p x\<^sub>s. x\<^sub>p \ A \ (x\<^sub>p, x\<^sub>s) \ Partitions x})" lemma tag_Times_injI: assumes a: "tag_Times A B x = tag_Times A B y"