diff -r 1f2788fb0b8b -r f1599e98c4d0 src/HOL/HOLCF/IOA/meta_theory/TL.thy --- a/src/HOL/HOLCF/IOA/meta_theory/TL.thy Wed Dec 30 21:56:12 2015 +0100 +++ b/src/HOL/HOLCF/IOA/meta_theory/TL.thy Wed Dec 30 21:57:52 2015 +0100 @@ -2,7 +2,7 @@ Author: Olaf Müller *) -section {* A General Temporal Logic *} +section \A General Temporal Logic\ theory TL imports Pred Sequence @@ -147,7 +147,7 @@ "s~=UU & s~=nil --> tsuffix s2 (TL$s) --> tsuffix s2 s" apply (unfold tsuffix_def suffix_def) apply auto -apply (tactic {* Seq_case_simp_tac @{context} "s" 1 *}) +apply (tactic \Seq_case_simp_tac @{context} "s" 1\) apply (rule_tac x = "a\s1" in exI) apply auto done