diff -r 6762c8445138 -r 9f5145281888 src/HOL/Library/Omega_Words_Fun.thy --- a/src/HOL/Library/Omega_Words_Fun.thy Sat Oct 10 16:40:43 2015 +0200 +++ b/src/HOL/Library/Omega_Words_Fun.thy Sat Oct 10 19:22:05 2015 +0200 @@ -44,17 +44,13 @@ \ definition - conc :: "['a list, 'a word] \ 'a word" (infixr "conc" 65) - where "w conc x == \n. if n < length w then w!n else x (n - length w)" + conc :: "['a list, 'a word] \ 'a word" (infixr "\" 65) + where "w \ x == \n. if n < length w then w!n else x (n - length w)" definition - iter :: "'a list \ 'a word" + iter :: "'a list \ 'a word" ("(_\<^sup>\)" [1000]) where "iter w == if w = [] then undefined else (\n. w!(n mod (length w)))" -notation (xsymbols) - conc (infixr "\" 65) and - iter ("(_\<^sup>\)" [1000]) - lemma conc_empty[simp]: "[] \ w = w" unfolding conc_def by auto