Nominal/Ex/ExLetRec.thy
changeset 2104 2205b572bc9b
parent 2101 e417be53916e
child 2105 e25b0fff0dd2
equal deleted inserted replaced
2103:e08e3c29dbc0 2104:2205b572bc9b
    31 thm trm_lts.distinct
    31 thm trm_lts.distinct
    32 thm trm_lts.supp
    32 thm trm_lts.supp
    33 thm trm_lts.fv[simplified trm_lts.supp]
    33 thm trm_lts.fv[simplified trm_lts.supp]
    34 
    34 
    35 declare permute_trm_raw_permute_lts_raw.simps[eqvt]
    35 declare permute_trm_raw_permute_lts_raw.simps[eqvt]
    36 declare alpha_gen_eqvt[eqvt]
       
    37 
    36 
    38 equivariance alpha_trm_raw
    37 equivariance alpha_trm_raw
    39 
    38 
    40 (* why is this not in HOL simpset? *)
    39 (* why is this not in HOL simpset? *)
    41 lemma set_sub: "{a, b} - {b} = {a} - {b}"
    40 lemma set_sub: "{a, b} - {b} = {a} - {b}"