# HG changeset patch # User Cezary Kaliszyk # Date 1306976963 -32400 # Node ID db0ed02eba6ec3ab9f95712d0b2cdc4c91bd60c0 # Parent 5ecb857e9de72b0357b445f7237507fa5d2ae4c2 Remove SMT diff -r 5ecb857e9de7 -r db0ed02eba6e Nominal/Ex/TypeSchemes.thy --- a/Nominal/Ex/TypeSchemes.thy Wed Jun 01 16:13:42 2011 +0900 +++ b/Nominal/Ex/TypeSchemes.thy Thu Jun 02 10:09:23 2011 +0900 @@ -427,13 +427,17 @@ apply (simp add: fresh_star_Un fresh_star_inter1) apply (simp add: alphas fresh_star_zero) apply auto[1] + apply (subgoal_tac "atom xa \ p \ (atom ` fset xs \ supp t)") + apply (simp add: inter_eqvt) + apply blast apply (subgoal_tac "atom xa \ supp(p \ t)") - apply (smt IntI image_iff inf_le1 permute_set_eq_image subsetD) + apply (simp add: IntI image_eqI) apply (drule subsetD[OF supp_subst]) - apply auto[1] apply (simp add: fresh_star_def fresh_def) + apply (subgoal_tac "x \ p \ (atom ` fset xs \ supp t)") + apply (simp add: ) apply (subgoal_tac "x \ supp(p \ t)") - apply (smt IntI inf_le1 inter_eqvt subsetD supp_eqvt) + apply (metis inf1I inter_eqvt mem_def supp_eqvt ) apply (rotate_tac 6) apply (drule sym) apply (simp add: subst_eqvt)