diff -r f122816d7729 -r 184d74813679 LFex.thy --- a/LFex.thy Thu Dec 03 12:33:05 2009 +0100 +++ b/LFex.thy Thu Dec 03 13:45:52 2009 +0100 @@ -266,17 +266,16 @@ 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 *}) - +apply(tactic {* simp_tac ((Simplifier.context @{context} empty_ss) addsimps @{thms perm_kind_def perm_ty_def perm_trm_def}) 1 *}) +apply(tactic {* clean_tac @{context} quot 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)) *} -*) 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 @@ -307,7 +306,7 @@ apply(tactic {* procedure_tac @{context} @{thm kind_ty_trm.induct} 1 *}) apply(tactic {* regularize_tac @{context} @{thms alpha_EQUIVs} 1 *}) apply(tactic {* all_inj_repabs_tac @{context} quot rel_refl trans2 1 *}) -apply(tactic {* clean_tac @{context} quot defs 1 *}) +apply(tactic {* clean_tac @{context} quot 1 *}) done print_quotients