Myhill_2.thy
changeset 385 e5e32faa2446
parent 372 2c56b20032a7
--- 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 \<equiv> {(x\<^isub>p, x\<^isub>s). x\<^isub>p @ x\<^isub>s = x}"
+  "Partitions x \<equiv> {(x\<^sub>p, x\<^sub>s). x\<^sub>p @ x\<^sub>s = x}"
 
 lemma conc_partitions_elim:
   assumes "x \<in> A \<cdot> B"
@@ -234,7 +234,7 @@
 definition 
   tag_Times :: "'a lang \<Rightarrow> 'a lang \<Rightarrow> 'a list \<Rightarrow> 'a lang \<times> 'a lang set"
 where
-  "tag_Times A B \<equiv> \<lambda>x. (\<approx>A `` {x}, {(\<approx>B `` {x\<^isub>s}) | x\<^isub>p x\<^isub>s. x\<^isub>p \<in> A \<and> (x\<^isub>p, x\<^isub>s) \<in> Partitions x})"
+  "tag_Times A B \<equiv> \<lambda>x. (\<approx>A `` {x}, {(\<approx>B `` {x\<^sub>s}) | x\<^sub>p x\<^sub>s. x\<^sub>p \<in> A \<and> (x\<^sub>p, x\<^sub>s) \<in> Partitions x})"
 
 lemma tag_Times_injI:
   assumes a: "tag_Times A B x = tag_Times A B y"