src/HOL/HOLCF/IOA/TLS.thy
changeset 62195 799a5306e2ed
parent 62193 0826f6b6ba09
child 62390 842917225d56
--- a/src/HOL/HOLCF/IOA/TLS.thy	Sat Jan 16 23:35:55 2016 +0100
+++ b/src/HOL/HOLCF/IOA/TLS.thy	Sun Jan 17 00:14:45 2016 +0100
@@ -123,9 +123,9 @@
 
 
 lemma ex2seq_nUUnnil: "ex2seq exec \<noteq> UU \<and> ex2seq exec \<noteq> nil"
-  apply (tactic \<open>pair_tac @{context} "exec" 1\<close>)
-  apply (tactic \<open>Seq_case_simp_tac @{context} "x2" 1\<close>)
-  apply (tactic \<open>pair_tac @{context} "a" 1\<close>)
+  apply (pair exec)
+  apply (Seq_case_simp x2)
+  apply (pair a)
   done
 
 
@@ -143,30 +143,30 @@
   apply (simp split add: split_if)
   text \<open>\<open>TL = UU\<close>\<close>
   apply (rule conjI)
-  apply (tactic \<open>pair_tac @{context} "ex" 1\<close>)
-  apply (tactic \<open>Seq_case_simp_tac @{context} "x2" 1\<close>)
-  apply (tactic \<open>pair_tac @{context} "a" 1\<close>)
-  apply (tactic \<open>Seq_case_simp_tac @{context} "s" 1\<close>)
-  apply (tactic \<open>pair_tac @{context} "a" 1\<close>)
+  apply (pair ex)
+  apply (Seq_case_simp x2)
+  apply (pair a)
+  apply (Seq_case_simp s)
+  apply (pair a)
   text \<open>\<open>TL = nil\<close>\<close>
   apply (rule conjI)
-  apply (tactic \<open>pair_tac @{context} "ex" 1\<close>)
-  apply (tactic \<open>Seq_case_tac @{context} "x2" 1\<close>)
+  apply (pair ex)
+  apply (Seq_case x2)
   apply (simp add: unlift_def)
   apply fast
   apply (simp add: unlift_def)
   apply fast
   apply (simp add: unlift_def)
-  apply (tactic \<open>pair_tac @{context} "a" 1\<close>)
-  apply (tactic \<open>Seq_case_simp_tac @{context} "s" 1\<close>)
-  apply (tactic \<open>pair_tac @{context} "a" 1\<close>)
+  apply (pair a)
+  apply (Seq_case_simp s)
+  apply (pair a)
   text \<open>\<open>TL = cons\<close>\<close>
   apply (simp add: unlift_def)
-  apply (tactic \<open>pair_tac @{context} "ex" 1\<close>)
-  apply (tactic \<open>Seq_case_simp_tac @{context} "x2" 1\<close>)
-  apply (tactic \<open>pair_tac @{context} "a" 1\<close>)
-  apply (tactic \<open>Seq_case_simp_tac @{context} "s" 1\<close>)
-  apply (tactic \<open>pair_tac @{context} "a" 1\<close>)
+  apply (pair ex)
+  apply (Seq_case_simp x2)
+  apply (pair a)
+  apply (Seq_case_simp s)
+  apply (pair a)
   done
 
 end