diff -r a44479bde681 -r 017e33849f4d Nominal/Ex/Weakening.thy --- a/Nominal/Ex/Weakening.thy Tue Mar 22 12:18:30 2016 +0000 +++ b/Nominal/Ex/Weakening.thy Thu Apr 19 13:57:17 2018 +0100 @@ -107,7 +107,7 @@ valid2 :: "(name \ ty) fset \ bool" where v2_Empty[intro]: "valid2 {||}" -| v2_Insert[intro]: "\(x, T) |\| Gamma; valid2 Gamma\ \ valid2 (insert_fset (x, T) Gamma)" +| v2_Insert[intro]: "\(x, T) |\| Gamma; valid2 Gamma\ \ valid2 (finsert (x, T) Gamma)" equivariance valid2 @@ -116,7 +116,7 @@ where t2_Var[intro]: "\valid2 \; (x, T) |\| \\ \ \ 2\ Var x : T" | t2_App[intro]: "\\ 2\ t1 : T1 \ T2; \ 2\ t2 : T1\ \ \ 2\ App t1 t2 : T2" - | t2_Lam[intro]: "\atom x \ \; insert_fset (x, T1) \ 2\ t : T2\ \ \ 2\ Lam [x]. t : T1 \ T2" + | t2_Lam[intro]: "\atom x \ \; finsert (x, T1) \ 2\ t : T2\ \ \ 2\ Lam [x]. t : T1 \ T2" equivariance typing2 @@ -133,12 +133,8 @@ apply(nominal_induct \ t T avoiding: x rule: typing2.strong_induct) apply(auto)[2] apply(rule t2_Lam) -apply(simp add: fresh_insert_fset fresh_ty) -apply(simp) -apply(drule_tac x="xa" in meta_spec) -apply(drule meta_mp) -apply(simp add: fresh_at_base) -apply(simp add: insert_fset_left_comm) +apply(simp add: fresh_finsert fresh_ty) +apply(force) done lemma weakening_version4: @@ -155,7 +151,7 @@ apply(rule_tac t= "Lam [x]. t" and s="Lam [a]. ((a \ x) \ t)" in subst) defer apply(rule t2_Lam) -apply(simp add: fresh_insert_fset) +apply(simp add: fresh_finsert) oops