src/HOL/Hoare_Parallel/OG_Tactics.thy
changeset 39159 0dec18004e75
parent 37136 e0c9d3e49e15
child 44928 7ef6505bde7f
--- a/src/HOL/Hoare_Parallel/OG_Tactics.thy	Mon Sep 06 19:11:01 2010 +0200
+++ b/src/HOL/Hoare_Parallel/OG_Tactics.thy	Mon Sep 06 19:13:10 2010 +0200
@@ -273,11 +273,11 @@
 lemmas ParallelConseq_list = INTER_def Collect_conj_eq length_map length_upt length_append list_length
 
 ML {*
-val before_interfree_simp_tac = (simp_tac (HOL_basic_ss addsimps [thm "com.simps", thm "post.simps"]))
+val before_interfree_simp_tac = simp_tac (HOL_basic_ss addsimps [@{thm com.simps}, @{thm post.simps}])
 
-val  interfree_simp_tac = (asm_simp_tac (HOL_ss addsimps [@{thm split}, thm "ball_Un", thm "ball_empty"]@(thms "my_simp_list")))
+val  interfree_simp_tac = asm_simp_tac (HOL_ss addsimps [@{thm split}, @{thm ball_Un}, @{thm ball_empty}] @ @{thms my_simp_list})
 
-val ParallelConseq = (simp_tac (HOL_basic_ss addsimps (thms "ParallelConseq_list")@(thms "my_simp_list")))
+val ParallelConseq = simp_tac (HOL_basic_ss addsimps @{thms ParallelConseq_list} @ @{thms my_simp_list})
 *}
 
 text {* The following tactic applies @{text tac} to each conjunct in a