rename_tac'd script
authorblanchet
Tue, 09 Sep 2014 20:51:36 +0200
changeset 58252 7e353ced895e
parent 58251 b13e5c3497f5
child 58253 30e7fecc9e42
rename_tac'd script
src/HOL/IMP/Abs_Int_ITP/Abs_Int2_ITP.thy
--- a/src/HOL/IMP/Abs_Int_ITP/Abs_Int2_ITP.thy	Tue Sep 09 20:51:36 2014 +0200
+++ b/src/HOL/IMP/Abs_Int_ITP/Abs_Int2_ITP.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -314,7 +314,7 @@
 apply(induction e arbitrary: r r' S S')
 apply(auto simp: test_num' Let_def split: option.splits prod.splits)
 apply (metis mono_gamma subsetD)
-apply(drule_tac x = "list" in mono_lookup)
+apply(rename_tac list a b c d, drule_tac x = "list" in mono_lookup)
 apply (metis mono_meet le_trans)
 apply (metis mono_meet mono_lookup mono_update)
 apply(metis mono_aval'' mono_filter_plus'[simplified le_prod_def] fst_conv snd_conv)