diff -r 3764566c1151 -r fe6eb116b341 LamEx.thy --- a/LamEx.thy Tue Nov 03 16:17:19 2009 +0100 +++ b/LamEx.thy Tue Nov 03 17:30:27 2009 +0100 @@ -166,7 +166,7 @@ ML {* val (rty, rel, rel_refl, rel_eqv) = lookup_quot_data @{context} qty *} ML {* val defs = @{thms Var_def App_def Lam_def perm_lam_def fv_def} *} ML {* val consts = lookup_quot_consts defs *} -ML {* val (trans2, reps_same, quot) = lookup_quot_thms @{context} "lam" *} +ML {* val (trans2, reps_same, absrep, quot) = lookup_quot_thms @{context} "lam" *} ML {* val rsp_thms = @{thms perm_rsp fresh_rsp rVar_rsp rApp_rsp rLam_rsp rfv_rsp} @ @{thms ho_all_prs ho_ex_prs} *} ML {* fun lift_thm_lam lthy t = lift_thm lthy qty "lam" rsp_thms defs t *}