| author | nipkow | 
| Tue, 06 Sep 2011 14:25:16 +0200 | |
| changeset 44744 | bdf8eb8f126b | 
| parent 41893 | dde7df1176b7 | 
| child 53015 | a1119cf551e8 | 
| permissions | -rw-r--r-- | 
| 26195 | 1 | theory W | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 2 | imports Nominal | 
| 26195 | 3 | begin | 
| 4 | ||
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 5 | text {* Example for strong induction rules avoiding sets of atoms. *}
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 6 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 7 | atom_decl tvar var | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 8 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 9 | abbreviation | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 10 |   "difference_list" :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list" ("_ - _" [60,60] 60) 
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 11 | where | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 12 | "xs - ys \<equiv> [x \<leftarrow> xs. x\<notin>set ys]" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 13 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 14 | lemma difference_eqvt_tvar[eqvt]: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 15 | fixes pi::"tvar prm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 16 | and Xs Ys::"tvar list" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 17 | shows "pi\<bullet>(Xs - Ys) = (pi\<bullet>Xs) - (pi\<bullet>Ys)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 18 | by (induct Xs) (simp_all add: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 19 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 20 | lemma difference_fresh: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 21 | fixes X::"tvar" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 22 | and Xs Ys::"tvar list" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 23 | assumes a: "X\<in>set Ys" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 24 | shows "X\<sharp>(Xs - Ys)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 25 | using a | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 26 | by (induct Xs) (auto simp add: fresh_list_nil fresh_list_cons fresh_atm) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 27 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 28 | lemma difference_supset: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 29 | fixes xs::"'a list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 30 | and ys::"'a list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 31 | and zs::"'a list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 32 | assumes asm: "set xs \<subseteq> set ys" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 33 | shows "xs - ys = []" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 34 | using asm | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 35 | by (induct xs) (auto) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 36 | |
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 37 | nominal_datatype ty = | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 38 | TVar "tvar" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 39 |   | Fun "ty" "ty" ("_\<rightarrow>_" [100,100] 100)
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 40 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 41 | nominal_datatype tyS = | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 42 | Ty "ty" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 43 |   | ALL "\<guillemotleft>tvar\<guillemotright>tyS" ("\<forall>[_]._" [100,100] 100)
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 44 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 45 | nominal_datatype trm = | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 46 | Var "var" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 47 | | App "trm" "trm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 48 |   | Lam "\<guillemotleft>var\<guillemotright>trm" ("Lam [_]._" [100,100] 100)
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 49 | | Let "\<guillemotleft>var\<guillemotright>trm" "trm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 50 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 51 | abbreviation | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 52 |   LetBe :: "var \<Rightarrow> trm \<Rightarrow> trm \<Rightarrow> trm" ("Let _ be _ in _" [100,100,100] 100)
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 53 | where | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 54 | "Let x be t1 in t2 \<equiv> trm.Let x t2 t1" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 55 | |
| 41798 | 56 | type_synonym | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 57 | Ctxt = "(var\<times>tyS) list" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 58 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 59 | text {* free type variables *}
 | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 60 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 61 | consts ftv :: "'a \<Rightarrow> tvar list" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 62 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 63 | overloading | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 64 |   ftv_prod \<equiv> "ftv :: ('a \<times> 'b) \<Rightarrow> tvar list"
 | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 65 | ftv_tvar \<equiv> "ftv :: tvar \<Rightarrow> tvar list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 66 | ftv_var \<equiv> "ftv :: var \<Rightarrow> tvar list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 67 | ftv_list \<equiv> "ftv :: 'a list \<Rightarrow> tvar list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 68 | ftv_ty \<equiv> "ftv :: ty \<Rightarrow> tvar list" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 69 | begin | 
| 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 70 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 71 | primrec | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 72 | ftv_prod | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 73 | where | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 74 | "ftv_prod (x, y) = (ftv x) @ (ftv y)" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 75 | |
| 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 76 | definition | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 77 | ftv_tvar :: "tvar \<Rightarrow> tvar list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 78 | where | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 79 | [simp]: "ftv_tvar X \<equiv> [(X::tvar)]" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 80 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 81 | definition | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 82 | ftv_var :: "var \<Rightarrow> tvar list" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 83 | where | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 84 | [simp]: "ftv_var x \<equiv> []" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 85 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 86 | primrec | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 87 | ftv_list | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 88 | where | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 89 | "ftv_list [] = []" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 90 | | "ftv_list (x#xs) = (ftv x)@(ftv_list xs)" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 91 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 92 | nominal_primrec | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 93 | ftv_ty :: "ty \<Rightarrow> tvar list" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 94 | where | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 95 | "ftv_ty (TVar X) = [X]" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 96 | | "ftv_ty (T1 \<rightarrow>T2) = (ftv_ty T1) @ (ftv_ty T2)" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 97 | by (rule TrueI)+ | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 98 | |
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 99 | end | 
| 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 100 | |
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 101 | lemma ftv_ty_eqvt[eqvt]: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 102 | fixes pi::"tvar prm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 103 | and T::"ty" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 104 | shows "pi\<bullet>(ftv T) = ftv (pi\<bullet>T)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 105 | by (nominal_induct T rule: ty.strong_induct) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 106 | (perm_simp add: append_eqvt)+ | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 107 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 108 | overloading | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 109 | ftv_tyS \<equiv> "ftv :: tyS \<Rightarrow> tvar list" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 110 | begin | 
| 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 111 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 112 | nominal_primrec | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 113 | ftv_tyS :: "tyS \<Rightarrow> tvar list" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 114 | where | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 115 | "ftv_tyS (Ty T) = ((ftv (T::ty))::tvar list)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 116 | | "ftv_tyS (\<forall>[X].S) = (ftv_tyS S) - [X]" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 117 | apply(finite_guess add: ftv_ty_eqvt fs_tvar1)+ | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 118 | apply(rule TrueI)+ | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 119 | apply(rule difference_fresh) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 120 | apply(simp) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 121 | apply(fresh_guess add: ftv_ty_eqvt fs_tvar1)+ | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 122 | done | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 123 | |
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 124 | end | 
| 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 125 | |
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 126 | lemma ftv_tyS_eqvt[eqvt]: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 127 | fixes pi::"tvar prm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 128 | and S::"tyS" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 129 | shows "pi\<bullet>(ftv S) = ftv (pi\<bullet>S)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 130 | apply(nominal_induct S rule: tyS.strong_induct) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 131 | apply(simp add: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 132 | apply(simp only: ftv_tyS.simps) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 133 | apply(simp only: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 134 | apply(simp add: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 135 | done | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 136 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 137 | lemma ftv_Ctxt_eqvt[eqvt]: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 138 | fixes pi::"tvar prm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 139 | and \<Gamma>::"Ctxt" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 140 | shows "pi\<bullet>(ftv \<Gamma>) = ftv (pi\<bullet>\<Gamma>)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 141 | by (induct \<Gamma>) (auto simp add: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 142 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 143 | text {* Valid *}
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 144 | inductive | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 145 | valid :: "Ctxt \<Rightarrow> bool" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 146 | where | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 147 | V_Nil[intro]: "valid []" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 148 | | V_Cons[intro]: "\<lbrakk>valid \<Gamma>;x\<sharp>\<Gamma>\<rbrakk>\<Longrightarrow> valid ((x,S)#\<Gamma>)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 149 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 150 | equivariance valid | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 151 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 152 | text {* General *}
 | 
| 39246 | 153 | primrec gen :: "ty \<Rightarrow> tvar list \<Rightarrow> tyS" where | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 154 | "gen T [] = Ty T" | 
| 39246 | 155 | | "gen T (X#Xs) = \<forall>[X].(gen T Xs)" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 156 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 157 | lemma gen_eqvt[eqvt]: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 158 | fixes pi::"tvar prm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 159 | shows "pi\<bullet>(gen T Xs) = gen (pi\<bullet>T) (pi\<bullet>Xs)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 160 | by (induct Xs) (simp_all add: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 161 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 162 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 163 | |
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 164 | abbreviation | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 165 | close :: "Ctxt \<Rightarrow> ty \<Rightarrow> tyS" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 166 | where | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 167 | "close \<Gamma> T \<equiv> gen T ((ftv T) - (ftv \<Gamma>))" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 168 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 169 | lemma close_eqvt[eqvt]: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 170 | fixes pi::"tvar prm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 171 | shows "pi\<bullet>(close \<Gamma> T) = close (pi\<bullet>\<Gamma>) (pi\<bullet>T)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 172 | by (simp_all only: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 173 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 174 | text {* Substitution *}
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 175 | |
| 41798 | 176 | type_synonym Subst = "(tvar\<times>ty) list" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 177 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 178 | consts | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 179 |   psubst :: "Subst \<Rightarrow> 'a \<Rightarrow> 'a"       ("_<_>" [100,60] 120)
 | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 180 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 181 | abbreviation | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 182 |   subst :: "'a \<Rightarrow> tvar \<Rightarrow> ty \<Rightarrow> 'a"  ("_[_::=_]" [100,100,100] 100)
 | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 183 | where | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 184 | "smth[X::=T] \<equiv> ([(X,T)])<smth>" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 185 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 186 | fun | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 187 | lookup :: "Subst \<Rightarrow> tvar \<Rightarrow> ty" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 188 | where | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 189 | "lookup [] X = TVar X" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 190 | | "lookup ((Y,T)#\<theta>) X = (if X=Y then T else lookup \<theta> X)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 191 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 192 | lemma lookup_eqvt[eqvt]: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 193 | fixes pi::"tvar prm" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 194 | shows "pi\<bullet>(lookup \<theta> X) = lookup (pi\<bullet>\<theta>) (pi\<bullet>X)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 195 | by (induct \<theta>) (auto simp add: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 196 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 197 | lemma lookup_fresh: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 198 | fixes X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 199 | assumes a: "X\<sharp>\<theta>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 200 | shows "lookup \<theta> X = TVar X" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 201 | using a | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 202 | by (induct \<theta>) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 203 | (auto simp add: fresh_list_cons fresh_prod fresh_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 204 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 205 | overloading | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 206 | psubst_ty \<equiv> "psubst :: Subst \<Rightarrow> ty \<Rightarrow> ty" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 207 | begin | 
| 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 208 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 209 | nominal_primrec | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 210 | psubst_ty | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 211 | where | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 212 | "\<theta><TVar X> = lookup \<theta> X" | 
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 213 | | "\<theta><T\<^isub>1 \<rightarrow> T\<^isub>2> = (\<theta><T\<^isub>1>) \<rightarrow> (\<theta><T\<^isub>2>)" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 214 | by (rule TrueI)+ | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 215 | |
| 29098 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 216 | end | 
| 
6b23a58cc67c
Unified syntax of nominal_primrec with the one used by fun(ction) and new
 berghofe parents: 
28655diff
changeset | 217 | |
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 218 | lemma psubst_ty_eqvt[eqvt]: | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 219 | fixes pi::"tvar prm" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 220 | and \<theta>::"Subst" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 221 | and T::"ty" | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 222 | shows "pi\<bullet>(\<theta><T>) = (pi\<bullet>\<theta>)<(pi\<bullet>T)>" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 223 | by (induct T rule: ty.induct) (simp_all add: eqvts) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 224 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 225 | overloading | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 226 | psubst_tyS \<equiv> "psubst :: Subst \<Rightarrow> tyS \<Rightarrow> tyS" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 227 | begin | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 228 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 229 | nominal_primrec | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 230 | psubst_tyS :: "Subst \<Rightarrow> tyS \<Rightarrow> tyS" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 231 | where | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 232 | "\<theta><(Ty T)> = Ty (\<theta><T>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 233 | | "X\<sharp>\<theta> \<Longrightarrow> \<theta><(\<forall>[X].S)> = \<forall>[X].(\<theta><S>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 234 | apply(finite_guess add: psubst_ty_eqvt fs_tvar1)+ | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 235 | apply(rule TrueI)+ | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 236 | apply(simp add: abs_fresh) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 237 | apply(fresh_guess add: psubst_ty_eqvt fs_tvar1)+ | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 238 | done | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 239 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 240 | end | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 241 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 242 | overloading | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 243 | psubst_Ctxt \<equiv> "psubst :: Subst \<Rightarrow> Ctxt \<Rightarrow> Ctxt" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 244 | begin | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 245 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 246 | fun | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 247 | psubst_Ctxt :: "Subst \<Rightarrow> Ctxt \<Rightarrow> Ctxt" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 248 | where | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 249 | "psubst_Ctxt \<theta> [] = []" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 250 | | "psubst_Ctxt \<theta> ((x,S)#\<Gamma>) = (x,\<theta><S>)#(psubst_Ctxt \<theta> \<Gamma>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 251 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 252 | end | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 253 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 254 | lemma fresh_lookup: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 255 | fixes X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 256 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 257 | and Y::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 258 | assumes asms: "X\<sharp>Y" "X\<sharp>\<theta>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 259 | shows "X\<sharp>(lookup \<theta> Y)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 260 | using asms | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 261 | by (induct \<theta>) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 262 | (auto simp add: fresh_list_cons fresh_prod fresh_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 263 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 264 | lemma fresh_psubst_ty: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 265 | fixes X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 266 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 267 | and T::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 268 | assumes asms: "X\<sharp>\<theta>" "X\<sharp>T" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 269 | shows "X\<sharp>\<theta><T>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 270 | using asms | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 271 | by (nominal_induct T rule: ty.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 272 | (auto simp add: fresh_list_append fresh_list_cons fresh_prod fresh_lookup) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 273 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 274 | lemma fresh_psubst_tyS: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 275 | fixes X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 276 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 277 | and S::"tyS" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 278 | assumes asms: "X\<sharp>\<theta>" "X\<sharp>S" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 279 | shows "X\<sharp>\<theta><S>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 280 | using asms | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 281 | by (nominal_induct S avoiding: \<theta> X rule: tyS.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 282 | (auto simp add: fresh_psubst_ty abs_fresh) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 283 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 284 | lemma fresh_psubst_Ctxt: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 285 | fixes X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 286 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 287 | and \<Gamma>::"Ctxt" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 288 | assumes asms: "X\<sharp>\<theta>" "X\<sharp>\<Gamma>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 289 | shows "X\<sharp>\<theta><\<Gamma>>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 290 | using asms | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 291 | by (induct \<Gamma>) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 292 | (auto simp add: fresh_psubst_tyS fresh_list_cons) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 293 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 294 | lemma subst_freshfact2_ty: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 295 | fixes X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 296 | and Y::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 297 | and T::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 298 | assumes asms: "X\<sharp>S" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 299 | shows "X\<sharp>T[X::=S]" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 300 | using asms | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 301 | by (nominal_induct T rule: ty.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 302 | (auto simp add: fresh_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 303 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 304 | text {* instance of a type scheme *}
 | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 305 | inductive | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 306 |   inst :: "ty \<Rightarrow> tyS \<Rightarrow> bool"("_ \<prec> _" [50,51] 50)  
 | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 307 | where | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 308 | I_Ty[intro]: "T \<prec> (Ty T)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 309 | | I_All[intro]: "\<lbrakk>X\<sharp>T'; T \<prec> S\<rbrakk> \<Longrightarrow> T[X::=T'] \<prec> \<forall>[X].S" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 310 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 311 | equivariance inst[tvar] | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 312 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 313 | nominal_inductive inst | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 314 | by (simp_all add: abs_fresh subst_freshfact2_ty) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 315 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 316 | lemma subst_forget_ty: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 317 | fixes T::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 318 | and X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 319 | assumes a: "X\<sharp>T" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 320 | shows "T[X::=S] = T" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 321 | using a | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 322 | by (nominal_induct T rule: ty.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 323 | (auto simp add: fresh_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 324 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 325 | lemma psubst_ty_lemma: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 326 | fixes \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 327 | and X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 328 | and T'::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 329 | and T::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 330 | assumes a: "X\<sharp>\<theta>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 331 | shows "\<theta><T[X::=T']> = (\<theta><T>)[X::=\<theta><T'>]" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 332 | using a | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 333 | apply(nominal_induct T avoiding: \<theta> X T' rule: ty.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 334 | apply(auto simp add: ty.inject lookup_fresh) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 335 | apply(rule sym) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 336 | apply(rule subst_forget_ty) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 337 | apply(rule fresh_lookup) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 338 | apply(simp_all add: fresh_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 339 | done | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 340 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 341 | lemma general_preserved: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 342 | fixes \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 343 | assumes a: "T \<prec> S" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 344 | shows "\<theta><T> \<prec> \<theta><S>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 345 | using a | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 346 | apply(nominal_induct T S avoiding: \<theta> rule: inst.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 347 | apply(auto)[1] | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 348 | apply(simp add: psubst_ty_lemma) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 349 | apply(rule_tac I_All) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 350 | apply(simp add: fresh_psubst_ty) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 351 | apply(simp) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 352 | done | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 353 | |
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 354 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 355 | text{* typing judgements *}
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 356 | inductive | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 357 |   typing :: "Ctxt \<Rightarrow> trm \<Rightarrow> ty \<Rightarrow> bool" (" _ \<turnstile> _ : _ " [60,60,60] 60) 
 | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 358 | where | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 359 | T_VAR[intro]: "\<lbrakk>valid \<Gamma>; (x,S)\<in>set \<Gamma>; T \<prec> S\<rbrakk>\<Longrightarrow> \<Gamma> \<turnstile> Var x : T" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 360 | | T_APP[intro]: "\<lbrakk>\<Gamma> \<turnstile> t\<^isub>1 : T\<^isub>1\<rightarrow>T\<^isub>2; \<Gamma> \<turnstile> t\<^isub>2 : T\<^isub>1\<rbrakk>\<Longrightarrow> \<Gamma> \<turnstile> App t\<^isub>1 t\<^isub>2 : T\<^isub>2" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 361 | | T_LAM[intro]: "\<lbrakk>x\<sharp>\<Gamma>;((x,Ty T\<^isub>1)#\<Gamma>) \<turnstile> t : T\<^isub>2\<rbrakk> \<Longrightarrow> \<Gamma> \<turnstile> Lam [x].t : T\<^isub>1\<rightarrow>T\<^isub>2" | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 362 | | T_LET[intro]: "\<lbrakk>x\<sharp>\<Gamma>; \<Gamma> \<turnstile> t\<^isub>1 : T\<^isub>1; ((x,close \<Gamma> T\<^isub>1)#\<Gamma>) \<turnstile> t\<^isub>2 : T\<^isub>2; set (ftv T\<^isub>1 - ftv \<Gamma>) \<sharp>* T\<^isub>2\<rbrakk> | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 363 | \<Longrightarrow> \<Gamma> \<turnstile> Let x be t\<^isub>1 in t\<^isub>2 : T\<^isub>2" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 364 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 365 | equivariance typing[tvar] | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 366 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 367 | lemma fresh_tvar_trm: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 368 | fixes X::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 369 | and t::"trm" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 370 | shows "X\<sharp>t" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 371 | by (nominal_induct t rule: trm.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 372 | (simp_all add: fresh_atm abs_fresh) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 373 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 374 | lemma ftv_ty: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 375 | fixes T::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 376 | shows "supp T = set (ftv T)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 377 | by (nominal_induct T rule: ty.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 378 | (simp_all add: ty.supp supp_atm) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 379 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 380 | lemma ftv_tyS: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 381 | fixes S::"tyS" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 382 | shows "supp S = set (ftv S)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 383 | by (nominal_induct S rule: tyS.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 384 | (auto simp add: tyS.supp abs_supp ftv_ty) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 385 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 386 | lemma ftv_Ctxt: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 387 | fixes \<Gamma>::"Ctxt" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 388 | shows "supp \<Gamma> = set (ftv \<Gamma>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 389 | apply (induct \<Gamma>) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 390 | apply (simp_all add: supp_list_nil supp_list_cons) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 391 | apply (case_tac a) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 392 | apply (simp add: supp_prod supp_atm ftv_tyS) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 393 | done | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 394 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 395 | lemma ftv_tvars: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 396 | fixes Tvs::"tvar list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 397 | shows "supp Tvs = set Tvs" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 398 | by (induct Tvs) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 399 | (simp_all add: supp_list_nil supp_list_cons supp_atm) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 400 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 401 | lemma difference_supp: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 402 | fixes xs ys::"tvar list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 403 | shows "((supp (xs - ys))::tvar set) = supp xs - supp ys" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 404 | by (induct xs) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 405 | (auto simp add: supp_list_nil supp_list_cons ftv_tvars) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 406 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 407 | lemma set_supp_eq: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 408 | fixes xs::"tvar list" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 409 | shows "set xs = supp xs" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 410 | by (induct xs) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 411 | (simp_all add: supp_list_nil supp_list_cons supp_atm) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 412 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 413 | nominal_inductive2 typing | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 414 | avoids T_LET: "set (ftv T\<^isub>1 - ftv \<Gamma>)" | 
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 415 | apply (simp add: fresh_star_def fresh_def ftv_Ctxt) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 416 | apply (simp add: fresh_star_def fresh_tvar_trm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 417 | apply assumption | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 418 | apply simp | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 419 | done | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 420 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 421 | lemma perm_fresh_fresh_aux: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 422 | "\<forall>(x,y)\<in>set (pi::tvar prm). x \<sharp> z \<and> y \<sharp> z \<Longrightarrow> pi \<bullet> (z::'a::pt_tvar) = z" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 423 | apply (induct pi rule: rev_induct) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 424 | apply simp | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 425 | apply (simp add: split_paired_all pt_tvar2) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 426 | apply (frule_tac x="(a, b)" in bspec) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 427 | apply simp | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 428 | apply (simp add: perm_fresh_fresh) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 429 | done | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 430 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 431 | lemma freshs_mem: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 432 | fixes S::"tvar set" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 433 | assumes "x \<in> S" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 434 | and "S \<sharp>* z" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 435 | shows "x \<sharp> z" | 
| 41893 | 436 | using assms by (simp add: fresh_star_def) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 437 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 438 | lemma fresh_gen_set: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 439 | fixes X::"tvar" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 440 | and Xs::"tvar list" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 441 | assumes asm: "X\<in>set Xs" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 442 | shows "X\<sharp>gen T Xs" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 443 | using asm | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 444 | apply(induct Xs) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 445 | apply(simp) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 446 | apply(case_tac "X=a") | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 447 | apply(simp add: abs_fresh) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 448 | apply(simp add: abs_fresh) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 449 | done | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 450 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 451 | lemma close_fresh: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 452 | fixes \<Gamma>::"Ctxt" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 453 | shows "\<forall>(X::tvar)\<in>set ((ftv T) - (ftv \<Gamma>)). X\<sharp>(close \<Gamma> T)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 454 | by (simp add: fresh_gen_set) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 455 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 456 | lemma gen_supp: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 457 | shows "(supp (gen T Xs)::tvar set) = supp T - supp Xs" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 458 | by (induct Xs) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 459 | (auto simp add: supp_list_nil supp_list_cons tyS.supp abs_supp supp_atm) | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 460 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 461 | lemma minus_Int_eq: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 462 | shows "T - (T - U) = T \<inter> U" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 463 | by blast | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 464 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 465 | lemma close_supp: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 466 | shows "supp (close \<Gamma> T) = set (ftv T) \<inter> set (ftv \<Gamma>)" | 
| 28655 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 467 | apply (simp add: gen_supp difference_supp ftv_ty ftv_Ctxt) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 468 | apply (simp only: set_supp_eq minus_Int_eq) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 469 | done | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 470 | |
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 471 | lemma better_T_LET: | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 472 | assumes x: "x\<sharp>\<Gamma>" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 473 | and t1: "\<Gamma> \<turnstile> t\<^isub>1 : T\<^isub>1" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 474 | and t2: "((x,close \<Gamma> T\<^isub>1)#\<Gamma>) \<turnstile> t\<^isub>2 : T\<^isub>2" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 475 | shows "\<Gamma> \<turnstile> Let x be t\<^isub>1 in t\<^isub>2 : T\<^isub>2" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 476 | proof - | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 477 | have fin: "finite (set (ftv T\<^isub>1 - ftv \<Gamma>))" by simp | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 478 | obtain pi where pi1: "(pi \<bullet> set (ftv T\<^isub>1 - ftv \<Gamma>)) \<sharp>* (T\<^isub>2, \<Gamma>)" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 479 | and pi2: "set pi \<subseteq> set (ftv T\<^isub>1 - ftv \<Gamma>) \<times> (pi \<bullet> set (ftv T\<^isub>1 - ftv \<Gamma>))" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 480 | by (rule at_set_avoiding [OF at_tvar_inst fin fs_tvar1, of "(T\<^isub>2, \<Gamma>)"]) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 481 | from pi1 have pi1': "(pi \<bullet> set (ftv T\<^isub>1 - ftv \<Gamma>)) \<sharp>* \<Gamma>" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 482 | by (simp add: fresh_star_prod) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 483 | have Gamma_fresh: "\<forall>(x,y)\<in>set pi. x \<sharp> \<Gamma> \<and> y \<sharp> \<Gamma>" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 484 | apply (rule ballI) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 485 | apply (simp add: split_paired_all) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 486 | apply (drule subsetD [OF pi2]) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 487 | apply (erule SigmaE) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 488 | apply (drule freshs_mem [OF _ pi1']) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 489 | apply (simp add: ftv_Ctxt [symmetric] fresh_def) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 490 | done | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 491 | have close_fresh': "\<forall>(x, y)\<in>set pi. x \<sharp> close \<Gamma> T\<^isub>1 \<and> y \<sharp> close \<Gamma> T\<^isub>1" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 492 | apply (rule ballI) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 493 | apply (simp add: split_paired_all) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 494 | apply (drule subsetD [OF pi2]) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 495 | apply (erule SigmaE) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 496 | apply (drule bspec [OF close_fresh]) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 497 | apply (drule freshs_mem [OF _ pi1']) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 498 | apply (simp add: fresh_def close_supp ftv_Ctxt) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 499 | done | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 500 | note x | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 501 | moreover from Gamma_fresh perm_boolI [OF t1, of pi] | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 502 | have "\<Gamma> \<turnstile> t\<^isub>1 : pi \<bullet> T\<^isub>1" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 503 | by (simp add: perm_fresh_fresh_aux eqvts fresh_tvar_trm) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 504 | moreover from t2 close_fresh' | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 505 | have "(x,(pi \<bullet> close \<Gamma> T\<^isub>1))#\<Gamma> \<turnstile> t\<^isub>2 : T\<^isub>2" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 506 | by (simp add: perm_fresh_fresh_aux) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 507 | with Gamma_fresh have "(x,close \<Gamma> (pi \<bullet> T\<^isub>1))#\<Gamma> \<turnstile> t\<^isub>2 : T\<^isub>2" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 508 | by (simp add: close_eqvt perm_fresh_fresh_aux) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 509 | moreover from pi1 Gamma_fresh | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 510 | have "set (ftv (pi \<bullet> T\<^isub>1) - ftv \<Gamma>) \<sharp>* T\<^isub>2" | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 511 | by (simp only: eqvts fresh_star_prod perm_fresh_fresh_aux) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 512 | ultimately show ?thesis by (rule T_LET) | 
| 
2822c56dd1cf
Example for using the generalized version of nominal_inductive.
 berghofe parents: 
26195diff
changeset | 513 | qed | 
| 26195 | 514 | |
| 32137 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 515 | lemma ftv_ty_subst: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 516 | fixes T::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 517 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 518 | and X Y ::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 519 | assumes a1: "X \<in> set (ftv T)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 520 | and a2: "Y \<in> set (ftv (lookup \<theta> X))" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 521 | shows "Y \<in> set (ftv (\<theta><T>))" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 522 | using a1 a2 | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 523 | by (nominal_induct T rule: ty.strong_induct) (auto) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 524 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 525 | lemma ftv_tyS_subst: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 526 | fixes S::"tyS" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 527 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 528 | and X Y::"tvar" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 529 | assumes a1: "X \<in> set (ftv S)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 530 | and a2: "Y \<in> set (ftv (lookup \<theta> X))" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 531 | shows "Y \<in> set (ftv (\<theta><S>))" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 532 | using a1 a2 | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 533 | by (nominal_induct S avoiding: \<theta> Y rule: tyS.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 534 | (auto simp add: ftv_ty_subst fresh_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 535 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 536 | lemma ftv_Ctxt_subst: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 537 | fixes \<Gamma>::"Ctxt" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 538 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 539 | assumes a1: "X \<in> set (ftv \<Gamma>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 540 | and a2: "Y \<in> set (ftv (lookup \<theta> X))" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 541 | shows "Y \<in> set (ftv (\<theta><\<Gamma>>))" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 542 | using a1 a2 | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 543 | by (induct \<Gamma>) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 544 | (auto simp add: ftv_tyS_subst) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 545 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 546 | lemma gen_preserved1: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 547 | assumes asm: "Xs \<sharp>* \<theta>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 548 | shows "\<theta><gen T Xs> = gen (\<theta><T>) Xs" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 549 | using asm | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 550 | by (induct Xs) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 551 | (auto simp add: fresh_star_def) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 552 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 553 | lemma gen_preserved2: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 554 | fixes T::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 555 | and \<Gamma>::"Ctxt" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 556 | assumes asm: "((ftv T) - (ftv \<Gamma>)) \<sharp>* \<theta>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 557 | shows "((ftv (\<theta><T>)) - (ftv (\<theta><\<Gamma>>))) = ((ftv T) - (ftv \<Gamma>))" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 558 | using asm | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 559 | apply(nominal_induct T rule: ty.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 560 | apply(auto simp add: fresh_star_def) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 561 | apply(simp add: lookup_fresh) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 562 | apply(simp add: ftv_Ctxt[symmetric]) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 563 | apply(fold fresh_def) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 564 | apply(rule fresh_psubst_Ctxt) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 565 | apply(assumption) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 566 | apply(assumption) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 567 | apply(rule difference_supset) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 568 | apply(auto) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 569 | apply(simp add: ftv_Ctxt_subst) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 570 | done | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 571 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 572 | lemma close_preserved: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 573 | fixes \<Gamma>::"Ctxt" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 574 | assumes asm: "((ftv T) - (ftv \<Gamma>)) \<sharp>* \<theta>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 575 | shows "\<theta><close \<Gamma> T> = close (\<theta><\<Gamma>>) (\<theta><T>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 576 | using asm | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 577 | by (simp add: gen_preserved1 gen_preserved2) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 578 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 579 | lemma var_fresh_for_ty: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 580 | fixes x::"var" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 581 | and T::"ty" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 582 | shows "x\<sharp>T" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 583 | by (nominal_induct T rule: ty.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 584 | (simp_all add: fresh_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 585 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 586 | lemma var_fresh_for_tyS: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 587 | fixes x::"var" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 588 | and S::"tyS" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 589 | shows "x\<sharp>S" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 590 | by (nominal_induct S rule: tyS.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 591 | (simp_all add: abs_fresh var_fresh_for_ty) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 592 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 593 | lemma psubst_fresh_Ctxt: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 594 | fixes x::"var" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 595 | and \<Gamma>::"Ctxt" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 596 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 597 | shows "x\<sharp>\<theta><\<Gamma>> = x\<sharp>\<Gamma>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 598 | by (induct \<Gamma>) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 599 | (auto simp add: fresh_list_cons fresh_list_nil fresh_prod var_fresh_for_tyS) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 600 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 601 | lemma psubst_valid: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 602 | fixes \<theta>::Subst | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 603 | and \<Gamma>::Ctxt | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 604 | assumes a: "valid \<Gamma>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 605 | shows "valid (\<theta><\<Gamma>>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 606 | using a | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 607 | by (induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 608 | (auto simp add: psubst_fresh_Ctxt) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 609 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 610 | lemma psubst_in: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 611 | fixes \<Gamma>::"Ctxt" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 612 | and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 613 | and pi::"tvar prm" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 614 | and S::"tyS" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 615 | assumes a: "(x,S)\<in>set \<Gamma>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 616 | shows "(x,\<theta><S>)\<in>set (\<theta><\<Gamma>>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 617 | using a | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 618 | by (induct \<Gamma>) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 619 | (auto simp add: calc_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 620 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 621 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 622 | lemma typing_preserved: | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 623 | fixes \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 624 | and pi::"tvar prm" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 625 | assumes a: "\<Gamma> \<turnstile> t : T" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 626 | shows "(\<theta><\<Gamma>>) \<turnstile> t : (\<theta><T>)" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 627 | using a | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 628 | proof (nominal_induct \<Gamma> t T avoiding: \<theta> rule: typing.strong_induct) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 629 | case (T_VAR \<Gamma> x S T) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 630 | have a1: "valid \<Gamma>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 631 | have a2: "(x, S) \<in> set \<Gamma>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 632 | have a3: "T \<prec> S" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 633 | have "valid (\<theta><\<Gamma>>)" using a1 by (simp add: psubst_valid) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 634 | moreover | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 635 | have "(x,\<theta><S>)\<in>set (\<theta><\<Gamma>>)" using a2 by (simp add: psubst_in) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 636 | moreover | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 637 | have "\<theta><T> \<prec> \<theta><S>" using a3 by (simp add: general_preserved) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 638 | ultimately show "(\<theta><\<Gamma>>) \<turnstile> Var x : (\<theta><T>)" by (simp add: typing.T_VAR) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 639 | next | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 640 | case (T_APP \<Gamma> t1 T1 T2 t2) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 641 | have "\<theta><\<Gamma>> \<turnstile> t1 : \<theta><T1 \<rightarrow> T2>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 642 | then have "\<theta><\<Gamma>> \<turnstile> t1 : (\<theta><T1>) \<rightarrow> (\<theta><T2>)" by simp | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 643 | moreover | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 644 | have "\<theta><\<Gamma>> \<turnstile> t2 : \<theta><T1>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 645 | ultimately show "\<theta><\<Gamma>> \<turnstile> App t1 t2 : \<theta><T2>" by (simp add: typing.T_APP) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 646 | next | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 647 | case (T_LAM x \<Gamma> T1 t T2) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 648 | fix pi::"tvar prm" and \<theta>::"Subst" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 649 | have "x\<sharp>\<Gamma>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 650 | then have "x\<sharp>\<theta><\<Gamma>>" by (simp add: psubst_fresh_Ctxt) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 651 | moreover | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 652 | have "\<theta><((x, Ty T1)#\<Gamma>)> \<turnstile> t : \<theta><T2>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 653 | then have "((x, Ty (\<theta><T1>))#(\<theta><\<Gamma>>)) \<turnstile> t : \<theta><T2>" by (simp add: calc_atm) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 654 | ultimately show "\<theta><\<Gamma>> \<turnstile> Lam [x].t : \<theta><T1 \<rightarrow> T2>" by (simp add: typing.T_LAM) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 655 | next | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 656 | case (T_LET x \<Gamma> t1 T1 t2 T2) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 657 | have vc: "((ftv T1) - (ftv \<Gamma>)) \<sharp>* \<theta>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 658 | have "x\<sharp>\<Gamma>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 659 | then have a1: "x\<sharp>\<theta><\<Gamma>>" by (simp add: calc_atm psubst_fresh_Ctxt) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 660 | have a2: "\<theta><\<Gamma>> \<turnstile> t1 : \<theta><T1>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 661 | have a3: "\<theta><((x, close \<Gamma> T1)#\<Gamma>)> \<turnstile> t2 : \<theta><T2>" by fact | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 662 | from a2 a3 show "\<theta><\<Gamma>> \<turnstile> Let x be t1 in t2 : \<theta><T2>" | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 663 | apply - | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 664 | apply(rule better_T_LET) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 665 | apply(rule a1) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 666 | apply(rule a2) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 667 | apply(simp add: close_preserved vc) | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 668 | done | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 669 | qed | 
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 670 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 671 | |
| 
3b260527fc11
tuned proofs and added some lemmas
 Christian Urban <urbanc@in.tum.de> parents: 
29608diff
changeset | 672 | |
| 26195 | 673 | end |