diff -r 7c26b31d2371 -r f5db9ede89b0 LamEx.thy --- a/LamEx.thy Wed Dec 02 17:16:44 2009 +0100 +++ b/LamEx.thy Wed Dec 02 20:54:59 2009 +0100 @@ -299,3 +299,55 @@ (* Simp starts hanging so don't know how to continue *) sorry +lemma real_alpha_pre: + assumes a: "t = [(a,b)]\s" "a\[b].s" + shows "rLam a t \ rLam b s" +sorry + +lemma perm_prs : "(id ---> option_map ABS_lam) ([b].REP_lam s) = [b].s" +sorry + +lemma perm_prs2: "(id ---> option_map ABS_lam) ((id ---> option_map REP_lam) ([b].(s::lam))) = [b].s" +sorry + +lemma real_alpha: + "\t = [(a, b)] \ s; a \ [b].s\ \ Lam a t = Lam b s" +apply (tactic {* procedure_tac @{context} @{thm real_alpha_pre} 1 *}) +prefer 2 +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* all_inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (tactic {* inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +apply (simp only: perm_prs) +prefer 2 +apply (tactic {* all_inj_repabs_tac @{context} rty [quot] [rel_refl] [trans2] 1 *}) +prefer 3 +apply (tactic {* clean_tac @{context} [quot] defs 1 *}) + +thm all_prs +thm REP_ABS_RSP +thm ball_reg_eqv_range + + +thm perm_lam_def +apply (simp only: perm_prs) + +apply (tactic {* regularize_tac @{context} [quot] 1 *}) + +done +