diff -r 76fa93b1fe8b -r 8f1bf5266ebc LFex.thy --- a/LFex.thy Thu Dec 03 11:58:46 2009 +0100 +++ b/LFex.thy Thu Dec 03 12:17:23 2009 +0100 @@ -264,16 +264,20 @@ using a0 a1 a2 a3 a4 a5 a6 a7 a8 a9 a10 a11 apply - apply(tactic {* procedure_tac @{context} @{thm akind_aty_atrm.induct} 1 *}) +apply(tactic {* regularize_tac @{context} @{thms alpha_EQUIVs} 1 *}) +prefer 2 +apply(tactic {* clean_tac @{context} quot defs 1 *}) + (* Profiling: ML_prf {* fun ith i = (#concl (fst (Subgoal.focus @{context} i (#goal (Isar.goal ()))))) *} ML_prf {* profile 2 Seq.list_of ((clean_tac @{context} quot defs 1) (ith 3)) *} ML_prf {* profile 2 Seq.list_of ((regularize_tac @{context} @{thms alpha_EQUIVs} 1) (ith 1)) *} *) -apply(tactic {* regularize_tac @{context} @{thms alpha_EQUIVs} 1 *}) -prefer 2 -apply(tactic {* clean_tac @{context} quot defs 1 *}) -apply(tactic {* all_inj_repabs_tac @{context} quot rel_refl trans2 1*}) +ML_prf {* PolyML.profiling 1 *} +ML_prf {* profile 2 Seq.list_of ((all_inj_repabs_tac @{context} quot rel_refl trans2 1) (#goal (Isar.goal ()))) *} + +apply(tactic {* all_inj_repabs_tac @{context} quot rel_refl trans2 1 *}) done (* Does not work: