src/HOL/HOLCF/IOA/TL.thy
changeset 62195 799a5306e2ed
parent 62194 0aabc5931361
child 62390 842917225d56
--- a/src/HOL/HOLCF/IOA/TL.thy	Sat Jan 16 23:35:55 2016 +0100
+++ b/src/HOL/HOLCF/IOA/TL.thy	Sun Jan 17 00:14:45 2016 +0100
@@ -113,7 +113,7 @@
 lemma tsuffix_TL [rule_format]: "s \<noteq> UU \<and> s \<noteq> nil \<longrightarrow> tsuffix s2 (TL $ s) \<longrightarrow> tsuffix s2 s"
   apply (unfold tsuffix_def suffix_def)
   apply auto
-  apply (tactic \<open>Seq_case_simp_tac @{context} "s" 1\<close>)
+  apply (Seq_case_simp s)
   apply (rule_tac x = "a \<leadsto> s1" in exI)
   apply auto
   done