| author | nipkow | 
| Tue, 11 Oct 2022 10:45:42 +0200 | |
| changeset 76259 | d1c26efb7a47 | 
| parent 74101 | d804e93ae9ff | 
| child 80138 | a30a1385f7d0 | 
| permissions | -rw-r--r-- | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1 | theory Class1 | 
| 66453 
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
 wenzelm parents: 
63167diff
changeset | 2 | imports "HOL-Nominal.Nominal" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3 | begin | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4 | |
| 63167 | 5 | section \<open>Term-Calculus from Urban's PhD\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7 | atom_decl name coname | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8 | |
| 63167 | 9 | text \<open>types\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 10 | |
| 74101 | 11 | no_notation not  ("NOT")
 | 
| 12 | ||
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 13 | nominal_datatype ty = | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 14 | PR "string" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 15 | | NOT "ty" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 16 |   | AND  "ty" "ty"   ("_ AND _" [100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 17 |   | OR   "ty" "ty"   ("_ OR _" [100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 18 |   | IMP  "ty" "ty"   ("_ IMP _" [100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 19 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 20 | instantiation ty :: size | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 21 | begin | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 22 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 23 | nominal_primrec size_ty | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 24 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 25 | "size (PR s) = (1::nat)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 26 | | "size (NOT T) = 1 + size T" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 27 | | "size (T1 AND T2) = 1 + size T1 + size T2" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 28 | | "size (T1 OR T2) = 1 + size T1 + size T2" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 29 | | "size (T1 IMP T2) = 1 + size T1 + size T2" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 30 | by (rule TrueI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 31 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 32 | instance .. | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 33 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 34 | end | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 35 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 36 | lemma ty_cases: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 37 | fixes T::ty | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 38 | shows "(\<exists>s. T=PR s) \<or> (\<exists>T'. T=NOT T') \<or> (\<exists>S U. T=S OR U) \<or> (\<exists>S U. T=S AND U) \<or> (\<exists>S U. T=S IMP U)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 39 | by (induct T rule:ty.induct) (auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 40 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 41 | lemma fresh_ty: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 42 | fixes a::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 43 | and x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 44 | and T::"ty" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 45 | shows "a\<sharp>T" and "x\<sharp>T" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 46 | by (nominal_induct T rule: ty.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 47 | (auto simp add: fresh_string) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 48 | |
| 63167 | 49 | text \<open>terms\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 50 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 51 | nominal_datatype trm = | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 52 | Ax "name" "coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 53 |   | Cut  "\<guillemotleft>coname\<guillemotright>trm" "\<guillemotleft>name\<guillemotright>trm"            ("Cut <_>._ (_)._" [100,100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 54 |   | NotR "\<guillemotleft>name\<guillemotright>trm" "coname"                 ("NotR (_)._ _" [100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 55 |   | NotL "\<guillemotleft>coname\<guillemotright>trm" "name"                 ("NotL <_>._ _" [100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 56 |   | AndR "\<guillemotleft>coname\<guillemotright>trm" "\<guillemotleft>coname\<guillemotright>trm" "coname" ("AndR <_>._ <_>._ _" [100,100,100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 57 |   | AndL1 "\<guillemotleft>name\<guillemotright>trm" "name"                  ("AndL1 (_)._ _" [100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 58 |   | AndL2 "\<guillemotleft>name\<guillemotright>trm" "name"                  ("AndL2 (_)._ _" [100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 59 |   | OrR1 "\<guillemotleft>coname\<guillemotright>trm" "coname"               ("OrR1 <_>._ _" [100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 60 |   | OrR2 "\<guillemotleft>coname\<guillemotright>trm" "coname"               ("OrR2 <_>._ _" [100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 61 |   | OrL "\<guillemotleft>name\<guillemotright>trm" "\<guillemotleft>name\<guillemotright>trm" "name"        ("OrL (_)._ (_)._ _" [100,100,100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 62 |   | ImpR "\<guillemotleft>name\<guillemotright>(\<guillemotleft>coname\<guillemotright>trm)" "coname"       ("ImpR (_).<_>._ _" [100,100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 63 |   | ImpL "\<guillemotleft>coname\<guillemotright>trm" "\<guillemotleft>name\<guillemotright>trm" "name"     ("ImpL <_>._ (_)._ _" [100,100,100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 64 | |
| 63167 | 65 | text \<open>named terms\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 66 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 67 | nominal_datatype ntrm = Na "\<guillemotleft>name\<guillemotright>trm" ("((_):_)" [100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 68 | |
| 63167 | 69 | text \<open>conamed terms\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 70 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 71 | nominal_datatype ctrm = Co "\<guillemotleft>coname\<guillemotright>trm" ("(<_>:_)" [100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 72 | |
| 63167 | 73 | text \<open>renaming functions\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 74 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 75 | nominal_primrec (freshness_context: "(d::coname,e::coname)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 76 |   crename :: "trm \<Rightarrow> coname \<Rightarrow> coname \<Rightarrow> trm"  ("_[_\<turnstile>c>_]" [100,100,100] 100) 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 77 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 78 | "(Ax x a)[d\<turnstile>c>e] = (if a=d then Ax x e else Ax x a)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 79 | | "\<lbrakk>a\<sharp>(d,e,N);x\<sharp>M\<rbrakk> \<Longrightarrow> (Cut <a>.M (x).N)[d\<turnstile>c>e] = Cut <a>.(M[d\<turnstile>c>e]) (x).(N[d\<turnstile>c>e])" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 80 | | "(NotR (x).M a)[d\<turnstile>c>e] = (if a=d then NotR (x).(M[d\<turnstile>c>e]) e else NotR (x).(M[d\<turnstile>c>e]) a)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 81 | | "a\<sharp>(d,e) \<Longrightarrow> (NotL <a>.M x)[d\<turnstile>c>e] = (NotL <a>.(M[d\<turnstile>c>e]) x)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 82 | | "\<lbrakk>a\<sharp>(d,e,N,c);b\<sharp>(d,e,M,c);b\<noteq>a\<rbrakk> \<Longrightarrow> (AndR <a>.M <b>.N c)[d\<turnstile>c>e] = | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 83 | (if c=d then AndR <a>.(M[d\<turnstile>c>e]) <b>.(N[d \<turnstile>c>e]) e else AndR <a>.(M[d\<turnstile>c>e]) <b>.(N[d\<turnstile>c>e]) c)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 84 | | "x\<sharp>y \<Longrightarrow> (AndL1 (x).M y)[d\<turnstile>c>e] = AndL1 (x).(M[d\<turnstile>c>e]) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 85 | | "x\<sharp>y \<Longrightarrow> (AndL2 (x).M y)[d\<turnstile>c>e] = AndL2 (x).(M[d\<turnstile>c>e]) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 86 | | "a\<sharp>(d,e,b) \<Longrightarrow> (OrR1 <a>.M b)[d\<turnstile>c>e] = (if b=d then OrR1 <a>.(M[d\<turnstile>c>e]) e else OrR1 <a>.(M[d\<turnstile>c>e]) b)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 87 | | "a\<sharp>(d,e,b) \<Longrightarrow> (OrR2 <a>.M b)[d\<turnstile>c>e] = (if b=d then OrR2 <a>.(M[d\<turnstile>c>e]) e else OrR2 <a>.(M[d\<turnstile>c>e]) b)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 88 | | "\<lbrakk>x\<sharp>(N,z);y\<sharp>(M,z);y\<noteq>x\<rbrakk> \<Longrightarrow> (OrL (x).M (y).N z)[d\<turnstile>c>e] = OrL (x).(M[d\<turnstile>c>e]) (y).(N[d\<turnstile>c>e]) z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 89 | | "a\<sharp>(d,e,b) \<Longrightarrow> (ImpR (x).<a>.M b)[d\<turnstile>c>e] = | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 90 | (if b=d then ImpR (x).<a>.(M[d\<turnstile>c>e]) e else ImpR (x).<a>.(M[d\<turnstile>c>e]) b)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 91 | | "\<lbrakk>a\<sharp>(d,e,N);x\<sharp>(M,y)\<rbrakk> \<Longrightarrow> (ImpL <a>.M (x).N y)[d\<turnstile>c>e] = ImpL <a>.(M[d\<turnstile>c>e]) (x).(N[d\<turnstile>c>e]) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 92 | apply(finite_guess)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 93 | apply(rule TrueI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 94 | apply(simp add: abs_fresh abs_supp fin_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 95 | apply(fresh_guess)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 96 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 97 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 98 | nominal_primrec (freshness_context: "(u::name,v::name)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 99 |   nrename :: "trm \<Rightarrow> name \<Rightarrow> name \<Rightarrow> trm"      ("_[_\<turnstile>n>_]" [100,100,100] 100) 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 100 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 101 | "(Ax x a)[u\<turnstile>n>v] = (if x=u then Ax v a else Ax x a)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 102 | | "\<lbrakk>a\<sharp>N;x\<sharp>(u,v,M)\<rbrakk> \<Longrightarrow> (Cut <a>.M (x).N)[u\<turnstile>n>v] = Cut <a>.(M[u\<turnstile>n>v]) (x).(N[u\<turnstile>n>v])" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 103 | | "x\<sharp>(u,v) \<Longrightarrow> (NotR (x).M a)[u\<turnstile>n>v] = NotR (x).(M[u\<turnstile>n>v]) a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 104 | | "(NotL <a>.M x)[u\<turnstile>n>v] = (if x=u then NotL <a>.(M[u\<turnstile>n>v]) v else NotL <a>.(M[u\<turnstile>n>v]) x)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 105 | | "\<lbrakk>a\<sharp>(N,c);b\<sharp>(M,c);b\<noteq>a\<rbrakk> \<Longrightarrow> (AndR <a>.M <b>.N c)[u\<turnstile>n>v] = AndR <a>.(M[u\<turnstile>n>v]) <b>.(N[u\<turnstile>n>v]) c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 106 | | "x\<sharp>(u,v,y) \<Longrightarrow> (AndL1 (x).M y)[u\<turnstile>n>v] = (if y=u then AndL1 (x).(M[u\<turnstile>n>v]) v else AndL1 (x).(M[u\<turnstile>n>v]) y)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 107 | | "x\<sharp>(u,v,y) \<Longrightarrow> (AndL2 (x).M y)[u\<turnstile>n>v] = (if y=u then AndL2 (x).(M[u\<turnstile>n>v]) v else AndL2 (x).(M[u\<turnstile>n>v]) y)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 108 | | "a\<sharp>b \<Longrightarrow> (OrR1 <a>.M b)[u\<turnstile>n>v] = OrR1 <a>.(M[u\<turnstile>n>v]) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 109 | | "a\<sharp>b \<Longrightarrow> (OrR2 <a>.M b)[u\<turnstile>n>v] = OrR2 <a>.(M[u\<turnstile>n>v]) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 110 | | "\<lbrakk>x\<sharp>(u,v,N,z);y\<sharp>(u,v,M,z);y\<noteq>x\<rbrakk> \<Longrightarrow> (OrL (x).M (y).N z)[u\<turnstile>n>v] = | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 111 | (if z=u then OrL (x).(M[u\<turnstile>n>v]) (y).(N[u\<turnstile>n>v]) v else OrL (x).(M[u\<turnstile>n>v]) (y).(N[u\<turnstile>n>v]) z)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 112 | | "\<lbrakk>a\<sharp>b; x\<sharp>(u,v)\<rbrakk> \<Longrightarrow> (ImpR (x).<a>.M b)[u\<turnstile>n>v] = ImpR (x).<a>.(M[u\<turnstile>n>v]) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 113 | | "\<lbrakk>a\<sharp>N;x\<sharp>(u,v,M,y)\<rbrakk> \<Longrightarrow> (ImpL <a>.M (x).N y)[u\<turnstile>n>v] = | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 114 | (if y=u then ImpL <a>.(M[u\<turnstile>n>v]) (x).(N[u\<turnstile>n>v]) v else ImpL <a>.(M[u\<turnstile>n>v]) (x).(N[u\<turnstile>n>v]) y)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 115 | apply(finite_guess)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 116 | apply(rule TrueI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 117 | apply(simp add: abs_fresh abs_supp fs_name1 fs_coname1)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 118 | apply(fresh_guess)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 119 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 120 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 121 | lemmas eq_bij = pt_bij[OF pt_name_inst, OF at_name_inst] pt_bij[OF pt_coname_inst, OF at_coname_inst] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 122 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 123 | lemma crename_name_eqvt[eqvt]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 124 | fixes pi::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 125 | shows "pi\<bullet>(M[d\<turnstile>c>e]) = (pi\<bullet>M)[(pi\<bullet>d)\<turnstile>c>(pi\<bullet>e)]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 126 | apply(nominal_induct M avoiding: d e rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 127 | apply(auto simp add: fresh_bij eq_bij) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 128 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 129 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 130 | lemma crename_coname_eqvt[eqvt]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 131 | fixes pi::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 132 | shows "pi\<bullet>(M[d\<turnstile>c>e]) = (pi\<bullet>M)[(pi\<bullet>d)\<turnstile>c>(pi\<bullet>e)]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 133 | apply(nominal_induct M avoiding: d e rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 134 | apply(auto simp add: fresh_bij eq_bij) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 135 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 136 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 137 | lemma nrename_name_eqvt[eqvt]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 138 | fixes pi::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 139 | shows "pi\<bullet>(M[x\<turnstile>n>y]) = (pi\<bullet>M)[(pi\<bullet>x)\<turnstile>n>(pi\<bullet>y)]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 140 | apply(nominal_induct M avoiding: x y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 141 | apply(auto simp add: fresh_bij eq_bij) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 142 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 143 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 144 | lemma nrename_coname_eqvt[eqvt]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 145 | fixes pi::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 146 | shows "pi\<bullet>(M[x\<turnstile>n>y]) = (pi\<bullet>M)[(pi\<bullet>x)\<turnstile>n>(pi\<bullet>y)]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 147 | apply(nominal_induct M avoiding: x y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 148 | apply(auto simp add: fresh_bij eq_bij) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 149 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 150 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 151 | lemmas rename_eqvts = crename_name_eqvt crename_coname_eqvt | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 152 | nrename_name_eqvt nrename_coname_eqvt | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 153 | lemma nrename_fresh: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 154 | assumes a: "x\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 155 | shows "M[x\<turnstile>n>y] = M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 156 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 157 | by (nominal_induct M avoiding: x y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 158 | (auto simp add: trm.inject fresh_atm abs_fresh fin_supp abs_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 159 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 160 | lemma crename_fresh: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 161 | assumes a: "a\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 162 | shows "M[a\<turnstile>c>b] = M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 163 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 164 | by (nominal_induct M avoiding: a b rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 165 | (auto simp add: trm.inject fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 166 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 167 | lemma nrename_nfresh: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 168 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 169 | shows "x\<sharp>y\<Longrightarrow>x\<sharp>M[x\<turnstile>n>y]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 170 | by (nominal_induct M avoiding: x y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 171 | (auto simp add: fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 172 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 173 | lemma crename_nfresh: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 174 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 175 | shows "x\<sharp>M\<Longrightarrow>x\<sharp>M[a\<turnstile>c>b]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 176 | by (nominal_induct M avoiding: a b rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 177 | (auto simp add: fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 178 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 179 | lemma crename_cfresh: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 180 | fixes a::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 181 | shows "a\<sharp>b\<Longrightarrow>a\<sharp>M[a\<turnstile>c>b]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 182 | by (nominal_induct M avoiding: a b rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 183 | (auto simp add: fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 184 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 185 | lemma nrename_cfresh: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 186 | fixes c::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 187 | shows "c\<sharp>M\<Longrightarrow>c\<sharp>M[x\<turnstile>n>y]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 188 | by (nominal_induct M avoiding: x y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 189 | (auto simp add: fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 190 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 191 | lemma nrename_nfresh': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 192 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 193 | shows "x\<sharp>(M,z,y)\<Longrightarrow>x\<sharp>M[z\<turnstile>n>y]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 194 | by (nominal_induct M avoiding: x z y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 195 | (auto simp add: fresh_prod fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 196 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 197 | lemma crename_cfresh': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 198 | fixes a::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 199 | shows "a\<sharp>(M,b,c)\<Longrightarrow>a\<sharp>M[b\<turnstile>c>c]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 200 | by (nominal_induct M avoiding: a b c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 201 | (auto simp add: fresh_prod fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 202 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 203 | lemma nrename_rename: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 204 | assumes a: "x'\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 205 | shows "([(x',x)]\<bullet>M)[x'\<turnstile>n>y]= M[x\<turnstile>n>y]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 206 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 207 | apply(nominal_induct M avoiding: x x' y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 208 | apply(auto simp add: abs_fresh fresh_bij fresh_atm fresh_prod fresh_right calc_atm abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 209 | apply(auto simp add: fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 210 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 211 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 212 | lemma crename_rename: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 213 | assumes a: "a'\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 214 | shows "([(a',a)]\<bullet>M)[a'\<turnstile>c>b]= M[a\<turnstile>c>b]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 215 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 216 | apply(nominal_induct M avoiding: a a' b rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 217 | apply(auto simp add: abs_fresh fresh_bij fresh_atm fresh_prod fresh_right calc_atm abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 218 | apply(auto simp add: fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 219 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 220 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 221 | lemmas rename_fresh = nrename_fresh crename_fresh | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 222 | nrename_nfresh crename_nfresh crename_cfresh nrename_cfresh | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 223 | nrename_nfresh' crename_cfresh' | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 224 | nrename_rename crename_rename | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 225 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 226 | lemma better_nrename_Cut: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 227 | assumes a: "x\<sharp>(u,v)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 228 | shows "(Cut <a>.M (x).N)[u\<turnstile>n>v] = Cut <a>.(M[u\<turnstile>n>v]) (x).(N[u\<turnstile>n>v])" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 229 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 230 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,a,x,u,v)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 231 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,a,x,u,v)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 232 | have eq1: "(Cut <a>.M (x).N) = (Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 233 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 234 | have "(Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N))[u\<turnstile>n>v] = | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 235 | Cut <a'>.(([(a',a)]\<bullet>M)[u\<turnstile>n>v]) (x').(([(x',x)]\<bullet>N)[u\<turnstile>n>v])" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 236 | using fs1 fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 237 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 238 | apply(rule nrename.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 239 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 240 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 241 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 242 | also have "\<dots> = Cut <a>.(M[u\<turnstile>n>v]) (x).(N[u\<turnstile>n>v])" using fs1 fs2 a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 243 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 244 | apply(simp add: trm.inject alpha fresh_atm fresh_prod rename_eqvts) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 245 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 246 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 247 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 248 | finally show "(Cut <a>.M (x).N)[u\<turnstile>n>v] = Cut <a>.(M[u\<turnstile>n>v]) (x).(N[u\<turnstile>n>v])" using eq1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 249 | by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 250 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 251 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 252 | lemma better_crename_Cut: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 253 | assumes a: "a\<sharp>(b,c)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 254 | shows "(Cut <a>.M (x).N)[b\<turnstile>c>c] = Cut <a>.(M[b\<turnstile>c>c]) (x).(N[b\<turnstile>c>c])" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 255 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 256 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,a,x,b,c)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 257 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,a,x,b,c)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 258 | have eq1: "(Cut <a>.M (x).N) = (Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 259 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 260 | have "(Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N))[b\<turnstile>c>c] = | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 261 | Cut <a'>.(([(a',a)]\<bullet>M)[b\<turnstile>c>c]) (x').(([(x',x)]\<bullet>N)[b\<turnstile>c>c])" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 262 | using fs1 fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 263 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 264 | apply(rule crename.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 265 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 266 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 267 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 268 | also have "\<dots> = Cut <a>.(M[b\<turnstile>c>c]) (x).(N[b\<turnstile>c>c])" using fs1 fs2 a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 269 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 270 | apply(simp add: trm.inject alpha fresh_atm fresh_prod rename_eqvts) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 271 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 272 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 273 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 274 | finally show "(Cut <a>.M (x).N)[b\<turnstile>c>c] = Cut <a>.(M[b\<turnstile>c>c]) (x).(N[b\<turnstile>c>c])" using eq1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 275 | by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 276 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 277 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 278 | lemma crename_id: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 279 | shows "M[a\<turnstile>c>a] = M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 280 | by (nominal_induct M avoiding: a rule: trm.strong_induct) (auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 281 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 282 | lemma nrename_id: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 283 | shows "M[x\<turnstile>n>x] = M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 284 | by (nominal_induct M avoiding: x rule: trm.strong_induct) (auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 285 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 286 | lemma nrename_swap: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 287 | shows "x\<sharp>M \<Longrightarrow> [(x,y)]\<bullet>M = M[y\<turnstile>n>x]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 288 | by (nominal_induct M avoiding: x y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 289 | (simp_all add: calc_atm fresh_atm trm.inject alpha abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 290 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 291 | lemma crename_swap: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 292 | shows "a\<sharp>M \<Longrightarrow> [(a,b)]\<bullet>M = M[b\<turnstile>c>a]" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 293 | by (nominal_induct M avoiding: a b rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 294 | (simp_all add: calc_atm fresh_atm trm.inject alpha abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 295 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 296 | lemma crename_ax: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 297 | assumes a: "M[a\<turnstile>c>b] = Ax x c" "c\<noteq>a" "c\<noteq>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 298 | shows "M = Ax x c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 299 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 300 | apply(nominal_induct M avoiding: a b x c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 301 | apply(simp_all add: trm.inject split: if_splits) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 302 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 303 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 304 | lemma nrename_ax: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 305 | assumes a: "M[x\<turnstile>n>y] = Ax z a" "z\<noteq>x" "z\<noteq>y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 306 | shows "M = Ax z a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 307 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 308 | apply(nominal_induct M avoiding: x y z a rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 309 | apply(simp_all add: trm.inject split: if_splits) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 310 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 311 | |
| 63167 | 312 | text \<open>substitution functions\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 313 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 314 | lemma fresh_perm_coname: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 315 | fixes c::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 316 | and pi::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 317 | and M::"trm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 318 | assumes a: "c\<sharp>pi" "c\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 319 | shows "c\<sharp>(pi\<bullet>M)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 320 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 321 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 322 | apply(simp add: fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 323 | apply(simp add: at_prm_fresh[OF at_coname_inst] fresh_list_rev) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 324 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 325 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 326 | lemma fresh_perm_name: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 327 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 328 | and pi::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 329 | and M::"trm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 330 | assumes a: "x\<sharp>pi" "x\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 331 | shows "x\<sharp>(pi\<bullet>M)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 332 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 333 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 334 | apply(simp add: fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 335 | apply(simp add: at_prm_fresh[OF at_name_inst] fresh_list_rev) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 336 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 337 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 338 | lemma fresh_fun_simp_NotL: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 339 | assumes a: "x'\<sharp>P" "x'\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 340 | shows "fresh_fun (\<lambda>x'. Cut <c>.P (x').NotL <a>.M x') = Cut <c>.P (x').NotL <a>.M x'" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 341 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 342 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 343 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 344 | apply(rule pt_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 345 | apply(rule at_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 346 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 347 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(c,P,a,M)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 348 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 349 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 350 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 351 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 352 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 353 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 354 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 355 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 356 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 357 | lemma fresh_fun_NotL[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 358 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 359 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 360 | shows "pi1\<bullet>fresh_fun (\<lambda>x'. Cut <c>.P (x').NotL <a>.M x')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 361 | fresh_fun (pi1\<bullet>(\<lambda>x'. Cut <c>.P (x').NotL <a>.M x'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 362 | and "pi2\<bullet>fresh_fun (\<lambda>x'. Cut <c>.P (x').NotL <a>.M x')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 363 | fresh_fun (pi2\<bullet>(\<lambda>x'. Cut <c>.P (x').NotL <a>.M x'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 364 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 365 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 366 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 367 | apply(auto simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 368 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 369 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 370 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 371 | apply(rule fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 372 | apply(rule fresh_perm_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 373 | apply(assumption) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 374 | apply(assumption) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 375 | apply(rule fresh_perm_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 376 | apply(assumption) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 377 | apply(assumption) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 378 | apply(simp add: at_prm_fresh[OF at_name_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 379 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 380 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,pi2\<bullet>P,pi2\<bullet>M,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 381 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 382 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 383 | apply(simp add: fresh_fun_simp_NotL calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 384 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 385 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 386 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 387 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 388 | lemma fresh_fun_simp_AndL1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 389 | assumes a: "z'\<sharp>P" "z'\<sharp>M" "z'\<sharp>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 390 | shows "fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL1 (x).M z') = Cut <c>.P (z').AndL1 (x).M z'" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 391 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 392 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 393 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 394 | apply(rule pt_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 395 | apply(rule at_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 396 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 397 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(c,P,x,M)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 398 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 399 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 400 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 401 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 402 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 403 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 404 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 405 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 406 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 407 | lemma fresh_fun_AndL1[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 408 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 409 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 410 | shows "pi1\<bullet>fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL1 (x).M z')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 411 | fresh_fun (pi1\<bullet>(\<lambda>z'. Cut <c>.P (z').AndL1 (x).M z'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 412 | and "pi2\<bullet>fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL1 (x).M z')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 413 | fresh_fun (pi2\<bullet>(\<lambda>z'. Cut <c>.P (z').AndL1 (x).M z'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 414 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 415 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 416 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,x,pi1\<bullet>P,pi1\<bullet>M,pi1\<bullet>x,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 417 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 418 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 419 | apply(simp add: fresh_fun_simp_AndL1 at_prm_fresh[OF at_name_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 420 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 421 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 422 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 423 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,x,pi2\<bullet>P,pi2\<bullet>M,pi2\<bullet>x,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 424 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 425 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 426 | apply(simp add: fresh_fun_simp_AndL1 calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 427 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 428 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 429 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 430 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 431 | lemma fresh_fun_simp_AndL2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 432 | assumes a: "z'\<sharp>P" "z'\<sharp>M" "z'\<sharp>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 433 | shows "fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL2 (x).M z') = Cut <c>.P (z').AndL2 (x).M z'" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 434 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 435 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 436 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 437 | apply(rule pt_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 438 | apply(rule at_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 439 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 440 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(c,P,x,M)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 441 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 442 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 443 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 444 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 445 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 446 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 447 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 448 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 449 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 450 | lemma fresh_fun_AndL2[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 451 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 452 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 453 | shows "pi1\<bullet>fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL2 (x).M z')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 454 | fresh_fun (pi1\<bullet>(\<lambda>z'. Cut <c>.P (z').AndL2 (x).M z'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 455 | and "pi2\<bullet>fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL2 (x).M z')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 456 | fresh_fun (pi2\<bullet>(\<lambda>z'. Cut <c>.P (z').AndL2 (x).M z'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 457 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 458 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 459 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,x,pi1\<bullet>P,pi1\<bullet>M,pi1\<bullet>x,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 460 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 461 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 462 | apply(simp add: fresh_fun_simp_AndL2 at_prm_fresh[OF at_name_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 463 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 464 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 465 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 466 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,x,pi2\<bullet>P,pi2\<bullet>M,pi2\<bullet>x,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 467 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 468 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 469 | apply(simp add: fresh_fun_simp_AndL2 calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 470 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 471 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 472 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 473 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 474 | lemma fresh_fun_simp_OrL: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 475 | assumes a: "z'\<sharp>P" "z'\<sharp>M" "z'\<sharp>N" "z'\<sharp>u" "z'\<sharp>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 476 | shows "fresh_fun (\<lambda>z'. Cut <c>.P (z').OrL (x).M (u).N z') = Cut <c>.P (z').OrL (x).M (u).N z'" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 477 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 478 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 479 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 480 | apply(rule pt_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 481 | apply(rule at_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 482 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 483 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(c,P,x,M,u,N)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 484 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 485 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 486 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 487 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 488 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 489 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 490 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 491 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 492 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 493 | lemma fresh_fun_OrL[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 494 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 495 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 496 | shows "pi1\<bullet>fresh_fun (\<lambda>z'. Cut <c>.P (z').OrL (x).M (u).N z')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 497 | fresh_fun (pi1\<bullet>(\<lambda>z'. Cut <c>.P (z').OrL (x).M (u).N z'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 498 | and "pi2\<bullet>fresh_fun (\<lambda>z'. Cut <c>.P (z').OrL (x).M (u).N z')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 499 | fresh_fun (pi2\<bullet>(\<lambda>z'. Cut <c>.P (z').OrL (x).M (u).N z'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 500 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 501 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 502 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,N,x,u,pi1\<bullet>P,pi1\<bullet>M,pi1\<bullet>N,pi1\<bullet>x,pi1\<bullet>u,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 503 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 504 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 505 | apply(simp add: fresh_fun_simp_OrL at_prm_fresh[OF at_name_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 506 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 507 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 508 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 509 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,N,x,u,pi2\<bullet>P,pi2\<bullet>M,pi2\<bullet>N,pi2\<bullet>x,pi2\<bullet>u,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 510 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 511 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 512 | apply(simp add: fresh_fun_simp_OrL calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 513 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 514 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 515 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 516 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 517 | lemma fresh_fun_simp_ImpL: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 518 | assumes a: "z'\<sharp>P" "z'\<sharp>M" "z'\<sharp>N" "z'\<sharp>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 519 | shows "fresh_fun (\<lambda>z'. Cut <c>.P (z').ImpL <a>.M (x).N z') = Cut <c>.P (z').ImpL <a>.M (x).N z'" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 520 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 521 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 522 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 523 | apply(rule pt_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 524 | apply(rule at_name_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 525 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 526 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(c,P,x,M,N)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 527 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 528 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 529 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 530 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 531 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 532 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 533 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 534 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 535 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 536 | lemma fresh_fun_ImpL[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 537 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 538 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 539 | shows "pi1\<bullet>fresh_fun (\<lambda>z'. Cut <c>.P (z').ImpL <a>.M (x).N z')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 540 | fresh_fun (pi1\<bullet>(\<lambda>z'. Cut <c>.P (z').ImpL <a>.M (x).N z'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 541 | and "pi2\<bullet>fresh_fun (\<lambda>z'. Cut <c>.P (z').ImpL <a>.M (x).N z')= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 542 | fresh_fun (pi2\<bullet>(\<lambda>z'. Cut <c>.P (z').ImpL <a>.M (x).N z'))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 543 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 544 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 545 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,N,x,pi1\<bullet>P,pi1\<bullet>M,pi1\<bullet>N,pi1\<bullet>x,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 546 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 547 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 548 | apply(simp add: fresh_fun_simp_ImpL at_prm_fresh[OF at_name_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 549 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 550 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 551 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 552 | apply(subgoal_tac "\<exists>n::name. n\<sharp>(P,M,N,x,pi2\<bullet>P,pi2\<bullet>M,pi2\<bullet>N,pi2\<bullet>x,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 553 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 554 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 555 | apply(simp add: fresh_fun_simp_ImpL calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 556 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 557 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 558 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 559 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 560 | lemma fresh_fun_simp_NotR: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 561 | assumes a: "a'\<sharp>P" "a'\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 562 | shows "fresh_fun (\<lambda>a'. Cut <a'>.(NotR (y).M a') (x).P) = Cut <a'>.(NotR (y).M a') (x).P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 563 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 564 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 565 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 566 | apply(rule pt_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 567 | apply(rule at_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 568 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 569 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(x,P,y,M)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 570 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 571 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 572 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 573 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 574 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 575 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 576 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 577 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 578 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 579 | lemma fresh_fun_NotR[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 580 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 581 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 582 | shows "pi1\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(NotR (y).M a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 583 | fresh_fun (pi1\<bullet>(\<lambda>a'. Cut <a'>.(NotR (y).M a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 584 | and "pi2\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(NotR (y).M a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 585 | fresh_fun (pi2\<bullet>(\<lambda>a'. Cut <a'>.(NotR (y).M a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 586 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 587 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 588 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,pi1\<bullet>P,pi1\<bullet>M,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 589 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 590 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 591 | apply(simp add: fresh_fun_simp_NotR calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 592 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 593 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 594 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 595 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,pi2\<bullet>P,pi2\<bullet>M,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 596 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 597 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 598 | apply(simp add: fresh_fun_simp_NotR at_prm_fresh[OF at_coname_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 599 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 600 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 601 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 602 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 603 | lemma fresh_fun_simp_AndR: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 604 | assumes a: "a'\<sharp>P" "a'\<sharp>M" "a'\<sharp>N" "a'\<sharp>b" "a'\<sharp>c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 605 | shows "fresh_fun (\<lambda>a'. Cut <a'>.(AndR <b>.M <c>.N a') (x).P) = Cut <a'>.(AndR <b>.M <c>.N a') (x).P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 606 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 607 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 608 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 609 | apply(rule pt_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 610 | apply(rule at_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 611 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 612 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(x,P,b,M,c,N)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 613 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 614 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 615 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 616 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 617 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 618 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 619 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 620 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 621 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 622 | lemma fresh_fun_AndR[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 623 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 624 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 625 | shows "pi1\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(AndR <b>.M <c>.N a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 626 | fresh_fun (pi1\<bullet>(\<lambda>a'. Cut <a'>.(AndR <b>.M <c>.N a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 627 | and "pi2\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(AndR <b>.M <c>.N a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 628 | fresh_fun (pi2\<bullet>(\<lambda>a'. Cut <a'>.(AndR <b>.M <c>.N a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 629 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 630 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 631 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,N,b,c,pi1\<bullet>P,pi1\<bullet>M,pi1\<bullet>N,pi1\<bullet>b,pi1\<bullet>c,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 632 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 633 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 634 | apply(simp add: fresh_fun_simp_AndR calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 635 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 636 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 637 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 638 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,N,b,c,pi2\<bullet>P,pi2\<bullet>M,pi2\<bullet>N,pi2\<bullet>b,pi2\<bullet>c,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 639 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 640 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 641 | apply(simp add: fresh_fun_simp_AndR at_prm_fresh[OF at_coname_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 642 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 643 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 644 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 645 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 646 | lemma fresh_fun_simp_OrR1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 647 | assumes a: "a'\<sharp>P" "a'\<sharp>M" "a'\<sharp>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 648 | shows "fresh_fun (\<lambda>a'. Cut <a'>.(OrR1 <b>.M a') (x).P) = Cut <a'>.(OrR1 <b>.M a') (x).P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 649 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 650 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 651 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 652 | apply(rule pt_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 653 | apply(rule at_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 654 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 655 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(x,P,b,M)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 656 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 657 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 658 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 659 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 660 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 661 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 662 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 663 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 664 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 665 | lemma fresh_fun_OrR1[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 666 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 667 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 668 | shows "pi1\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(OrR1 <b>.M a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 669 | fresh_fun (pi1\<bullet>(\<lambda>a'. Cut <a'>.(OrR1 <b>.M a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 670 | and "pi2\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(OrR1 <b>.M a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 671 | fresh_fun (pi2\<bullet>(\<lambda>a'. Cut <a'>.(OrR1 <b>.M a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 672 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 673 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 674 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,b,pi1\<bullet>P,pi1\<bullet>M,pi1\<bullet>b,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 675 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 676 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 677 | apply(simp add: fresh_fun_simp_OrR1 calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 678 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 679 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 680 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 681 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,b,pi2\<bullet>P,pi2\<bullet>M,pi2\<bullet>b,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 682 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 683 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 684 | apply(simp add: fresh_fun_simp_OrR1 at_prm_fresh[OF at_coname_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 685 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 686 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 687 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 688 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 689 | lemma fresh_fun_simp_OrR2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 690 | assumes a: "a'\<sharp>P" "a'\<sharp>M" "a'\<sharp>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 691 | shows "fresh_fun (\<lambda>a'. Cut <a'>.(OrR2 <b>.M a') (x).P) = Cut <a'>.(OrR2 <b>.M a') (x).P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 692 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 693 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 694 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 695 | apply(rule pt_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 696 | apply(rule at_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 697 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 698 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(x,P,b,M)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 699 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 700 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 701 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 702 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 703 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 704 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 705 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 706 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 707 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 708 | lemma fresh_fun_OrR2[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 709 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 710 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 711 | shows "pi1\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(OrR2 <b>.M a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 712 | fresh_fun (pi1\<bullet>(\<lambda>a'. Cut <a'>.(OrR2 <b>.M a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 713 | and "pi2\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(OrR2 <b>.M a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 714 | fresh_fun (pi2\<bullet>(\<lambda>a'. Cut <a'>.(OrR2 <b>.M a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 715 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 716 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 717 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,b,pi1\<bullet>P,pi1\<bullet>M,pi1\<bullet>b,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 718 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 719 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 720 | apply(simp add: fresh_fun_simp_OrR2 calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 721 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 722 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 723 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 724 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,b,pi2\<bullet>P,pi2\<bullet>M,pi2\<bullet>b,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 725 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 726 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 727 | apply(simp add: fresh_fun_simp_OrR2 at_prm_fresh[OF at_coname_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 728 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 729 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 730 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 731 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 732 | lemma fresh_fun_simp_ImpR: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 733 | assumes a: "a'\<sharp>P" "a'\<sharp>M" "a'\<sharp>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 734 | shows "fresh_fun (\<lambda>a'. Cut <a'>.(ImpR (y).<b>.M a') (x).P) = Cut <a'>.(ImpR (y).<b>.M a') (x).P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 735 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 736 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 737 | apply(rule fresh_fun_app) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 738 | apply(rule pt_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 739 | apply(rule at_coname_inst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 740 | apply(finite_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 741 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(x,P,y,b,M)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 742 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 743 | apply(rule_tac x="n" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 744 | apply(simp add: fresh_prod abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 745 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 746 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 747 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 748 | apply(fresh_guess) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 749 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 750 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 751 | lemma fresh_fun_ImpR[eqvt_force]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 752 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 753 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 754 | shows "pi1\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(ImpR (y).<b>.M a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 755 | fresh_fun (pi1\<bullet>(\<lambda>a'. Cut <a'>.(ImpR (y).<b>.M a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 756 | and "pi2\<bullet>fresh_fun (\<lambda>a'. Cut <a'>.(ImpR (y).<b>.M a') (x).P)= | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 757 | fresh_fun (pi2\<bullet>(\<lambda>a'. Cut <a'>.(ImpR (y).<b>.M a') (x).P))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 758 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 759 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 760 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,b,pi1\<bullet>P,pi1\<bullet>M,pi1\<bullet>b,pi1)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 761 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 762 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 763 | apply(simp add: fresh_fun_simp_ImpR calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 764 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 765 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 766 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 767 | apply(subgoal_tac "\<exists>n::coname. n\<sharp>(P,M,b,pi2\<bullet>P,pi2\<bullet>M,pi2\<bullet>b,pi2)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 768 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 769 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 770 | apply(simp add: fresh_fun_simp_ImpR at_prm_fresh[OF at_coname_inst] swap_simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 771 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 772 | apply(simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 773 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 774 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 775 | nominal_primrec (freshness_context: "(y::name,c::coname,P::trm)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 776 |   substn :: "trm \<Rightarrow> name   \<Rightarrow> coname \<Rightarrow> trm \<Rightarrow> trm" ("_{_:=<_>._}" [100,100,100,100] 100) 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 777 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 778 |   "(Ax x a){y:=<c>.P} = (if x=y then Cut <c>.P (y).Ax y a else Ax x a)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 779 | | "\<lbrakk>a\<sharp>(c,P,N);x\<sharp>(y,P,M)\<rbrakk> \<Longrightarrow> (Cut <a>.M (x).N){y:=<c>.P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 780 |   (if M=Ax y a then Cut <c>.P (x).(N{y:=<c>.P}) else Cut <a>.(M{y:=<c>.P}) (x).(N{y:=<c>.P}))" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 781 | | "x\<sharp>(y,P) \<Longrightarrow> (NotR (x).M a){y:=<c>.P} = NotR (x).(M{y:=<c>.P}) a" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 782 | | "a\<sharp>(c,P) \<Longrightarrow> (NotL <a>.M x){y:=<c>.P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 783 |   (if x=y then fresh_fun (\<lambda>x'. Cut <c>.P (x').NotL <a>.(M{y:=<c>.P}) x') else NotL <a>.(M{y:=<c>.P}) x)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 784 | | "\<lbrakk>a\<sharp>(c,P,N,d);b\<sharp>(c,P,M,d);b\<noteq>a\<rbrakk> \<Longrightarrow> | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 785 |   (AndR <a>.M <b>.N d){y:=<c>.P} = AndR <a>.(M{y:=<c>.P}) <b>.(N{y:=<c>.P}) d" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 786 | | "x\<sharp>(y,P,z) \<Longrightarrow> (AndL1 (x).M z){y:=<c>.P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 787 |   (if z=y then fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL1 (x).(M{y:=<c>.P}) z') 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 788 |    else AndL1 (x).(M{y:=<c>.P}) z)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 789 | | "x\<sharp>(y,P,z) \<Longrightarrow> (AndL2 (x).M z){y:=<c>.P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 790 |   (if z=y then fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL2 (x).(M{y:=<c>.P}) z') 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 791 |    else AndL2 (x).(M{y:=<c>.P}) z)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 792 | | "a\<sharp>(c,P,b) \<Longrightarrow> (OrR1 <a>.M b){y:=<c>.P} = OrR1 <a>.(M{y:=<c>.P}) b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 793 | | "a\<sharp>(c,P,b) \<Longrightarrow> (OrR2 <a>.M b){y:=<c>.P} = OrR2 <a>.(M{y:=<c>.P}) b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 794 | | "\<lbrakk>x\<sharp>(y,N,P,z);u\<sharp>(y,M,P,z);x\<noteq>u\<rbrakk> \<Longrightarrow> (OrL (x).M (u).N z){y:=<c>.P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 795 |   (if z=y then fresh_fun (\<lambda>z'. Cut <c>.P (z').OrL (x).(M{y:=<c>.P}) (u).(N{y:=<c>.P}) z') 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 796 |    else OrL (x).(M{y:=<c>.P}) (u).(N{y:=<c>.P}) z)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 797 | | "\<lbrakk>a\<sharp>(b,c,P); x\<sharp>(y,P)\<rbrakk> \<Longrightarrow> (ImpR (x).<a>.M b){y:=<c>.P} = ImpR (x).<a>.(M{y:=<c>.P}) b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 798 | | "\<lbrakk>a\<sharp>(N,c,P);x\<sharp>(y,P,M,z)\<rbrakk> \<Longrightarrow> (ImpL <a>.M (x).N z){y:=<c>.P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 799 |   (if y=z then fresh_fun (\<lambda>z'. Cut <c>.P (z').ImpL <a>.(M{y:=<c>.P}) (x).(N{y:=<c>.P}) z') 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 800 |    else ImpL <a>.(M{y:=<c>.P}) (x).(N{y:=<c>.P}) z)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 801 | apply(finite_guess)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 802 | apply(rule TrueI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 803 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 804 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 805 | apply(subgoal_tac "\<exists>x::name. x\<sharp>(x1,P,y1)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 806 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 807 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 808 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 809 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 810 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 811 | apply(subgoal_tac "\<exists>x::name. x\<sharp>(x1,P,y1)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 812 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 813 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 814 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 815 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 816 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 817 | apply(subgoal_tac "\<exists>x::name. x\<sharp>(x1,P,y1)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 818 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 819 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 820 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 821 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 822 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 823 | apply(subgoal_tac "\<exists>x::name. x\<sharp>(x1,P,y1,x3,y2)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 824 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 825 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 826 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 827 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 828 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 829 | apply(subgoal_tac "\<exists>x::name. x\<sharp>(x1,P,y1,x3,y2)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 830 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 831 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 832 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 833 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 834 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 835 | apply(subgoal_tac "\<exists>x::name. x\<sharp>(x3,P,y1,y2)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 836 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 837 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 838 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 839 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 840 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 841 | apply(subgoal_tac "\<exists>x::name. x\<sharp>(x3,P,y1,y2)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 842 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 843 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 844 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 845 | apply(fresh_guess)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 846 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 847 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 848 | nominal_primrec (freshness_context: "(d::name,z::coname,P::trm)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 849 |   substc :: "trm \<Rightarrow> coname \<Rightarrow> name   \<Rightarrow> trm \<Rightarrow> trm" ("_{_:=(_)._}" [100,100,100,100] 100)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 850 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 851 |   "(Ax x a){d:=(z).P} = (if d=a then Cut <a>.(Ax x a) (z).P else Ax x a)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 852 | | "\<lbrakk>a\<sharp>(d,P,N);x\<sharp>(z,P,M)\<rbrakk> \<Longrightarrow> (Cut <a>.M (x).N){d:=(z).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 853 |   (if N=Ax x d then Cut <a>.(M{d:=(z).P}) (z).P else Cut <a>.(M{d:=(z).P}) (x).(N{d:=(z).P}))" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 854 | | "x\<sharp>(z,P) \<Longrightarrow> (NotR (x).M a){d:=(z).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 855 |   (if d=a then fresh_fun (\<lambda>a'. Cut <a'>.NotR (x).(M{d:=(z).P}) a' (z).P) else NotR (x).(M{d:=(z).P}) a)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 856 | | "a\<sharp>(d,P) \<Longrightarrow> (NotL <a>.M x){d:=(z).P} = NotL <a>.(M{d:=(z).P}) x" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 857 | | "\<lbrakk>a\<sharp>(P,c,N,d);b\<sharp>(P,c,M,d);b\<noteq>a\<rbrakk> \<Longrightarrow> (AndR <a>.M <b>.N c){d:=(z).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 858 |   (if d=c then fresh_fun (\<lambda>a'. Cut <a'>.(AndR <a>.(M{d:=(z).P}) <b>.(N{d:=(z).P}) a') (z).P)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 859 |    else AndR <a>.(M{d:=(z).P}) <b>.(N{d:=(z).P}) c)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 860 | | "x\<sharp>(y,z,P) \<Longrightarrow> (AndL1 (x).M y){d:=(z).P} = AndL1 (x).(M{d:=(z).P}) y"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 861 | | "x\<sharp>(y,P,z) \<Longrightarrow> (AndL2 (x).M y){d:=(z).P} = AndL2 (x).(M{d:=(z).P}) y"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 862 | | "a\<sharp>(d,P,b) \<Longrightarrow> (OrR1 <a>.M b){d:=(z).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 863 |   (if d=b then fresh_fun (\<lambda>a'. Cut <a'>.OrR1 <a>.(M{d:=(z).P}) a' (z).P) else OrR1 <a>.(M{d:=(z).P}) b)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 864 | | "a\<sharp>(d,P,b) \<Longrightarrow> (OrR2 <a>.M b){d:=(z).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 865 |   (if d=b then fresh_fun (\<lambda>a'. Cut <a'>.OrR2 <a>.(M{d:=(z).P}) a' (z).P) else OrR2 <a>.(M{d:=(z).P}) b)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 866 | | "\<lbrakk>x\<sharp>(N,z,P,u);y\<sharp>(M,z,P,u);x\<noteq>y\<rbrakk> \<Longrightarrow> (OrL (x).M (y).N u){d:=(z).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 867 |   OrL (x).(M{d:=(z).P}) (y).(N{d:=(z).P}) u" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 868 | | "\<lbrakk>a\<sharp>(b,d,P); x\<sharp>(z,P)\<rbrakk> \<Longrightarrow> (ImpR (x).<a>.M b){d:=(z).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 869 |   (if d=b then fresh_fun (\<lambda>a'. Cut <a'>.ImpR (x).<a>.(M{d:=(z).P}) a' (z).P) 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 870 |    else ImpR (x).<a>.(M{d:=(z).P}) b)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 871 | | "\<lbrakk>a\<sharp>(N,d,P);x\<sharp>(y,z,P,M)\<rbrakk> \<Longrightarrow> (ImpL <a>.M (x).N y){d:=(z).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 872 |   ImpL <a>.(M{d:=(z).P}) (x).(N{d:=(z).P}) y"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 873 | apply(finite_guess)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 874 | apply(rule TrueI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 875 | apply(simp add: abs_fresh abs_supp fs_name1 fs_coname1)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 876 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 877 | apply(subgoal_tac "\<exists>x::coname. x\<sharp>(x1,P,y1)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 878 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 879 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 880 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 881 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 882 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 883 | apply(subgoal_tac "\<exists>x::coname. x\<sharp>(x1,P,y1,x3,y2)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 884 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 885 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 886 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 887 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 888 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 889 | apply(subgoal_tac "\<exists>x::coname. x\<sharp>(x1,P,y1,x3,y2)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 890 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 891 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 892 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 893 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 894 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 895 | apply(subgoal_tac "\<exists>x::coname. x\<sharp>(x1,P,y1)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 896 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 897 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 898 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 899 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 900 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 901 | apply(subgoal_tac "\<exists>x::coname. x\<sharp>(x1,P,y1)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 902 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 903 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 904 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 905 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 906 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 907 | apply(subgoal_tac "\<exists>x::coname. x\<sharp>(x1,P,x2,y1)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 908 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 909 | apply(simp add: fresh_fun_simp_ImpR abs_fresh fresh_atm abs_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 910 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 911 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 912 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 913 | apply(subgoal_tac "\<exists>x::coname. x\<sharp>(x1,P,x2,y1)", erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 914 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 915 | apply(simp add: fresh_fun_simp_ImpR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 916 | apply(rule exists_fresh', simp add: fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 917 | apply(simp add: abs_fresh abs_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 918 | apply(fresh_guess add: abs_fresh fresh_prod)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 919 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 920 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 921 | lemma csubst_eqvt[eqvt]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 922 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 923 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 924 |   shows "pi1\<bullet>(M{c:=(x).N}) = (pi1\<bullet>M){(pi1\<bullet>c):=(pi1\<bullet>x).(pi1\<bullet>N)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 925 |   and   "pi2\<bullet>(M{c:=(x).N}) = (pi2\<bullet>M){(pi2\<bullet>c):=(pi2\<bullet>x).(pi2\<bullet>N)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 926 | apply(nominal_induct M avoiding: c x N rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 927 | apply(auto simp add: eq_bij fresh_bij eqvts) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 928 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 929 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 930 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 931 | lemma nsubst_eqvt[eqvt]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 932 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 933 | and pi2::"coname prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 934 |   shows "pi1\<bullet>(M{x:=<c>.N}) = (pi1\<bullet>M){(pi1\<bullet>x):=<(pi1\<bullet>c)>.(pi1\<bullet>N)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 935 |   and   "pi2\<bullet>(M{x:=<c>.N}) = (pi2\<bullet>M){(pi2\<bullet>x):=<(pi2\<bullet>c)>.(pi2\<bullet>N)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 936 | apply(nominal_induct M avoiding: c x N rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 937 | apply(auto simp add: eq_bij fresh_bij eqvts) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 938 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 939 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 940 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 941 | lemma supp_subst1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 942 |   shows "supp (M{y:=<c>.P}) \<subseteq> ((supp M) - {y}) \<union> (supp P)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 943 | apply(nominal_induct M avoiding: y P c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 944 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 945 | apply(auto simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 946 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 947 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 948 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 949 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 950 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 951 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 952 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 953 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 954 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 955 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 956 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 957 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 958 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 959 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 960 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 961 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 962 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 963 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 964 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 965 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 966 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 967 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 968 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 969 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 970 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 971 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 972 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 973 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 974 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 975 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 976 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 977 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 978 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 979 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 980 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 981 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 982 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 983 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 984 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 985 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 986 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 987 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 988 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 989 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 990 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 991 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 992 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 993 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 994 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 995 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 996 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 997 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 998 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 999 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1000 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1001 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1002 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1003 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1004 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1005 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1006 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1007 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1008 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1009 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1010 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1011 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1012 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1013 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1014 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1015 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1016 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1017 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1018 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1019 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1020 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1021 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1022 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1023 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1024 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1025 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1026 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1027 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1028 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1029 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1030 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1031 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1032 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1033 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1034 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1035 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1036 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1037 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1038 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1039 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1040 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1041 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1042 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1043 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1044 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1045 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1046 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1047 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1048 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1049 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1050 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1051 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1052 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1053 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1054 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1055 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1056 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1057 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1058 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1059 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1060 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1061 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1062 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1063 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1064 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1065 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1066 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1067 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1068 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1069 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1070 | lemma supp_subst2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1071 |   shows "supp (M{y:=<c>.P}) \<subseteq> supp (M) \<union> ((supp P) - {c})"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1072 | apply(nominal_induct M avoiding: y P c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1073 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1074 | apply(auto simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1075 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1076 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1077 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1078 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1079 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1080 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1081 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1082 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1083 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1084 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1085 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1086 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1087 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1088 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1089 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1090 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1091 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1092 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1093 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1094 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1095 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1096 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1097 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1098 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1099 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1100 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1101 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1102 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1103 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1104 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1105 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1106 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1107 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1108 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1109 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1110 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1111 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1112 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1113 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1114 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1115 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1116 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1117 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1118 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1119 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1120 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1121 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1122 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1123 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1124 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1125 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1126 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1127 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1128 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1129 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1130 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1131 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1132 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1133 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1134 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1135 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1136 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1137 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1138 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1139 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1140 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1141 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1142 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1143 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1144 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1145 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1146 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1147 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1148 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1149 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1150 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1151 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1152 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1153 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1154 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1155 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1156 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1157 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1158 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1159 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1160 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1161 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1162 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1163 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1164 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1165 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1166 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1167 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1168 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1169 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1170 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1171 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1172 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1173 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1174 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1175 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1176 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1177 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1178 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1179 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1180 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1181 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1182 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1183 | lemma supp_subst3: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1184 |   shows "supp (M{c:=(x).P}) \<subseteq> ((supp M) - {c}) \<union> (supp P)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1185 | apply(nominal_induct M avoiding: x P c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1186 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1187 | apply(auto simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1188 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1189 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1190 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1191 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1192 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1193 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1194 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1195 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1196 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1197 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1198 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1199 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1200 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1201 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1202 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1203 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1204 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1205 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1206 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1207 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1208 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1209 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1210 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1211 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1212 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1213 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1214 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1215 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1216 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1217 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1218 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1219 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1220 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1221 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1222 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1223 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1224 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1225 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1226 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1227 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1228 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1229 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1230 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1231 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1232 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1233 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1234 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1235 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1236 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1237 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1238 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1239 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1240 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1241 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1242 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1243 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1244 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1245 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1246 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1247 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1248 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1249 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1250 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1251 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1252 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1253 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1254 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1255 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1256 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1257 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1258 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1259 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1260 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1261 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1262 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1263 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1264 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1265 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1266 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1267 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1268 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1269 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1270 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1271 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1272 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1273 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1274 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1275 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1276 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1277 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1278 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1279 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1280 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1281 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1282 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1283 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1284 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1285 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1286 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1287 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1288 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1289 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1290 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1291 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1292 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1293 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1294 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1295 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1296 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1297 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1298 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1299 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1300 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1301 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1302 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1303 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1304 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1305 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1306 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1307 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1308 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1309 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1310 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1311 | lemma supp_subst4: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1312 |   shows "supp (M{c:=(x).P}) \<subseteq> (supp M) \<union> ((supp P) - {x})"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1313 | apply(nominal_induct M avoiding: x P c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1314 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1315 | apply(auto simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1316 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1317 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1318 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1319 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1320 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1321 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1322 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1323 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1324 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1325 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1326 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1327 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1328 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1329 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1330 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1331 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1332 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1333 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1334 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1335 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1336 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1337 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1338 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1339 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1340 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1341 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1342 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1343 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1344 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1345 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1346 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1347 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1348 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1349 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1350 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1351 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1352 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1353 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1354 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1355 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1356 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1357 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1358 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1359 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1360 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1361 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1362 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1363 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1364 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1365 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1366 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1367 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1368 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1369 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1370 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1371 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1372 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1373 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1374 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1375 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1376 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1377 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1378 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1379 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1380 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1381 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1382 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1383 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1384 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1385 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1386 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1387 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1388 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1389 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1390 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1391 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1392 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1393 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1394 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1395 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1396 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1397 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1398 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1399 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1400 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1401 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1402 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1403 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1404 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1405 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1406 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1407 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1408 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1409 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1410 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1411 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1412 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1413 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1414 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1415 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1416 | lemma supp_subst5: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1417 |   shows "(supp M - {y}) \<subseteq> supp (M{y:=<c>.P})"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1418 | apply(nominal_induct M avoiding: y P c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1419 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1420 | apply(auto simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1421 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1422 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1423 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1424 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1425 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1426 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1427 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1428 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1429 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1430 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1431 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1432 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1433 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1434 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1435 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1436 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1437 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1438 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1439 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1440 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1441 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1442 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1443 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1444 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1445 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1446 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1447 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1448 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1449 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1450 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1451 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1452 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1453 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1454 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1455 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1456 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1457 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1458 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1459 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1460 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1461 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1462 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1463 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1464 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1465 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1466 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1467 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1468 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1469 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1470 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1471 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1472 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1473 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1474 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1475 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1476 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1477 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1478 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1479 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1480 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1481 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1482 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1483 | lemma supp_subst6: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1484 |   shows "(supp M) \<subseteq> ((supp (M{y:=<c>.P}))::coname set)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1485 | apply(nominal_induct M avoiding: y P c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1486 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1487 | apply(auto simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1488 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1489 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1490 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1491 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1492 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1493 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1494 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1495 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1496 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1497 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1498 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1499 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1500 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1501 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1502 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1503 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1504 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1505 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1506 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1507 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1508 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1509 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1510 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1511 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1512 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1513 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1514 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1515 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1516 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1517 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1518 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1519 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1520 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1521 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1522 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},P,name1,trm2{y:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1523 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1524 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1525 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1526 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1527 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1528 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1529 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1530 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1531 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1532 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1533 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1534 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1535 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1536 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1537 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1538 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1539 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1540 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1541 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1542 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1543 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1544 | apply(simp add: fresh_def abs_supp trm.supp supp_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1545 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1546 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1547 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1548 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1549 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1550 | lemma supp_subst7: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1551 |   shows "(supp M - {c}) \<subseteq>  supp (M{c:=(x).P})"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1552 | apply(nominal_induct M avoiding: x P c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1553 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1554 | apply(auto simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1555 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1556 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1557 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1558 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1559 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1560 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1561 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1562 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1563 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1564 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1565 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1566 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1567 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1568 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1569 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1570 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1571 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1572 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1573 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1574 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1575 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1576 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1577 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1578 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1579 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1580 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1581 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1582 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1583 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1584 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1585 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1586 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1587 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1588 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1589 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1590 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1591 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1592 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1593 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1594 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1595 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1596 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1597 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1598 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1599 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1600 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1601 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1602 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1603 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1604 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1605 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1606 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1607 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1608 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1609 | lemma supp_subst8: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1610 |   shows "(supp M) \<subseteq> ((supp (M{c:=(x).P}))::name set)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1611 | apply(nominal_induct M avoiding: x P c rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1612 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1613 | apply(auto simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1614 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1615 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1616 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1617 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1618 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1619 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1620 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1621 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1622 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1623 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1624 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1625 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1626 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1627 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1628 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1629 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1630 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1631 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1632 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1633 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1634 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1635 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1636 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1637 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1638 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1639 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1640 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1641 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1642 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1643 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1644 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1645 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1646 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1647 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1648 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1649 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1650 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1651 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1652 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1653 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1654 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1655 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1656 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1657 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1658 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1659 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1660 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1661 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1662 | apply(simp add: fresh_def abs_supp trm.supp supp_atm fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1663 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1664 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1665 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1666 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1667 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1668 | lemmas subst_supp = supp_subst1 supp_subst2 supp_subst3 supp_subst4 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1669 | supp_subst5 supp_subst6 supp_subst7 supp_subst8 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1670 | lemma subst_fresh: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1671 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1672 | and c::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1673 |   shows "x\<sharp>P \<Longrightarrow> x\<sharp>M{x:=<c>.P}"   
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1674 |   and   "b\<sharp>P \<Longrightarrow> b\<sharp>M{b:=(y).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1675 |   and   "x\<sharp>(M,P) \<Longrightarrow> x\<sharp>M{y:=<c>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1676 |   and   "x\<sharp>M \<Longrightarrow> x\<sharp>M{c:=(x).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1677 |   and   "x\<sharp>(M,P) \<Longrightarrow> x\<sharp>M{c:=(y).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1678 |   and   "b\<sharp>(M,P) \<Longrightarrow> b\<sharp>M{c:=(y).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1679 |   and   "b\<sharp>M \<Longrightarrow> b\<sharp>M{y:=<b>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1680 |   and   "b\<sharp>(M,P) \<Longrightarrow> b\<sharp>M{y:=<c>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1681 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1682 | apply(insert subst_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1683 | apply(simp_all add: fresh_def supp_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1684 | apply(blast)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1685 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1686 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1687 | lemma forget: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1688 |   shows "x\<sharp>M \<Longrightarrow> M{x:=<c>.P} = M"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1689 |   and   "c\<sharp>M \<Longrightarrow> M{c:=(x).P} = M"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1690 | apply(nominal_induct M avoiding: x c P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1691 | apply(auto simp add: fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1692 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1693 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1694 | lemma substc_rename1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1695 | assumes a: "c\<sharp>(M,a)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1696 |   shows "M{a:=(x).N} = ([(c,a)]\<bullet>M){c:=(x).N}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1697 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1698 | proof(nominal_induct M avoiding: c a x N rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1699 | case (Ax z d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1700 | then show ?case by (auto simp add: fresh_prod fresh_atm calc_atm trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1701 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1702 | case NotL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1703 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1704 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1705 | case (NotR y M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1706 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1707 | by(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1708 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1709 | case (AndR c1 M c2 M' c3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1710 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1711 | apply(auto simp add: fresh_prod calc_atm fresh_atm abs_fresh fresh_left) | 
| 73932 
fd21b4a93043
added opaque_combs and renamed hide_lams to opaque_lifting
 desharna parents: 
71989diff
changeset | 1712 | apply (metis (erased, opaque_lifting)) | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1713 | by metis | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1714 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1715 | case AndL1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1716 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1717 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1718 | case AndL2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1719 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1720 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1721 | case (OrR1 d M e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1722 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1723 | by(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1724 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1725 | case (OrR2 d M e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1726 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1727 | by(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1728 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1729 | case (OrL x1 M x2 M' x3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1730 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1731 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1732 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1733 | case ImpL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1734 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1735 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1736 | metis | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1737 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1738 | case (ImpR y d M e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1739 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1740 | by(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1741 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1742 | case (Cut d M y M') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1743 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1744 | by(simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1745 | (metis crename.simps(1) crename_id crename_rename) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1746 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1747 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1748 | lemma substc_rename2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1749 | assumes a: "y\<sharp>(N,x)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1750 |   shows "M{a:=(x).N} = M{a:=(y).([(y,x)]\<bullet>N)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1751 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1752 | proof(nominal_induct M avoiding: a x y N rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1753 | case (Ax z d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1754 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1755 | by (auto simp add: fresh_prod fresh_atm calc_atm trm.inject alpha perm_swap fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1756 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1757 | case NotL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1758 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1759 | by (auto simp add: fresh_prod fresh_atm calc_atm trm.inject alpha perm_swap fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1760 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1761 | case (NotR y M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1762 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1763 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1764 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(N,M{d:=(y).([(y,x)]\<bullet>N)},[(y,x)]\<bullet>N)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1765 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1766 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1767 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1768 | apply(simp add: trm.inject alpha perm_swap fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1769 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1770 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1771 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1772 | case (AndR c1 M c2 M' c3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1773 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1774 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1775 | apply(subgoal_tac | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1776 |        "\<exists>a'::coname. a'\<sharp>(N,M{c3:=(y).([(y,x)]\<bullet>N)},M'{c3:=(y).([(y,x)]\<bullet>N)},[(y,x)]\<bullet>N,c1,c2,c3)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1777 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1778 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1779 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1780 | apply (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh subst_fresh perm_swap fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1781 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1782 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1783 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1784 | case AndL1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1785 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1786 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1787 | case AndL2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1788 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1789 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1790 | case (OrR1 d M e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1791 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1792 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1793 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(N,M{e:=(y).([(y,x)]\<bullet>N)},[(y,x)]\<bullet>N,d,e)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1794 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1795 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1796 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1797 | apply(simp add: trm.inject alpha perm_swap fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1798 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1799 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1800 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1801 | case (OrR2 d M e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1802 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1803 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1804 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(N,M{e:=(y).([(y,x)]\<bullet>N)},[(y,x)]\<bullet>N,d,e)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1805 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1806 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1807 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1808 | apply(simp add: trm.inject alpha perm_swap fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1809 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1810 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1811 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1812 | case (OrL x1 M x2 M' x3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1813 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1814 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1815 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1816 | case ImpL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1817 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1818 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1819 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1820 | case (ImpR y d M e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1821 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1822 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1823 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(N,M{e:=(y).([(y,x)]\<bullet>N)},[(y,x)]\<bullet>N,d,e)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1824 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1825 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1826 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1827 | apply(simp add: trm.inject alpha perm_swap fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1828 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1829 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1830 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1831 | case (Cut d M y M') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1832 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1833 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1834 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1835 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1836 | lemma substn_rename3: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1837 | assumes a: "y\<sharp>(M,x)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1838 |   shows "M{x:=<a>.N} = ([(y,x)]\<bullet>M){y:=<a>.N}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1839 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1840 | proof(nominal_induct M avoiding: a x y N rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1841 | case (Ax z d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1842 | then show ?case by (auto simp add: fresh_prod fresh_atm calc_atm trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1843 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1844 | case NotR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1845 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1846 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1847 | case (NotL d M z) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1848 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1849 | by(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1850 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1851 | case (AndR c1 M c2 M' c3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1852 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1853 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1854 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1855 | case OrR1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1856 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1857 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1858 | case OrR2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1859 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1860 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1861 | case (AndL1 u M v) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1862 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1863 | by(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1864 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1865 | case (AndL2 u M v) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1866 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1867 | by(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1868 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1869 | case (OrL x1 M x2 M' x3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1870 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1871 | by(simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1872 | (metis (poly_guards_query)) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1873 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1874 | case ImpR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1875 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1876 | by(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_left abs_supp fin_supp fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1877 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1878 | case (ImpL d M v M' u) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1879 | then show ?case | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1880 | by(simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1881 | (metis (poly_guards_query)) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1882 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1883 | case (Cut d M y M') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1884 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1885 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1886 | apply(drule pt_bij1[OF pt_name_inst, OF at_name_inst]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1887 | apply(simp add: calc_atm) | 
| 56073 
29e308b56d23
enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
 nipkow parents: 
53015diff
changeset | 1888 | apply metis | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1889 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1890 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1891 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1892 | lemma substn_rename4: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1893 | assumes a: "c\<sharp>(N,a)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1894 |   shows "M{x:=<a>.N} = M{x:=<c>.([(c,a)]\<bullet>N)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1895 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1896 | proof(nominal_induct M avoiding: x c a N rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1897 | case (Ax z d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1898 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1899 | by (auto simp add: fresh_prod fresh_atm calc_atm trm.inject alpha perm_swap fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1900 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1901 | case NotR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1902 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1903 | by (auto simp add: fresh_prod fresh_atm calc_atm trm.inject alpha perm_swap fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1904 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1905 | case (NotL d M y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1906 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1907 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1908 |     apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(N,M{x:=<c>.([(c,a)]\<bullet>N)},[(c,a)]\<bullet>N)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1909 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1910 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1911 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1912 | apply(simp add: trm.inject alpha perm_swap fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1913 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1914 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1915 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1916 | case (OrL x1 M x2 M' x3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1917 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1918 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1919 | apply(subgoal_tac | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1920 |        "\<exists>a'::name. a'\<sharp>(N,M{x:=<c>.([(c,a)]\<bullet>N)},M'{x:=<c>.([(c,a)]\<bullet>N)},[(c,a)]\<bullet>N,x1,x2,x3)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1921 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1922 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1923 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1924 | apply (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh subst_fresh perm_swap fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1925 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1926 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1927 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1928 | case OrR1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1929 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1930 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1931 | case OrR2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1932 | then show ?case by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1933 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1934 | case (AndL1 u M v) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1935 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1936 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1937 |     apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(N,M{x:=<c>.([(c,a)]\<bullet>N)},[(c,a)]\<bullet>N,u,v)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1938 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1939 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1940 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1941 | apply(simp add: trm.inject alpha perm_swap fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1942 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1943 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1944 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1945 | case (AndL2 u M v) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1946 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1947 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1948 |     apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(N,M{x:=<c>.([(c,a)]\<bullet>N)},[(c,a)]\<bullet>N,u,v)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1949 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1950 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1951 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1952 | apply(simp add: trm.inject alpha perm_swap fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1953 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1954 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1955 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1956 | case (AndR c1 M c2 M' c3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1957 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1958 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1959 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1960 | case ImpR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1961 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1962 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1963 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1964 | case (ImpL d M y M' u) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1965 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1966 | apply(auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1967 |     apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(N,M{u:=<c>.([(c,a)]\<bullet>N)},M'{u:=<c>.([(c,a)]\<bullet>N)},[(c,a)]\<bullet>N,y,u)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1968 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1969 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1970 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1971 | apply(simp add: trm.inject alpha perm_swap fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1972 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1973 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1974 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1975 | case (Cut d M y M') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1976 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1977 | by (auto simp add: calc_atm trm.inject alpha fresh_atm abs_fresh fresh_prod fresh_left perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1978 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1979 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1980 | lemma subst_rename5: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1981 | assumes a: "c'\<sharp>(c,N)" "x'\<sharp>(x,M)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1982 |   shows "M{x:=<c>.N} = ([(x',x)]\<bullet>M){x':=<c'>.([(c',c)]\<bullet>N)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1983 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1984 |   have "M{x:=<c>.N} = ([(x',x)]\<bullet>M){x':=<c>.N}" using a by (simp add: substn_rename3)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1985 |   also have "\<dots> = ([(x',x)]\<bullet>M){x':=<c'>.([(c',c)]\<bullet>N)}" using a by (simp add: substn_rename4)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1986 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1987 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1988 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1989 | lemma subst_rename6: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1990 | assumes a: "c'\<sharp>(c,M)" "x'\<sharp>(x,N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1991 |   shows "M{c:=(x).N} = ([(c',c)]\<bullet>M){c':=(x').([(x',x)]\<bullet>N)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1992 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1993 |   have "M{c:=(x).N} = ([(c',c)]\<bullet>M){c':=(x).N}" using a by (simp add: substc_rename1)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1994 |   also have "\<dots> = ([(c',c)]\<bullet>M){c':=(x').([(x',x)]\<bullet>N)}" using a by (simp add: substc_rename2)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1995 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1996 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1997 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1998 | lemmas subst_rename = substc_rename1 substc_rename2 substn_rename3 substn_rename4 subst_rename5 subst_rename6 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 1999 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2000 | lemma better_Cut_substn[simp]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2001 | assumes a: "a\<sharp>[c].P" "x\<sharp>(y,P)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2002 |   shows "(Cut <a>.M (x).N){y:=<c>.P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2003 |   (if M=Ax y a then Cut <c>.P (x).(N{y:=<c>.P}) else Cut <a>.(M{y:=<c>.P}) (x).(N{y:=<c>.P}))"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2004 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2005 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,c,P,x,y)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2006 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,c,P,a)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2007 | have eq1: "(Cut <a>.M (x).N) = (Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2008 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2009 | have eq2: "(M=Ax y a) = (([(a',a)]\<bullet>M)=Ax y a')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2010 | apply(auto simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2011 | apply(drule pt_bij1[OF pt_coname_inst, OF at_coname_inst]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2012 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2013 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2014 |   have "(Cut <a>.M (x).N){y:=<c>.P} = (Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N)){y:=<c>.P}" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2015 | using eq1 by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2016 |   also have "\<dots> = (if ([(a',a)]\<bullet>M)=Ax y a' then Cut <c>.P (x').(([(x',x)]\<bullet>N){y:=<c>.P}) 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2017 |                               else Cut <a'>.(([(a',a)]\<bullet>M){y:=<c>.P}) (x').(([(x',x)]\<bullet>N){y:=<c>.P}))" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2018 | using fs1 fs2 by (auto simp add: fresh_prod fresh_left calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2019 |   also have "\<dots> =(if M=Ax y a then Cut <c>.P (x).(N{y:=<c>.P}) else Cut <a>.(M{y:=<c>.P}) (x).(N{y:=<c>.P}))"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2020 | using fs1 fs2 a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2021 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2022 | apply(simp only: eq2[symmetric]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2023 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2024 | apply(simp_all add: alpha fresh_atm fresh_prod subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2025 | apply(simp_all add: eqvts perm_fresh_fresh calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2026 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2027 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2028 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2029 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2030 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2031 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2032 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2033 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2034 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2035 | lemma better_Cut_substc[simp]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2036 | assumes a: "a\<sharp>(c,P)" "x\<sharp>[y].P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2037 |   shows "(Cut <a>.M (x).N){c:=(y).P} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2038 |   (if N=Ax x c then Cut <a>.(M{c:=(y).P}) (y).P else Cut <a>.(M{c:=(y).P}) (x).(N{c:=(y).P}))" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2039 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2040 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,c,P,x,y)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2041 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,c,P,a)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2042 | have eq1: "(Cut <a>.M (x).N) = (Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N))" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2043 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2044 | have eq2: "(N=Ax x c) = (([(x',x)]\<bullet>N)=Ax x' c)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2045 | apply(auto simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2046 | apply(drule pt_bij1[OF pt_name_inst, OF at_name_inst]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2047 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2048 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2049 |   have "(Cut <a>.M (x).N){c:=(y).P} = (Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N)){c:=(y).P}" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2050 | using eq1 by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2051 |   also have "\<dots> = (if ([(x',x)]\<bullet>N)=Ax x' c then  Cut <a'>.(([(a',a)]\<bullet>M){c:=(y).P}) (y).P
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2052 |                               else Cut <a'>.(([(a',a)]\<bullet>M){c:=(y).P}) (x').(([(x',x)]\<bullet>N){c:=(y).P}))" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2053 | using fs1 fs2 by (simp add: fresh_prod fresh_left calc_atm fresh_atm trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2054 |   also have "\<dots> =(if N=Ax x c then Cut <a>.(M{c:=(y).P}) (y).P else Cut <a>.(M{c:=(y).P}) (x).(N{c:=(y).P}))"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2055 | using fs1 fs2 a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2056 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2057 | apply(simp only: eq2[symmetric]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2058 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2059 | apply(simp_all add: alpha fresh_atm fresh_prod subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2060 | apply(simp_all add: eqvts perm_fresh_fresh calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2061 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2062 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2063 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2064 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2065 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2066 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2067 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2068 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2069 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2070 | lemma better_Cut_substn': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2071 | assumes a: "a\<sharp>[c].P" "y\<sharp>(N,x)" "M\<noteq>Ax y a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2072 |   shows "(Cut <a>.M (x).N){y:=<c>.P} = Cut <a>.(M{y:=<c>.P}) (x).N"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2073 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2074 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2075 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2076 | apply(subgoal_tac "Cut <a>.M (x).N = Cut <a>.M (ca).([(ca,x)]\<bullet>N)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2077 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2078 | apply(subgoal_tac"y\<sharp>([(ca,x)]\<bullet>N)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2079 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2080 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2081 | apply(auto simp add: fresh_left calc_atm fresh_prod fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2082 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2083 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2084 | apply(simp add: alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2085 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2086 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2087 | lemma better_NotR_substc: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2088 | assumes a: "d\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2089 |   shows "(NotR (x).M d){d:=(z).P} = fresh_fun (\<lambda>a'. Cut <a'>.NotR (x).M a' (z).P)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2090 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2091 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2092 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2093 | apply(subgoal_tac "NotR (x).M d = NotR (c).([(c,x)]\<bullet>M) d") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2094 | apply(auto simp add: fresh_left calc_atm forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2095 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2096 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2097 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2098 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2099 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2100 | apply(perm_simp add: trm.inject alpha fresh_prod fresh_atm fresh_left, auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2101 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2102 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2103 | lemma better_NotL_substn: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2104 | assumes a: "y\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2105 |   shows "(NotL <a>.M y){y:=<c>.P} = fresh_fun (\<lambda>x'. Cut <c>.P (x').NotL <a>.M x')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2106 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2107 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2108 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2109 | apply(subgoal_tac "NotL <a>.M y = NotL <ca>.([(ca,a)]\<bullet>M) y") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2110 | apply(auto simp add: fresh_left calc_atm forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2111 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2112 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2113 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2114 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2115 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2116 | apply(perm_simp add: trm.inject alpha fresh_prod fresh_atm fresh_left, auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2117 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2118 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2119 | lemma better_AndL1_substn: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2120 | assumes a: "y\<sharp>[x].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2121 |   shows "(AndL1 (x).M y){y:=<c>.P} = fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL1 (x).M z')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2122 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2123 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2124 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2125 | apply(subgoal_tac "AndL1 (x).M y = AndL1 (ca).([(ca,x)]\<bullet>M) y") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2126 | apply(auto simp add: fresh_left calc_atm forget abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2127 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2128 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2129 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2130 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2131 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2132 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2133 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2134 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2135 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2136 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2137 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2138 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2139 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2140 | apply(perm_simp add: trm.inject alpha fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2141 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2142 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2143 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2144 | lemma better_AndL2_substn: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2145 | assumes a: "y\<sharp>[x].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2146 |   shows "(AndL2 (x).M y){y:=<c>.P} = fresh_fun (\<lambda>z'. Cut <c>.P (z').AndL2 (x).M z')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2147 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2148 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2149 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2150 | apply(subgoal_tac "AndL2 (x).M y = AndL2 (ca).([(ca,x)]\<bullet>M) y") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2151 | apply(auto simp add: fresh_left calc_atm forget abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2152 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2153 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2154 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2155 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2156 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2157 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2158 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2159 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2160 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2161 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2162 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2163 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2164 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2165 | apply(perm_simp add: trm.inject alpha fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2166 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2167 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2168 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2169 | lemma better_AndR_substc: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2170 | assumes a: "c\<sharp>([a].M,[b].N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2171 |   shows "(AndR <a>.M <b>.N c){c:=(z).P} = fresh_fun (\<lambda>a'. Cut <a'>.(AndR <a>.M <b>.N a') (z).P)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2172 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2173 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2174 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2175 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2176 | apply(subgoal_tac "AndR <a>.M <b>.N c = AndR <ca>.([(ca,a)]\<bullet>M) <caa>.([(caa,b)]\<bullet>N) c") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2177 | apply(auto simp add: fresh_left calc_atm forget abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2178 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2179 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2180 | apply(auto simp add: fresh_left calc_atm fresh_prod fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2181 | apply(auto simp add: fresh_left calc_atm fresh_prod fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2182 | apply(auto simp add: fresh_prod fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2183 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2184 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2185 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2186 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2187 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2188 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2189 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2190 | apply(auto simp add: fresh_left calc_atm abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2191 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2192 | apply(auto simp add: fresh_left calc_atm abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2193 | apply(perm_simp add: trm.inject alpha fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2194 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2195 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2196 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2197 | lemma better_OrL_substn: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2198 | assumes a: "x\<sharp>([y].M,[z].N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2199 |   shows "(OrL (y).M (z).N x){x:=<c>.P} = fresh_fun (\<lambda>z'. Cut <c>.P (z').OrL (y).M (z).N z')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2200 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2201 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2202 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2203 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2204 | apply(subgoal_tac "OrL (y).M (z).N x = OrL (ca).([(ca,y)]\<bullet>M) (caa).([(caa,z)]\<bullet>N) x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2205 | apply(auto simp add: fresh_left calc_atm forget abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2206 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2207 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2208 | apply(auto simp add: fresh_left calc_atm fresh_prod fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2209 | apply(auto simp add: fresh_left calc_atm fresh_prod fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2210 | apply(auto simp add: fresh_prod fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2211 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2212 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2213 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2214 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2215 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2216 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2217 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2218 | apply(auto simp add: fresh_left calc_atm abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2219 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2220 | apply(auto simp add: fresh_left calc_atm abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2221 | apply(perm_simp add: trm.inject alpha fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2222 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2223 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2224 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2225 | lemma better_OrR1_substc: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2226 | assumes a: "d\<sharp>[a].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2227 |   shows "(OrR1 <a>.M d){d:=(z).P} = fresh_fun (\<lambda>a'. Cut <a'>.OrR1 <a>.M a' (z).P)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2228 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2229 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2230 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2231 | apply(subgoal_tac "OrR1 <a>.M d = OrR1 <c>.([(c,a)]\<bullet>M) d") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2232 | apply(auto simp add: fresh_left calc_atm forget abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2233 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2234 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2235 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2236 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2237 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2238 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2239 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2240 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2241 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2242 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2243 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2244 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2245 | apply(perm_simp add: trm.inject alpha fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2246 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2247 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2248 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2249 | lemma better_OrR2_substc: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2250 | assumes a: "d\<sharp>[a].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2251 |   shows "(OrR2 <a>.M d){d:=(z).P} = fresh_fun (\<lambda>a'. Cut <a'>.OrR2 <a>.M a' (z).P)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2252 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2253 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2254 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2255 | apply(subgoal_tac "OrR2 <a>.M d = OrR2 <c>.([(c,a)]\<bullet>M) d") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2256 | apply(auto simp add: fresh_left calc_atm forget abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2257 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2258 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2259 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2260 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2261 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2262 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2263 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2264 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2265 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2266 | apply(simp add: trm.inject alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2267 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2268 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2269 | apply(perm_simp add: trm.inject alpha fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2270 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2271 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2272 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2273 | lemma better_ImpR_substc: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2274 | assumes a: "d\<sharp>[a].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2275 |   shows "(ImpR (x).<a>.M d){d:=(z).P} = fresh_fun (\<lambda>a'. Cut <a'>.ImpR (x).<a>.M a' (z).P)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2276 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2277 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2278 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2279 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2280 | apply(subgoal_tac "ImpR (x).<a>.M d = ImpR (ca).<c>.([(c,a)]\<bullet>[(ca,x)]\<bullet>M) d") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2281 | apply(auto simp add: fresh_left calc_atm forget abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2282 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2283 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2284 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2285 | apply(simp add: trm.inject alpha fresh_prod fresh_atm abs_perm abs_fresh fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2286 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2287 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2288 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2289 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2290 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2291 | apply(simp add: trm.inject alpha fresh_prod fresh_atm abs_perm fresh_left calc_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2292 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2293 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2294 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2295 | apply(perm_simp add: trm.inject alpha fresh_left calc_atm fresh_prod fresh_atm abs_fresh abs_perm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2296 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2297 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2298 | lemma better_ImpL_substn: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2299 | assumes a: "y\<sharp>(M,[x].N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2300 |   shows "(ImpL <a>.M (x).N y){y:=<c>.P} = fresh_fun (\<lambda>z'. Cut <c>.P (z').ImpL <a>.M (x).N z')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2301 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2302 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2303 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2304 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2305 | apply(subgoal_tac "ImpL <a>.M (x).N y = ImpL <ca>.([(ca,a)]\<bullet>M) (caa).([(caa,x)]\<bullet>N) y") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2306 | apply(auto simp add: fresh_left calc_atm forget abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2307 | apply(rule_tac f="fresh_fun" in arg_cong) | 
| 39302 
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
 nipkow parents: 
39198diff
changeset | 2308 | apply(simp add: fun_eq_iff) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2309 | apply(rule allI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2310 | apply(simp add: trm.inject alpha fresh_prod fresh_atm abs_perm abs_fresh fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2311 | apply(rule forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2312 | apply(simp add: fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2313 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2314 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2315 | apply(perm_simp add: trm.inject alpha fresh_left calc_atm fresh_prod fresh_atm abs_fresh abs_perm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2316 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2317 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2318 | lemma freshn_after_substc: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2319 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2320 |   assumes a: "x\<sharp>M{c:=(y).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2321 | shows "x\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2322 | using a supp_subst8 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2323 | apply(simp add: fresh_def) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2324 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2325 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2326 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2327 | lemma freshn_after_substn: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2328 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2329 |   assumes a: "x\<sharp>M{y:=<c>.P}" "x\<noteq>y"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2330 | shows "x\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2331 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2332 | using a supp_subst5 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2333 | apply(simp add: fresh_def) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2334 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2335 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2336 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2337 | lemma freshc_after_substc: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2338 | fixes a::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2339 |   assumes a: "a\<sharp>M{c:=(y).P}" "a\<noteq>c"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2340 | shows "a\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2341 | using a supp_subst7 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2342 | apply(simp add: fresh_def) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2343 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2344 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2345 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2346 | lemma freshc_after_substn: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2347 | fixes a::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2348 |   assumes a: "a\<sharp>M{y:=<c>.P}" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2349 | shows "a\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2350 | using a supp_subst6 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2351 | apply(simp add: fresh_def) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2352 | apply(blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2353 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2354 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2355 | lemma substn_crename_comm: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2356 | assumes a: "c\<noteq>a" "c\<noteq>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2357 |   shows "M{x:=<c>.P}[a\<turnstile>c>b] = M[a\<turnstile>c>b]{x:=<c>.(P[a\<turnstile>c>b])}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2358 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2359 | apply(nominal_induct M avoiding: x c P a b rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2360 | apply(auto simp add: subst_fresh rename_fresh trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2361 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,x,c)") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2362 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2363 | apply(subgoal_tac "Cut <c>.P (x).Ax x a = Cut <c>.P (x').Ax x' a") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2364 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2365 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2366 | apply(rule crename.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2367 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2368 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2369 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2370 | apply(simp add: alpha trm.inject calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2371 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2372 | apply(simp add: alpha trm.inject calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2373 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2374 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2375 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2376 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2377 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2378 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2379 | apply(simp add: crename_id) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2380 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2381 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2382 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2383 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2384 | apply(auto simp add: fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2385 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2386 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2387 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2388 | apply(auto simp add: fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2389 | apply(drule crename_ax) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2390 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2391 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2392 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2393 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<c>.P},P,P[a\<turnstile>c>b],x,trm[a\<turnstile>c>b]{x:=<c>.P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2394 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2395 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2396 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2397 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2398 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2399 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2400 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2401 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2402 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2403 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<c>.P},P,P[a\<turnstile>c>b],name1,trm[a\<turnstile>c>b]{x:=<c>.P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2404 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2405 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2406 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2407 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2408 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2409 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2410 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2411 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2412 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2413 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<c>.P},P,P[a\<turnstile>c>b],name1,trm[a\<turnstile>c>b]{x:=<c>.P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2414 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2415 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2416 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2417 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2418 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2419 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2420 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2421 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2422 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2423 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{x:=<c>.P},trm2{x:=<c>.P},P,P[a\<turnstile>c>b],name1,name2,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2424 |                                   trm1[a\<turnstile>c>b]{x:=<c>.P[a\<turnstile>c>b]},trm2[a\<turnstile>c>b]{x:=<c>.P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2425 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2426 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2427 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2428 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2429 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2430 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2431 | apply(simp add: rename_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2432 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2433 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2434 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},trm2{name2:=<c>.P},P,P[a\<turnstile>c>b],name1,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2435 |                                   trm1[a\<turnstile>c>b]{name2:=<c>.P[a\<turnstile>c>b]},trm2[a\<turnstile>c>b]{name2:=<c>.P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2436 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2437 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2438 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2439 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2440 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2441 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2442 | apply(simp add: rename_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2443 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2444 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2445 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2446 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2447 | lemma substc_crename_comm: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2448 | assumes a: "c\<noteq>a" "c\<noteq>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2449 |   shows "M{c:=(x).P}[a\<turnstile>c>b] = M[a\<turnstile>c>b]{c:=(x).(P[a\<turnstile>c>b])}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2450 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2451 | apply(nominal_induct M avoiding: x c P a b rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2452 | apply(auto simp add: subst_fresh rename_fresh trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2453 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2454 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2455 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2456 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2457 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2458 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2459 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2460 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2461 | apply(drule crename_ax) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2462 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2463 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2464 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2465 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(a,b,trm{coname:=(x).P},P,P[a\<turnstile>c>b],x,trm[a\<turnstile>c>b]{coname:=(x).P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2466 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2467 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2468 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2469 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2470 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2471 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2472 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2473 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2474 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2475 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(coname1,coname2,a,b,trm1{coname3:=(x).P},trm2{coname3:=(x).P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2476 |                    P,P[a\<turnstile>c>b],x,trm1[a\<turnstile>c>b]{coname3:=(x).P[a\<turnstile>c>b]},trm2[a\<turnstile>c>b]{coname3:=(x).P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2477 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2478 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2479 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2480 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2481 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2482 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2483 | apply(simp add: rename_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2484 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2485 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2486 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(coname1,trm{coname2:=(x).P},P,P[a\<turnstile>c>b],a,b,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2487 |                          trm[a\<turnstile>c>b]{coname2:=(x).P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2488 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2489 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2490 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2491 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2492 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2493 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2494 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2495 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2496 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2497 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(coname1,trm{coname2:=(x).P},P,P[a\<turnstile>c>b],a,b,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2498 |                          trm[a\<turnstile>c>b]{coname2:=(x).P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2499 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2500 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2501 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2502 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2503 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2504 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2505 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2506 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2507 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2508 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(coname1,trm{coname2:=(x).P},P,P[a\<turnstile>c>b],a,b,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2509 |                          trm[a\<turnstile>c>b]{coname2:=(x).P[a\<turnstile>c>b]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2510 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2511 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2512 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2513 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2514 | apply(rule better_crename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2515 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2516 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2517 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2518 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2519 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2520 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2521 | lemma substn_nrename_comm: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2522 | assumes a: "x\<noteq>y" "x\<noteq>z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2523 |   shows "M{x:=<c>.P}[y\<turnstile>n>z] = M[y\<turnstile>n>z]{x:=<c>.(P[y\<turnstile>n>z])}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2524 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2525 | apply(nominal_induct M avoiding: x c P y z rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2526 | apply(auto simp add: subst_fresh rename_fresh trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2527 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2528 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2529 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2530 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2531 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2532 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2533 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2534 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2535 | apply(drule nrename_ax) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2536 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2537 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2538 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2539 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(y,z,trm{x:=<c>.P},P,P[y\<turnstile>n>z],x,trm[y\<turnstile>n>z]{x:=<c>.P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2540 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2541 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2542 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2543 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2544 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2545 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2546 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2547 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2548 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2549 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<c>.P},P,P[y\<turnstile>n>z],name1,trm[y\<turnstile>n>z]{x:=<c>.P[y\<turnstile>n>z]},y,z)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2550 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2551 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2552 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2553 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2554 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2555 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2556 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2557 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2558 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2559 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(y,z,trm{x:=<c>.P},P,P[y\<turnstile>n>z],name1,trm[y\<turnstile>n>z]{x:=<c>.P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2560 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2561 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2562 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2563 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2564 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2565 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2566 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2567 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2568 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2569 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{x:=<c>.P},trm2{x:=<c>.P},P,P[y\<turnstile>n>z],name1,name2,y,z,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2570 |                                   trm1[y\<turnstile>n>z]{x:=<c>.P[y\<turnstile>n>z]},trm2[y\<turnstile>n>z]{x:=<c>.P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2571 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2572 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2573 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2574 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2575 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2576 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2577 | apply(simp add: rename_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2578 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2579 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2580 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},trm2{name2:=<c>.P},P,P[y\<turnstile>n>z],y,z,name1,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2581 |                                   trm1[y\<turnstile>n>z]{name2:=<c>.P[y\<turnstile>n>z]},trm2[y\<turnstile>n>z]{name2:=<c>.P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2582 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2583 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2584 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2585 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2586 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2587 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2588 | apply(simp add: rename_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2589 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2590 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2591 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2592 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2593 | lemma substc_nrename_comm: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2594 | assumes a: "x\<noteq>y" "x\<noteq>z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2595 |   shows "M{c:=(x).P}[y\<turnstile>n>z] = M[y\<turnstile>n>z]{c:=(x).(P[y\<turnstile>n>z])}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2596 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2597 | apply(nominal_induct M avoiding: x c P y z rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2598 | apply(auto simp add: subst_fresh rename_fresh trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2599 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2600 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2601 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2602 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2603 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2604 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2605 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2606 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2607 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2608 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2609 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2610 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2611 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2612 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2613 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2614 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2615 | apply(drule nrename_ax) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2616 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2617 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2618 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2619 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2620 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2621 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2622 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2623 | apply(drule nrename_ax) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2624 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2625 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2626 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2627 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(y,z,trm{coname:=(x).P},P,P[y\<turnstile>n>z],x,trm[y\<turnstile>n>z]{coname:=(x).P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2628 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2629 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2630 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2631 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2632 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2633 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2634 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2635 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2636 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2637 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(coname1,coname2,y,z,trm1{coname3:=(x).P},trm2{coname3:=(x).P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2638 |                    P,P[y\<turnstile>n>z],x,trm1[y\<turnstile>n>z]{coname3:=(x).P[y\<turnstile>n>z]},trm2[y\<turnstile>n>z]{coname3:=(x).P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2639 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2640 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2641 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2642 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2643 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2644 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2645 | apply(simp add: rename_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2646 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2647 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2648 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(coname1,trm{coname2:=(x).P},P,P[y\<turnstile>n>z],y,z,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2649 |                          trm[y\<turnstile>n>z]{coname2:=(x).P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2650 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2651 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2652 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2653 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2654 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2655 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2656 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2657 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2658 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2659 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(coname1,trm{coname2:=(x).P},P,P[y\<turnstile>n>z],y,z,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2660 |                          trm[y\<turnstile>n>z]{coname2:=(x).P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2661 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2662 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2663 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2664 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2665 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2666 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2667 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2668 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2669 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2670 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(coname1,trm{coname2:=(x).P},P,P[y\<turnstile>n>z],y,z,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2671 |                          trm[y\<turnstile>n>z]{coname2:=(x).P[y\<turnstile>n>z]})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2672 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2673 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2674 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2675 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2676 | apply(rule better_nrename_Cut) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2677 | apply(simp add: fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2678 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2679 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2680 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2681 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2682 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2683 | lemma substn_crename_comm': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2684 | assumes a: "a\<noteq>c" "a\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2685 |   shows "M{x:=<c>.P}[a\<turnstile>c>b] = M[a\<turnstile>c>b]{x:=<c>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2686 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2687 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2688 | assume a1: "a\<noteq>c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2689 | assume a2: "a\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2690 | obtain c'::"coname" where fs2: "c'\<sharp>(c,P,a,b)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2691 |   have eq: "M{x:=<c>.P} = M{x:=<c'>.([(c',c)]\<bullet>P)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2692 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2693 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2694 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2695 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2696 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2697 |    have eq': "M[a\<turnstile>c>b]{x:=<c>.P} = M[a\<turnstile>c>b]{x:=<c'>.([(c',c)]\<bullet>P)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2698 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2699 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2700 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2701 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2702 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2703 | have eq2: "([(c',c)]\<bullet>P)[a\<turnstile>c>b] = ([(c',c)]\<bullet>P)" using fs2 a2 a1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2704 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2705 | apply(rule rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2706 | apply(simp add: fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2707 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2708 |   have "M{x:=<c>.P}[a\<turnstile>c>b] = M{x:=<c'>.([(c',c)]\<bullet>P)}[a\<turnstile>c>b]" using eq by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2709 |   also have "\<dots> = M[a\<turnstile>c>b]{x:=<c'>.(([(c',c)]\<bullet>P)[a\<turnstile>c>b])}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2710 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2711 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2712 | apply(rule substn_crename_comm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2713 | apply(simp_all add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2714 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2715 |   also have "\<dots> = M[a\<turnstile>c>b]{x:=<c'>.(([(c',c)]\<bullet>P))}" using eq2 by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2716 |   also have "\<dots> = M[a\<turnstile>c>b]{x:=<c>.P}" using eq' by simp 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2717 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2718 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2719 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2720 | lemma substc_crename_comm': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2721 | assumes a: "c\<noteq>a" "c\<noteq>b" "a\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2722 |   shows "M{c:=(x).P}[a\<turnstile>c>b] = M[a\<turnstile>c>b]{c:=(x).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2723 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2724 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2725 | assume a1: "c\<noteq>a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2726 | assume a1': "c\<noteq>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2727 | assume a2: "a\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2728 | obtain c'::"coname" where fs2: "c'\<sharp>(c,M,a,b)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2729 |   have eq: "M{c:=(x).P} = ([(c',c)]\<bullet>M){c':=(x).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2730 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2731 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2732 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2733 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2734 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2735 |    have eq': "([(c',c)]\<bullet>(M[a\<turnstile>c>b])){c':=(x).P} = M[a\<turnstile>c>b]{c:=(x).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2736 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2737 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2738 | apply(rule subst_rename[symmetric]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2739 | apply(simp add: rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2740 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2741 | have eq2: "([(c',c)]\<bullet>M)[a\<turnstile>c>b] = ([(c',c)]\<bullet>(M[a\<turnstile>c>b]))" using fs2 a2 a1 a1' | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2742 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2743 | apply(simp add: rename_eqvts) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2744 | apply(simp add: fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2745 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2746 |   have "M{c:=(x).P}[a\<turnstile>c>b] = ([(c',c)]\<bullet>M){c':=(x).P}[a\<turnstile>c>b]" using eq by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2747 |   also have "\<dots> = ([(c',c)]\<bullet>M)[a\<turnstile>c>b]{c':=(x).P[a\<turnstile>c>b]}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2748 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2749 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2750 | apply(rule substc_crename_comm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2751 | apply(simp_all add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2752 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2753 |   also have "\<dots> = ([(c',c)]\<bullet>(M[a\<turnstile>c>b])){c':=(x).P[a\<turnstile>c>b]}" using eq2 by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2754 |   also have "\<dots> = ([(c',c)]\<bullet>(M[a\<turnstile>c>b])){c':=(x).P}" using a2 by (simp add: rename_fresh)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2755 |   also have "\<dots> = M[a\<turnstile>c>b]{c:=(x).P}" using eq' by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2756 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2757 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2758 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2759 | lemma substn_nrename_comm': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2760 | assumes a: "x\<noteq>y" "x\<noteq>z" "y\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2761 |   shows "M{x:=<c>.P}[y\<turnstile>n>z] = M[y\<turnstile>n>z]{x:=<c>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2762 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2763 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2764 | assume a1: "x\<noteq>y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2765 | assume a1': "x\<noteq>z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2766 | assume a2: "y\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2767 | obtain x'::"name" where fs2: "x'\<sharp>(x,M,y,z)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2768 |   have eq: "M{x:=<c>.P} = ([(x',x)]\<bullet>M){x':=<c>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2769 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2770 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2771 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2772 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2773 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2774 |    have eq': "([(x',x)]\<bullet>(M[y\<turnstile>n>z])){x':=<c>.P} = M[y\<turnstile>n>z]{x:=<c>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2775 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2776 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2777 | apply(rule subst_rename[symmetric]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2778 | apply(simp add: rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2779 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2780 | have eq2: "([(x',x)]\<bullet>M)[y\<turnstile>n>z] = ([(x',x)]\<bullet>(M[y\<turnstile>n>z]))" using fs2 a2 a1 a1' | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2781 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2782 | apply(simp add: rename_eqvts) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2783 | apply(simp add: fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2784 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2785 |   have "M{x:=<c>.P}[y\<turnstile>n>z] = ([(x',x)]\<bullet>M){x':=<c>.P}[y\<turnstile>n>z]" using eq by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2786 |   also have "\<dots> = ([(x',x)]\<bullet>M)[y\<turnstile>n>z]{x':=<c>.P[y\<turnstile>n>z]}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2787 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2788 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2789 | apply(rule substn_nrename_comm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2790 | apply(simp_all add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2791 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2792 |   also have "\<dots> = ([(x',x)]\<bullet>(M[y\<turnstile>n>z])){x':=<c>.P[y\<turnstile>n>z]}" using eq2 by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2793 |   also have "\<dots> = ([(x',x)]\<bullet>(M[y\<turnstile>n>z])){x':=<c>.P}" using a2 by (simp add: rename_fresh)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2794 |   also have "\<dots> = M[y\<turnstile>n>z]{x:=<c>.P}" using eq' by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2795 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2796 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2797 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2798 | lemma substc_nrename_comm': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2799 | assumes a: "x\<noteq>y" "y\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2800 |   shows "M{c:=(x).P}[y\<turnstile>n>z] = M[y\<turnstile>n>z]{c:=(x).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2801 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2802 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2803 | assume a1: "x\<noteq>y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2804 | assume a2: "y\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2805 | obtain x'::"name" where fs2: "x'\<sharp>(x,P,y,z)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2806 |   have eq: "M{c:=(x).P} = M{c:=(x').([(x',x)]\<bullet>P)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2807 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2808 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2809 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2810 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2811 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2812 |    have eq': "M[y\<turnstile>n>z]{c:=(x).P} = M[y\<turnstile>n>z]{c:=(x').([(x',x)]\<bullet>P)}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2813 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2814 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2815 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2816 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2817 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2818 | have eq2: "([(x',x)]\<bullet>P)[y\<turnstile>n>z] = ([(x',x)]\<bullet>P)" using fs2 a2 a1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2819 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2820 | apply(rule rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2821 | apply(simp add: fresh_left calc_atm fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2822 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2823 |   have "M{c:=(x).P}[y\<turnstile>n>z] = M{c:=(x').([(x',x)]\<bullet>P)}[y\<turnstile>n>z]" using eq by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2824 |   also have "\<dots> = M[y\<turnstile>n>z]{c:=(x').(([(x',x)]\<bullet>P)[y\<turnstile>n>z])}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2825 | using fs2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2826 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2827 | apply(rule substc_nrename_comm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2828 | apply(simp_all add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2829 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2830 |   also have "\<dots> = M[y\<turnstile>n>z]{c:=(x').(([(x',x)]\<bullet>P))}" using eq2 by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2831 |   also have "\<dots> = M[y\<turnstile>n>z]{c:=(x).P}" using eq' by simp 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2832 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2833 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2834 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2835 | lemmas subst_comm = substn_crename_comm substc_crename_comm | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2836 | substn_nrename_comm substc_nrename_comm | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2837 | lemmas subst_comm' = substn_crename_comm' substc_crename_comm' | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2838 | substn_nrename_comm' substc_nrename_comm' | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2839 | |
| 63167 | 2840 | text \<open>typing contexts\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2841 | |
| 41798 | 2842 | type_synonym ctxtn = "(name\<times>ty) list" | 
| 2843 | type_synonym ctxtc = "(coname\<times>ty) list" | |
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2844 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2845 | inductive | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2846 | validc :: "ctxtc \<Rightarrow> bool" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2847 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2848 | vc1[intro]: "validc []" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2849 | | vc2[intro]: "\<lbrakk>a\<sharp>\<Delta>; validc \<Delta>\<rbrakk> \<Longrightarrow> validc ((a,T)#\<Delta>)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2850 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2851 | equivariance validc | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2852 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2853 | inductive | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2854 | validn :: "ctxtn \<Rightarrow> bool" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2855 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2856 | vn1[intro]: "validn []" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2857 | | vn2[intro]: "\<lbrakk>x\<sharp>\<Gamma>; validn \<Gamma>\<rbrakk> \<Longrightarrow> validn ((x,T)#\<Gamma>)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2858 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2859 | equivariance validn | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2860 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2861 | lemma fresh_ctxt: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2862 | fixes a::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2863 | and x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2864 | and \<Gamma>::"ctxtn" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2865 | and \<Delta>::"ctxtc" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2866 | shows "a\<sharp>\<Gamma>" and "x\<sharp>\<Delta>" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2867 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2868 | show "a\<sharp>\<Gamma>" by (induct \<Gamma>) (auto simp add: fresh_list_nil fresh_list_cons fresh_prod fresh_atm fresh_ty) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2869 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2870 | show "x\<sharp>\<Delta>" by (induct \<Delta>) (auto simp add: fresh_list_nil fresh_list_cons fresh_prod fresh_atm fresh_ty) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2871 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2872 | |
| 63167 | 2873 | text \<open>cut-reductions\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2874 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2875 | declare abs_perm[eqvt] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2876 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2877 | inductive | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2878 | fin :: "trm \<Rightarrow> name \<Rightarrow> bool" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2879 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2880 | [intro]: "fin (Ax x a) x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2881 | | [intro]: "x\<sharp>M \<Longrightarrow> fin (NotL <a>.M x) x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2882 | | [intro]: "y\<sharp>[x].M \<Longrightarrow> fin (AndL1 (x).M y) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2883 | | [intro]: "y\<sharp>[x].M \<Longrightarrow> fin (AndL2 (x).M y) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2884 | | [intro]: "\<lbrakk>z\<sharp>[x].M;z\<sharp>[y].N\<rbrakk> \<Longrightarrow> fin (OrL (x).M (y).N z) z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2885 | | [intro]: "\<lbrakk>y\<sharp>M;y\<sharp>[x].N\<rbrakk> \<Longrightarrow> fin (ImpL <a>.M (x).N y) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2886 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2887 | equivariance fin | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2888 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2889 | lemma fin_Ax_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2890 | assumes a: "fin (Ax x a) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2891 | shows "x=y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2892 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2893 | apply(erule_tac fin.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2894 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2895 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2896 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2897 | lemma fin_NotL_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2898 | assumes a: "fin (NotL <a>.M x) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2899 | shows "x=y \<and> x\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2900 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2901 | apply(erule_tac fin.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2902 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2903 | apply(subgoal_tac "y\<sharp>[aa].Ma") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2904 | apply(drule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2905 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2906 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2907 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2908 | lemma fin_AndL1_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2909 | assumes a: "fin (AndL1 (x).M y) z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2910 | shows "z=y \<and> z\<sharp>[x].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2911 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2912 | apply(erule_tac fin.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2913 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2914 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2915 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2916 | lemma fin_AndL2_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2917 | assumes a: "fin (AndL2 (x).M y) z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2918 | shows "z=y \<and> z\<sharp>[x].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2919 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2920 | apply(erule_tac fin.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2921 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2922 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2923 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2924 | lemma fin_OrL_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2925 | assumes a: "fin (OrL (x).M (y).N u) z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2926 | shows "z=u \<and> z\<sharp>[x].M \<and> z\<sharp>[y].N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2927 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2928 | apply(erule_tac fin.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2929 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2930 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2931 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2932 | lemma fin_ImpL_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2933 | assumes a: "fin (ImpL <a>.M (x).N z) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2934 | shows "z=y \<and> z\<sharp>M \<and> z\<sharp>[x].N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2935 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2936 | apply(erule_tac fin.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2937 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2938 | apply(subgoal_tac "y\<sharp>[aa].Ma") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2939 | apply(drule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2940 | apply(simp_all add: abs_fresh) | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 2941 | apply (metis abs_fresh(5)) | 
| 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 2942 | done | 
| 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 2943 | |
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2944 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2945 | lemma fin_rest_elims: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2946 | shows "fin (Cut <a>.M (x).N) y \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2947 | and "fin (NotR (x).M c) y \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2948 | and "fin (AndR <a>.M <b>.N c) y \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2949 | and "fin (OrR1 <a>.M b) y \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2950 | and "fin (OrR2 <a>.M b) y \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2951 | and "fin (ImpR (x).<a>.M b) y \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2952 | by (erule fin.cases, simp_all add: trm.inject)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2953 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2954 | lemmas fin_elims = fin_Ax_elim fin_NotL_elim fin_AndL1_elim fin_AndL2_elim fin_OrL_elim | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2955 | fin_ImpL_elim fin_rest_elims | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2956 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2957 | lemma fin_rename: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2958 | shows "fin M x \<Longrightarrow> fin ([(x',x)]\<bullet>M) x'" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2959 | by (induct rule: fin.induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2960 | (auto simp add: calc_atm simp add: fresh_left abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2961 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2962 | lemma not_fin_subst1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2963 | assumes a: "\<not>(fin M x)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2964 |   shows "\<not>(fin (M{c:=(y).P}) x)"
 | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 2965 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2966 | apply(nominal_induct M avoiding: x c y P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2967 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2968 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2969 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2970 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2971 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm{coname:=(y).P},P,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2972 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2973 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2974 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2975 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2976 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2977 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2978 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2979 | apply(drule fin_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2980 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2981 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2982 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2983 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm1{coname3:=(y).P},trm2{coname3:=(y).P},P,coname1,coname2,coname3,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2984 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2985 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2986 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2987 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2988 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2989 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm1{coname3:=(y).P},trm2{coname3:=(y).P},P,coname1,coname2,coname3,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2990 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2991 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2992 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2993 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2994 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2995 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2996 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2997 | apply(drule fin_AndL1_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2998 | apply(auto simp add: abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 2999 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3000 | apply(subgoal_tac "name2\<sharp>[name1]. trm") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3001 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3002 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3003 | apply(drule fin_AndL2_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3004 | apply(auto simp add: abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3005 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3006 | apply(subgoal_tac "name2\<sharp>[name1].trm") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3007 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3008 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3009 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm{coname2:=(y).P},coname1,P,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3010 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3011 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3012 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3013 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3014 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3015 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3016 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3017 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm{coname2:=(y).P},coname1,P,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3018 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3019 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3020 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3021 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3022 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3023 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3024 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3025 | apply(drule fin_OrL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3026 | apply(auto simp add: abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3027 | apply(drule freshn_after_substc)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3028 | apply(subgoal_tac "name3\<sharp>[name1].trm1 \<and> name3\<sharp>[name2].trm2") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3029 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3030 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3031 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm{coname2:=(y).P},coname1,P,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3032 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3033 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3034 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3035 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3036 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3037 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3038 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3039 | apply(drule fin_ImpL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3040 | apply(auto simp add: abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3041 | apply(drule freshn_after_substc)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3042 | apply(subgoal_tac "x\<sharp>[name1].trm2") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3043 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3044 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3045 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3046 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3047 | lemma not_fin_subst2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3048 | assumes a: "\<not>(fin M x)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3049 |   shows "\<not>(fin (M{y:=<c>.P}) x)"
 | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 3050 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3051 | apply(nominal_induct M avoiding: x c y P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3052 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3053 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3054 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3055 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3056 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3057 | apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(trm{y:=<c>.P},P,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3058 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3059 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3060 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3061 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3062 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3063 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3064 | apply(drule fin_NotL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3065 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3066 | apply(drule freshn_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3067 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3068 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3069 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3070 | apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(trm{y:=<c>.P},P,name1,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3071 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3072 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3073 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3074 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3075 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3076 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3077 | apply(drule fin_AndL1_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3078 | apply(auto simp add: abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3079 | apply(drule freshn_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3080 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3081 | apply(subgoal_tac "name2\<sharp>[name1]. trm") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3082 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3083 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3084 | apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(trm{y:=<c>.P},P,name1,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3085 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3086 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3087 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3088 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3089 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3090 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3091 | apply(drule fin_AndL2_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3092 | apply(auto simp add: abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3093 | apply(drule freshn_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3094 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3095 | apply(subgoal_tac "name2\<sharp>[name1].trm") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3096 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3097 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3098 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3099 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3100 | apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(trm1{y:=<c>.P},trm2{y:=<c>.P},name1,name2,P,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3101 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3102 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3103 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3104 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3105 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3106 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3107 | apply(drule fin_OrL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3108 | apply(auto simp add: abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3109 | apply(drule freshn_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3110 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3111 | apply(drule freshn_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3112 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3113 | apply(subgoal_tac "name3\<sharp>[name1].trm1 \<and> name3\<sharp>[name2].trm2") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3114 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3115 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3116 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3117 | apply(subgoal_tac "\<exists>a'::name. a'\<sharp>(trm1{name2:=<c>.P},trm2{name2:=<c>.P},name1,P,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3118 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3119 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3120 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3121 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3122 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3123 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3124 | apply(drule fin_ImpL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3125 | apply(auto simp add: abs_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3126 | apply(drule freshn_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3127 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3128 | apply(drule freshn_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3129 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3130 | apply(subgoal_tac "x\<sharp>[name1].trm2") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3131 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3132 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3133 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3134 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3135 | lemma fin_subst1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3136 | assumes a: "fin M x" "x\<noteq>y" "x\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3137 |   shows "fin (M{y:=<c>.P}) x"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3138 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3139 | apply(nominal_induct M avoiding: x y c P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3140 | apply(auto dest!: fin_elims simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3141 | apply(rule fin.intros, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3142 | apply(rule fin.intros, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3143 | apply(rule fin.intros, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3144 | apply(rule fin.intros, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3145 | apply(rule fin.intros, simp add: subst_fresh abs_fresh, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3146 | apply(rule fin.intros, simp add: subst_fresh abs_fresh, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3147 | apply(rule fin.intros, simp add: subst_fresh abs_fresh, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3148 | apply(rule fin.intros, simp add: subst_fresh abs_fresh, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3149 | apply(rule fin.intros, simp add: subst_fresh abs_fresh, simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3150 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3151 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3152 | lemma fin_subst2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3153 | assumes a: "fin M y" "x\<noteq>y" "y\<sharp>P" "M\<noteq>Ax y c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3154 |   shows "fin (M{c:=(x).P}) y"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3155 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3156 | apply(nominal_induct M avoiding: x y c P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3157 | apply(drule fin_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3158 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3159 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3160 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3161 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3162 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3163 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3164 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3165 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3166 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3167 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3168 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3169 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3170 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3171 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3172 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3173 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3174 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3175 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3176 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3177 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3178 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3179 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3180 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3181 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3182 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3183 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3184 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3185 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3186 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3187 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3188 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3189 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3190 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3191 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3192 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3193 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3194 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3195 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3196 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3197 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3198 | lemma fin_substn_nrename: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3199 | assumes a: "fin M x" "x\<noteq>y" "x\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3200 |   shows "M[x\<turnstile>n>y]{y:=<c>.P} = Cut <c>.P (x).(M{y:=<c>.P})"
 | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 3201 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3202 | apply(nominal_induct M avoiding: x y c P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3203 | apply(drule fin_Ax_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3204 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3205 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3206 | apply(simp add: alpha calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3207 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3208 | apply(drule fin_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3209 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3210 | apply(drule fin_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3211 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3212 | apply(drule fin_NotL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3213 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3214 | apply(subgoal_tac "\<exists>z::name. z\<sharp>(trm,y,x,P,trm[x\<turnstile>n>y]{y:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3215 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3216 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3217 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3218 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3219 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3220 | apply(simp add: nsubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3221 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3222 | apply(simp add: nrename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3223 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3224 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3225 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3226 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3227 | apply(drule fin_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3228 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3229 | apply(drule fin_AndL1_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3230 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3231 | apply(subgoal_tac "\<exists>z::name. z\<sharp>(name2,name1,P,trm[name2\<turnstile>n>y]{y:=<c>.P},y,P,trm)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3232 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3233 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3234 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3235 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3236 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3237 | apply(simp add: nsubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3238 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3239 | apply(simp add: nrename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3240 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3241 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3242 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3243 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3244 | apply(drule fin_AndL2_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3245 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3246 | apply(subgoal_tac "\<exists>z::name. z\<sharp>(name2,name1,P,trm[name2\<turnstile>n>y]{y:=<c>.P},y,P,trm)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3247 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3248 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3249 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3250 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3251 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3252 | apply(simp add: nsubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3253 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3254 | apply(simp add: nrename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3255 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3256 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3257 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3258 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3259 | apply(drule fin_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3260 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3261 | apply(drule fin_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3262 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3263 | apply(drule fin_OrL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3264 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3265 | apply(simp add: subst_fresh rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3266 | apply(subgoal_tac "\<exists>z::name. z\<sharp>(name3,name2,name1,P,trm1[name3\<turnstile>n>y]{y:=<c>.P},trm2[name3\<turnstile>n>y]{y:=<c>.P},y,P,trm1,trm2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3267 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3268 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3269 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3270 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3271 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3272 | apply(simp add: nsubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3273 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3274 | apply(simp add: nrename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3275 | apply(simp add: nsubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3276 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3277 | apply(simp add: nrename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3278 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3279 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3280 | apply(drule fin_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3281 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3282 | apply(drule fin_ImpL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3283 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3284 | apply(simp add: subst_fresh rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3285 | apply(subgoal_tac "\<exists>z::name. z\<sharp>(name1,x,P,trm1[x\<turnstile>n>y]{y:=<c>.P},trm2[x\<turnstile>n>y]{y:=<c>.P},y,P,trm1,trm2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3286 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3287 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3288 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3289 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3290 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3291 | apply(simp add: nsubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3292 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3293 | apply(simp add: nrename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3294 | apply(simp add: nsubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3295 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3296 | apply(simp add: nrename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3297 | apply(rule exists_fresh') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3298 | apply(rule fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3299 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3300 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3301 | inductive | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3302 | fic :: "trm \<Rightarrow> coname \<Rightarrow> bool" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3303 | where | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3304 | [intro]: "fic (Ax x a) a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3305 | | [intro]: "a\<sharp>M \<Longrightarrow> fic (NotR (x).M a) a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3306 | | [intro]: "\<lbrakk>c\<sharp>[a].M;c\<sharp>[b].N\<rbrakk> \<Longrightarrow> fic (AndR <a>.M <b>.N c) c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3307 | | [intro]: "b\<sharp>[a].M \<Longrightarrow> fic (OrR1 <a>.M b) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3308 | | [intro]: "b\<sharp>[a].M \<Longrightarrow> fic (OrR2 <a>.M b) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3309 | | [intro]: "\<lbrakk>b\<sharp>[a].M\<rbrakk> \<Longrightarrow> fic (ImpR (x).<a>.M b) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3310 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3311 | equivariance fic | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3312 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3313 | lemma fic_Ax_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3314 | assumes a: "fic (Ax x a) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3315 | shows "a=b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3316 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3317 | apply(erule_tac fic.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3318 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3319 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3320 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3321 | lemma fic_NotR_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3322 | assumes a: "fic (NotR (x).M a) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3323 | shows "a=b \<and> b\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3324 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3325 | apply(erule_tac fic.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3326 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3327 | apply(subgoal_tac "b\<sharp>[xa].Ma") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3328 | apply(drule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3329 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3330 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3331 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3332 | lemma fic_OrR1_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3333 | assumes a: "fic (OrR1 <a>.M b) c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3334 | shows "b=c \<and> c\<sharp>[a].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3335 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3336 | apply(erule_tac fic.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3337 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3338 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3339 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3340 | lemma fic_OrR2_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3341 | assumes a: "fic (OrR2 <a>.M b) c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3342 | shows "b=c \<and> c\<sharp>[a].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3343 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3344 | apply(erule_tac fic.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3345 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3346 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3347 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3348 | lemma fic_AndR_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3349 | assumes a: "fic (AndR <a>.M <b>.N c) d" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3350 | shows "c=d \<and> d\<sharp>[a].M \<and> d\<sharp>[b].N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3351 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3352 | apply(erule_tac fic.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3353 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3354 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3355 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3356 | lemma fic_ImpR_elim: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3357 | assumes a: "fic (ImpR (x).<a>.M b) c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3358 | shows "b=c \<and> b\<sharp>[a].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3359 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3360 | apply(erule_tac fic.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3361 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3362 | apply(subgoal_tac "c\<sharp>[xa].[aa].Ma") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3363 | apply(drule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3364 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3365 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3366 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3367 | lemma fic_rest_elims: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3368 | shows "fic (Cut <a>.M (x).N) d \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3369 | and "fic (NotL <a>.M x) d \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3370 | and "fic (OrL (x).M (y).N z) d \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3371 | and "fic (AndL1 (x).M y) d \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3372 | and "fic (AndL2 (x).M y) d \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3373 | and "fic (ImpL <a>.M (x).N y) d \<Longrightarrow> False" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3374 | by (erule fic.cases, simp_all add: trm.inject)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3375 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3376 | lemmas fic_elims = fic_Ax_elim fic_NotR_elim fic_OrR1_elim fic_OrR2_elim fic_AndR_elim | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3377 | fic_ImpR_elim fic_rest_elims | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3378 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3379 | lemma fic_rename: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3380 | shows "fic M a \<Longrightarrow> fic ([(a',a)]\<bullet>M) a'" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3381 | by (induct rule: fic.induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3382 | (auto simp add: calc_atm simp add: fresh_left abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3383 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3384 | lemma not_fic_subst1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3385 | assumes a: "\<not>(fic M a)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3386 |   shows "\<not>(fic (M{y:=<c>.P}) a)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3387 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3388 | apply(nominal_induct M avoiding: a c y P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3389 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3390 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3391 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3392 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3393 | apply(drule fic_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3394 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3395 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3396 | apply(simp add: fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3397 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3398 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3399 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3400 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3401 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3402 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3403 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3404 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3405 | apply(drule fic_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3406 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3407 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3408 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3409 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3410 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3411 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3412 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3413 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3414 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3415 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3416 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3417 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3418 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3419 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{y:=<c>.P},P,name1,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3420 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3421 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3422 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3423 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3424 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3425 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3426 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3427 | apply(drule fic_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3428 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3429 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3430 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3431 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3432 | apply(drule fic_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3433 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3434 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3435 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3436 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3437 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{y:=<c>.P},trm2{y:=<c>.P},P,name1,name2,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3438 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3439 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3440 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3441 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3442 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3443 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3444 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3445 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3446 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3447 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3448 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3449 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},trm2{name2:=<c>.P},P,name1,name2,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3450 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3451 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3452 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3453 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3454 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3455 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3456 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3457 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3458 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3459 | lemma not_fic_subst2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3460 | assumes a: "\<not>(fic M a)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3461 |   shows "\<not>(fic (M{c:=(y).P}) a)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3462 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3463 | apply(nominal_induct M avoiding: a c y P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3464 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3465 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3466 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3467 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3468 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm{coname:=(y).P},P,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3469 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3470 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3471 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3472 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3473 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3474 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3475 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3476 | apply(drule freshc_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3477 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3478 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3479 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3480 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm1{coname3:=(y).P},trm2{coname3:=(y).P},P,coname1,coname2,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3481 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3482 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3483 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3484 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3485 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3486 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3487 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3488 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3489 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3490 | apply(drule freshc_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3491 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3492 | apply(drule freshc_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3493 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3494 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3495 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3496 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3497 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm{coname2:=(y).P},P,coname1,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3498 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3499 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3500 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3501 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3502 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3503 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3504 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3505 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3506 | apply(drule freshc_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3507 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3508 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3509 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm{coname2:=(y).P},P,coname1,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3510 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3511 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3512 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3513 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3514 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3515 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3516 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3517 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3518 | apply(drule freshc_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3519 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3520 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3521 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3522 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm{coname2:=(y).P},P,coname1,a)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3523 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3524 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3525 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3526 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3527 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3528 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3529 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3530 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3531 | apply(drule freshc_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3532 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3533 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3534 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3535 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3536 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3537 | lemma fic_subst1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3538 | assumes a: "fic M a" "a\<noteq>b" "a\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3539 |   shows "fic (M{b:=(x).P}) a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3540 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3541 | apply(nominal_induct M avoiding: x b a P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3542 | apply(drule fic_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3543 | apply(simp add: fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3544 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3545 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3546 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3547 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3548 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3549 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3550 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3551 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3552 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3553 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3554 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3555 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3556 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3557 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3558 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3559 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3560 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3561 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3562 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3563 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3564 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3565 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3566 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3567 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3568 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3569 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3570 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3571 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3572 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3573 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3574 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3575 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3576 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3577 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3578 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3579 | lemma fic_subst2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3580 | assumes a: "fic M a" "c\<noteq>a" "a\<sharp>P" "M\<noteq>Ax x a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3581 |   shows "fic (M{x:=<c>.P}) a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3582 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3583 | apply(nominal_induct M avoiding: x a c P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3584 | apply(drule fic_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3585 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3586 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3587 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3588 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3589 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3590 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3591 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3592 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3593 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3594 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3595 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3596 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3597 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3598 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3599 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3600 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3601 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3602 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3603 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3604 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3605 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3606 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3607 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3608 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3609 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3610 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3611 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3612 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3613 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3614 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3615 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3616 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3617 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3618 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3619 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3620 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3621 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3622 | lemma fic_substc_crename: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3623 | assumes a: "fic M a" "a\<noteq>b" "a\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3624 |   shows "M[a\<turnstile>c>b]{b:=(y).P} = Cut <a>.(M{b:=(y).P}) (y).P"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3625 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3626 | apply(nominal_induct M avoiding: a b y P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3627 | apply(drule fic_Ax_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3628 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3629 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3630 | apply(simp add: alpha calc_atm fresh_atm trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3631 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3632 | apply(drule fic_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3633 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3634 | apply(drule fic_NotR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3635 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3636 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3637 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3638 | apply(simp add: trm.inject alpha fresh_atm fresh_prod fresh_atm calc_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3639 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3640 | apply(simp add: csubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3641 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3642 | apply(simp add: crename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3643 | apply(rule subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3644 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3645 | apply(drule fic_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3646 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3647 | apply(drule fic_AndR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3648 | apply(simp add: abs_fresh fresh_atm subst_fresh rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3649 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3650 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3651 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3652 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3653 | apply(simp add: csubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3654 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3655 | apply(simp add: csubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3656 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3657 | apply(simp add: subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3658 | apply(drule fic_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3659 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3660 | apply(drule fic_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3661 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3662 | apply(drule fic_OrR1_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3663 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3664 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3665 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3666 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3667 | apply(simp add: csubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3668 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3669 | apply(simp add: subst_fresh rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3670 | apply(drule fic_OrR2_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3671 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3672 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3673 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3674 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3675 | apply(simp add: csubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3676 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3677 | apply(simp add: subst_fresh rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3678 | apply(drule fic_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3679 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3680 | apply(drule fic_ImpR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3681 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3682 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3683 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3684 | apply(simp add: trm.inject alpha fresh_atm calc_atm abs_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3685 | apply(simp add: csubst_eqvt calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3686 | apply(simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3687 | apply(simp add: subst_fresh rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3688 | apply(drule fic_rest_elims) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3689 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3690 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3691 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3692 | inductive | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3693 |   l_redu :: "trm \<Rightarrow> trm \<Rightarrow> bool" ("_ \<longrightarrow>\<^sub>l _" [100,100] 100)
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3694 | where | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3695 | LAxR: "\<lbrakk>x\<sharp>M; a\<sharp>b; fic M a\<rbrakk> \<Longrightarrow> Cut <a>.M (x).(Ax x b) \<longrightarrow>\<^sub>l M[a\<turnstile>c>b]" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3696 | | LAxL: "\<lbrakk>a\<sharp>M; x\<sharp>y; fin M x\<rbrakk> \<Longrightarrow> Cut <a>.(Ax y a) (x).M \<longrightarrow>\<^sub>l M[x\<turnstile>n>y]" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3697 | | LNot: "\<lbrakk>y\<sharp>(M,N); x\<sharp>(N,y); a\<sharp>(M,N,b); b\<sharp>M; y\<noteq>x; b\<noteq>a\<rbrakk> \<Longrightarrow> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3698 | Cut <a>.(NotR (x).M a) (y).(NotL <b>.N y) \<longrightarrow>\<^sub>l Cut <b>.N (x).M" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3699 | | LAnd1: "\<lbrakk>b\<sharp>([a1].M1,[a2].M2,N,a1,a2); y\<sharp>([x].N,M1,M2,x); x\<sharp>(M1,M2); a1\<sharp>(M2,N); a2\<sharp>(M1,N); a1\<noteq>a2\<rbrakk> \<Longrightarrow> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3700 | Cut <b>.(AndR <a1>.M1 <a2>.M2 b) (y).(AndL1 (x).N y) \<longrightarrow>\<^sub>l Cut <a1>.M1 (x).N" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3701 | | LAnd2: "\<lbrakk>b\<sharp>([a1].M1,[a2].M2,N,a1,a2); y\<sharp>([x].N,M1,M2,x); x\<sharp>(M1,M2); a1\<sharp>(M2,N); a2\<sharp>(M1,N); a1\<noteq>a2\<rbrakk> \<Longrightarrow> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3702 | Cut <b>.(AndR <a1>.M1 <a2>.M2 b) (y).(AndL2 (x).N y) \<longrightarrow>\<^sub>l Cut <a2>.M2 (x).N" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3703 | | LOr1: "\<lbrakk>b\<sharp>([a].M,N1,N2,a); y\<sharp>([x1].N1,[x2].N2,M,x1,x2); x1\<sharp>(M,N2); x2\<sharp>(M,N1); a\<sharp>(N1,N2); x1\<noteq>x2\<rbrakk> \<Longrightarrow> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3704 | Cut <b>.(OrR1 <a>.M b) (y).(OrL (x1).N1 (x2).N2 y) \<longrightarrow>\<^sub>l Cut <a>.M (x1).N1" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3705 | | LOr2: "\<lbrakk>b\<sharp>([a].M,N1,N2,a); y\<sharp>([x1].N1,[x2].N2,M,x1,x2); x1\<sharp>(M,N2); x2\<sharp>(M,N1); a\<sharp>(N1,N2); x1\<noteq>x2\<rbrakk> \<Longrightarrow> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3706 | Cut <b>.(OrR2 <a>.M b) (y).(OrL (x1).N1 (x2).N2 y) \<longrightarrow>\<^sub>l Cut <a>.M (x2).N2" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3707 | | LImp: "\<lbrakk>z\<sharp>(N,[y].P,[x].M,y,x); b\<sharp>([a].M,[c].N,P,c,a); x\<sharp>(N,[y].P,y); | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3708 | c\<sharp>(P,[a].M,b,a); a\<sharp>([c].N,P); y\<sharp>(N,[x].M)\<rbrakk> \<Longrightarrow> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3709 | Cut <b>.(ImpR (x).<a>.M b) (z).(ImpL <c>.N (y).P z) \<longrightarrow>\<^sub>l Cut <a>.(Cut <c>.N (x).M) (y).P" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3710 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3711 | equivariance l_redu | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3712 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3713 | lemma l_redu_eqvt': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3714 | fixes pi1::"name prm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3715 | and pi2::"coname prm" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3716 | shows "(pi1\<bullet>M) \<longrightarrow>\<^sub>l (pi1\<bullet>M') \<Longrightarrow> M \<longrightarrow>\<^sub>l M'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3717 | and "(pi2\<bullet>M) \<longrightarrow>\<^sub>l (pi2\<bullet>M') \<Longrightarrow> M \<longrightarrow>\<^sub>l M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3718 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3719 | apply(drule_tac pi="rev pi1" in l_redu.eqvt(1)) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3720 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3721 | apply(drule_tac pi="rev pi2" in l_redu.eqvt(2)) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3722 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3723 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3724 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3725 | nominal_inductive l_redu | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3726 | apply(simp_all add: abs_fresh fresh_atm rename_fresh fresh_prod abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3727 | apply(force)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3728 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3729 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3730 | lemma fresh_l_redu: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3731 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3732 | and a::"coname" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3733 | shows "M \<longrightarrow>\<^sub>l M' \<Longrightarrow> x\<sharp>M \<Longrightarrow> x\<sharp>M'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3734 | and "M \<longrightarrow>\<^sub>l M' \<Longrightarrow> a\<sharp>M \<Longrightarrow> a\<sharp>M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3735 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3736 | apply(induct rule: l_redu.induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3737 | apply(auto simp add: abs_fresh rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3738 | apply(case_tac "xa=x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3739 | apply(simp add: rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3740 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3741 | apply(simp add: fresh_prod abs_fresh abs_supp fin_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3742 | apply(induct rule: l_redu.induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3743 | apply(auto simp add: abs_fresh rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3744 | apply(case_tac "aa=a") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3745 | apply(simp add: rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3746 | apply(simp add: rename_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3747 | apply(simp add: fresh_prod abs_fresh abs_supp fin_supp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3748 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3749 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3750 | lemma better_LAxR_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3751 | shows "fic M a \<Longrightarrow> Cut <a>.M (x).(Ax x b) \<longrightarrow>\<^sub>l M[a\<turnstile>c>b]" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3752 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3753 | assume fin: "fic M a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3754 | obtain x'::"name" where fs1: "x'\<sharp>(M,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3755 | obtain a'::"coname" where fs2: "a'\<sharp>(a,M,b)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3756 | have "Cut <a>.M (x).(Ax x b) = Cut <a'>.([(a',a)]\<bullet>M) (x').(Ax x' b)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3757 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3758 | also have "\<dots> \<longrightarrow>\<^sub>l ([(a',a)]\<bullet>M)[a'\<turnstile>c>b]" using fs1 fs2 fin | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3759 | by (auto intro: l_redu.intros simp add: fresh_left calc_atm fic_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3760 | also have "\<dots> = M[a\<turnstile>c>b]" using fs1 fs2 by (simp add: crename_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3761 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3762 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3763 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3764 | lemma better_LAxL_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3765 | shows "fin M x \<Longrightarrow> Cut <a>.(Ax y a) (x).M \<longrightarrow>\<^sub>l M[x\<turnstile>n>y]" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3766 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3767 | assume fin: "fin M x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3768 | obtain x'::"name" where fs1: "x'\<sharp>(y,M,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3769 | obtain a'::"coname" where fs2: "a'\<sharp>(a,M)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3770 | have "Cut <a>.(Ax y a) (x).M = Cut <a'>.(Ax y a') (x').([(x',x)]\<bullet>M)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3771 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3772 | also have "\<dots> \<longrightarrow>\<^sub>l ([(x',x)]\<bullet>M)[x'\<turnstile>n>y]" using fs1 fs2 fin | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3773 | by (auto intro: l_redu.intros simp add: fresh_left calc_atm fin_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3774 | also have "\<dots> = M[x\<turnstile>n>y]" using fs1 fs2 by (simp add: nrename_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3775 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3776 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3777 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3778 | lemma better_LNot_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3779 | shows "\<lbrakk>y\<sharp>N; a\<sharp>M\<rbrakk> \<Longrightarrow> Cut <a>.(NotR (x).M a) (y).(NotL <b>.N y) \<longrightarrow>\<^sub>l Cut <b>.N (x).M" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3780 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3781 | assume fs: "y\<sharp>N" "a\<sharp>M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3782 | obtain x'::"name" where f1: "x'\<sharp>(y,N,M,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3783 | obtain y'::"name" where f2: "y'\<sharp>(y,N,M,x,x')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3784 | obtain a'::"coname" where f3: "a'\<sharp>(a,M,N,b)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3785 | obtain b'::"coname" where f4: "b'\<sharp>(a,M,N,b,a')" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3786 | have "Cut <a>.(NotR (x).M a) (y).(NotL <b>.N y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3787 | = Cut <a'>.(NotR (x).([(a',a)]\<bullet>M) a') (y').(NotL <b>.([(y',y)]\<bullet>N) y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3788 | using f1 f2 f3 f4 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3789 | by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3790 | also have "\<dots> = Cut <a'>.(NotR (x).M a') (y').(NotL <b>.N y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3791 | using f1 f2 f3 f4 fs by (perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3792 | also have "\<dots> = Cut <a'>.(NotR (x').([(x',x)]\<bullet>M) a') (y').(NotL <b'>.([(b',b)]\<bullet>N) y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3793 | using f1 f2 f3 f4 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3794 | by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3795 | also have "\<dots> \<longrightarrow>\<^sub>l Cut <b'>.([(b',b)]\<bullet>N) (x').([(x',x)]\<bullet>M)" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3796 | using f1 f2 f3 f4 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3797 | by (auto intro: l_redu.intros simp add: fresh_prod fresh_left calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3798 | also have "\<dots> = Cut <b>.N (x).M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3799 | using f1 f2 f3 f4 by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3800 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3801 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3802 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3803 | lemma better_LAnd1_intro[intro]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3804 | shows "\<lbrakk>a\<sharp>([b1].M1,[b2].M2); y\<sharp>[x].N\<rbrakk> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3805 | \<Longrightarrow> Cut <a>.(AndR <b1>.M1 <b2>.M2 a) (y).(AndL1 (x).N y) \<longrightarrow>\<^sub>l Cut <b1>.M1 (x).N" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3806 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3807 | assume fs: "a\<sharp>([b1].M1,[b2].M2)" "y\<sharp>[x].N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3808 | obtain x'::"name" where f1: "x'\<sharp>(y,N,M1,M2,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3809 | obtain y'::"name" where f2: "y'\<sharp>(y,N,M1,M2,x,x')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3810 | obtain a'::"coname" where f3: "a'\<sharp>(a,M1,M2,N,b1,b2)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3811 | obtain b1'::"coname" where f4:"b1'\<sharp>(a,M1,M2,N,b1,b2,a')" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3812 | obtain b2'::"coname" where f5:"b2'\<sharp>(a,M1,M2,N,b1,b2,a',b1')" by (rule exists_fresh(2),rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3813 | have "Cut <a>.(AndR <b1>.M1 <b2>.M2 a) (y).(AndL1 (x).N y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3814 | = Cut <a'>.(AndR <b1>.M1 <b2>.M2 a') (y').(AndL1 (x).N y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3815 | using f1 f2 f3 f4 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3816 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3817 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3818 | apply(auto simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3819 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3820 | also have "\<dots> = Cut <a'>.(AndR <b1'>.([(b1',b1)]\<bullet>M1) <b2'>.([(b2',b2)]\<bullet>M2) a') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3821 | (y').(AndL1 (x').([(x',x)]\<bullet>N) y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3822 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3823 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3824 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3825 | done | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3826 | also have "\<dots> \<longrightarrow>\<^sub>l Cut <b1'>.([(b1',b1)]\<bullet>M1) (x').([(x',x)]\<bullet>N)" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3827 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3828 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3829 | apply(rule l_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3830 | apply(auto simp add: abs_fresh fresh_prod fresh_left calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3831 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3832 | also have "\<dots> = Cut <b1>.M1 (x).N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3833 | using f1 f2 f3 f4 f5 fs by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3834 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3835 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3836 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3837 | lemma better_LAnd2_intro[intro]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3838 | shows "\<lbrakk>a\<sharp>([b1].M1,[b2].M2); y\<sharp>[x].N\<rbrakk> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3839 | \<Longrightarrow> Cut <a>.(AndR <b1>.M1 <b2>.M2 a) (y).(AndL2 (x).N y) \<longrightarrow>\<^sub>l Cut <b2>.M2 (x).N" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3840 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3841 | assume fs: "a\<sharp>([b1].M1,[b2].M2)" "y\<sharp>[x].N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3842 | obtain x'::"name" where f1: "x'\<sharp>(y,N,M1,M2,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3843 | obtain y'::"name" where f2: "y'\<sharp>(y,N,M1,M2,x,x')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3844 | obtain a'::"coname" where f3: "a'\<sharp>(a,M1,M2,N,b1,b2)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3845 | obtain b1'::"coname" where f4:"b1'\<sharp>(a,M1,M2,N,b1,b2,a')" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3846 | obtain b2'::"coname" where f5:"b2'\<sharp>(a,M1,M2,N,b1,b2,a',b1')" by (rule exists_fresh(2),rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3847 | have "Cut <a>.(AndR <b1>.M1 <b2>.M2 a) (y).(AndL2 (x).N y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3848 | = Cut <a'>.(AndR <b1>.M1 <b2>.M2 a') (y').(AndL2 (x).N y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3849 | using f1 f2 f3 f4 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3850 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3851 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3852 | apply(auto simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3853 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3854 | also have "\<dots> = Cut <a'>.(AndR <b1'>.([(b1',b1)]\<bullet>M1) <b2'>.([(b2',b2)]\<bullet>M2) a') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3855 | (y').(AndL2 (x').([(x',x)]\<bullet>N) y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3856 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3857 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3858 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3859 | done | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3860 | also have "\<dots> \<longrightarrow>\<^sub>l Cut <b2'>.([(b2',b2)]\<bullet>M2) (x').([(x',x)]\<bullet>N)" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3861 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3862 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3863 | apply(rule l_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3864 | apply(auto simp add: abs_fresh fresh_prod fresh_left calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3865 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3866 | also have "\<dots> = Cut <b2>.M2 (x).N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3867 | using f1 f2 f3 f4 f5 fs by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3868 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3869 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3870 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3871 | lemma better_LOr1_intro[intro]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3872 | shows "\<lbrakk>y\<sharp>([x1].N1,[x2].N2); b\<sharp>[a].M\<rbrakk> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3873 | \<Longrightarrow> Cut <b>.(OrR1 <a>.M b) (y).(OrL (x1).N1 (x2).N2 y) \<longrightarrow>\<^sub>l Cut <a>.M (x1).N1" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3874 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3875 | assume fs: "y\<sharp>([x1].N1,[x2].N2)" "b\<sharp>[a].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3876 | obtain y'::"name" where f1: "y'\<sharp>(y,M,N1,N2,x1,x2)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3877 | obtain x1'::"name" where f2: "x1'\<sharp>(y,M,N1,N2,x1,x2,y')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3878 | obtain x2'::"name" where f3: "x2'\<sharp>(y,M,N1,N2,x1,x2,y',x1')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3879 | obtain a'::"coname" where f4: "a'\<sharp>(a,N1,N2,M,b)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3880 | obtain b'::"coname" where f5: "b'\<sharp>(a,N1,N2,M,b,a')" by (rule exists_fresh(2),rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3881 | have "Cut <b>.(OrR1 <a>.M b) (y).(OrL (x1).N1 (x2).N2 y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3882 | = Cut <b'>.(OrR1 <a>.M b') (y').(OrL (x1).N1 (x2).N2 y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3883 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3884 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3885 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3886 | apply(auto simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3887 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3888 | also have "\<dots> = Cut <b'>.(OrR1 <a'>.([(a',a)]\<bullet>M) b') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3889 | (y').(OrL (x1').([(x1',x1)]\<bullet>N1) (x2').([(x2',x2)]\<bullet>N2) y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3890 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3891 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3892 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3893 | done | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3894 | also have "\<dots> \<longrightarrow>\<^sub>l Cut <a'>.([(a',a)]\<bullet>M) (x1').([(x1',x1)]\<bullet>N1)" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3895 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3896 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3897 | apply(rule l_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3898 | apply(auto simp add: abs_fresh fresh_prod fresh_left calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3899 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3900 | also have "\<dots> = Cut <a>.M (x1).N1" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3901 | using f1 f2 f3 f4 f5 fs by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3902 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3903 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3904 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3905 | lemma better_LOr2_intro[intro]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3906 | shows "\<lbrakk>y\<sharp>([x1].N1,[x2].N2); b\<sharp>[a].M\<rbrakk> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3907 | \<Longrightarrow> Cut <b>.(OrR2 <a>.M b) (y).(OrL (x1).N1 (x2).N2 y) \<longrightarrow>\<^sub>l Cut <a>.M (x2).N2" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3908 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3909 | assume fs: "y\<sharp>([x1].N1,[x2].N2)" "b\<sharp>[a].M" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3910 | obtain y'::"name" where f1: "y'\<sharp>(y,M,N1,N2,x1,x2)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3911 | obtain x1'::"name" where f2: "x1'\<sharp>(y,M,N1,N2,x1,x2,y')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3912 | obtain x2'::"name" where f3: "x2'\<sharp>(y,M,N1,N2,x1,x2,y',x1')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3913 | obtain a'::"coname" where f4: "a'\<sharp>(a,N1,N2,M,b)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3914 | obtain b'::"coname" where f5: "b'\<sharp>(a,N1,N2,M,b,a')" by (rule exists_fresh(2),rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3915 | have "Cut <b>.(OrR2 <a>.M b) (y).(OrL (x1).N1 (x2).N2 y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3916 | = Cut <b'>.(OrR2 <a>.M b') (y').(OrL (x1).N1 (x2).N2 y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3917 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3918 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3919 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3920 | apply(auto simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3921 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3922 | also have "\<dots> = Cut <b'>.(OrR2 <a'>.([(a',a)]\<bullet>M) b') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3923 | (y').(OrL (x1').([(x1',x1)]\<bullet>N1) (x2').([(x2',x2)]\<bullet>N2) y')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3924 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3925 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3926 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3927 | done | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3928 | also have "\<dots> \<longrightarrow>\<^sub>l Cut <a'>.([(a',a)]\<bullet>M) (x2').([(x2',x2)]\<bullet>N2)" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3929 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3930 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3931 | apply(rule l_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3932 | apply(auto simp add: abs_fresh fresh_prod fresh_left calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3933 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3934 | also have "\<dots> = Cut <a>.M (x2).N2" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3935 | using f1 f2 f3 f4 f5 fs by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3936 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3937 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3938 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3939 | lemma better_LImp_intro[intro]: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3940 | shows "\<lbrakk>z\<sharp>(N,[y].P); b\<sharp>[a].M; a\<sharp>N\<rbrakk> | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3941 | \<Longrightarrow> Cut <b>.(ImpR (x).<a>.M b) (z).(ImpL <c>.N (y).P z) \<longrightarrow>\<^sub>l Cut <a>.(Cut <c>.N (x).M) (y).P" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3942 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3943 | assume fs: "z\<sharp>(N,[y].P)" "b\<sharp>[a].M" "a\<sharp>N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3944 | obtain y'::"name" where f1: "y'\<sharp>(y,M,N,P,z,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3945 | obtain x'::"name" where f2: "x'\<sharp>(y,M,N,P,z,x,y')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3946 | obtain z'::"name" where f3: "z'\<sharp>(y,M,N,P,z,x,y',x')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3947 | obtain a'::"coname" where f4: "a'\<sharp>(a,N,P,M,b)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3948 | obtain b'::"coname" where f5: "b'\<sharp>(a,N,P,M,b,c,a')" by (rule exists_fresh(2),rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3949 | obtain c'::"coname" where f6: "c'\<sharp>(a,N,P,M,b,c,a',b')" by (rule exists_fresh(2),rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3950 | have " Cut <b>.(ImpR (x).<a>.M b) (z).(ImpL <c>.N (y).P z) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3951 | = Cut <b'>.(ImpR (x).<a>.M b') (z').(ImpL <c>.N (y).P z')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3952 | using f1 f2 f3 f4 f5 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3953 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3954 | apply(perm_simp add: trm.inject alpha calc_atm fresh_prod fresh_left fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3955 | apply(auto simp add: perm_fresh_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3956 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3957 | also have "\<dots> = Cut <b'>.(ImpR (x').<a'>.([(a',a)]\<bullet>([(x',x)]\<bullet>M)) b') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3958 | (z').(ImpL <c'>.([(c',c)]\<bullet>N) (y').([(y',y)]\<bullet>P) z')" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3959 | using f1 f2 f3 f4 f5 f6 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3960 | apply(rule_tac sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3961 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3962 | apply(simp add: alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3963 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3964 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3965 | apply(simp add: alpha fresh_prod fresh_atm abs_perm calc_atm fresh_left abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3966 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3967 | apply(simp add: alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3968 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3969 | apply(simp add: alpha fresh_prod fresh_atm abs_perm calc_atm fresh_left abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3970 | apply(simp add: alpha fresh_prod fresh_atm abs_perm calc_atm fresh_left abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3971 | done | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 3972 | also have "\<dots> \<longrightarrow>\<^sub>l Cut <a'>.(Cut <c'>.([(c',c)]\<bullet>N) (x').([(a',a)]\<bullet>[(x',x)]\<bullet>M)) (y').([(y',y)]\<bullet>P)" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3973 | using f1 f2 f3 f4 f5 f6 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3974 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3975 | apply(rule l_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3976 | apply(auto simp add: abs_fresh fresh_prod fresh_left calc_atm fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3977 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3978 | also have "\<dots> = Cut <a>.(Cut <c>.N (x).M) (y).P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3979 | using f1 f2 f3 f4 f5 f6 fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3980 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3981 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3982 | apply(simp add: alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3983 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3984 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3985 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3986 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3987 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3988 | apply(perm_simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3989 | apply(auto simp add: fresh_prod fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3990 | apply(perm_simp add: alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3991 | apply(perm_simp add: alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3992 | apply(perm_simp add: alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3993 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3994 | apply(perm_simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3995 | apply(rule_tac pi="[(a',a)]" in pt_bij4[OF pt_coname_inst, OF at_coname_inst]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3996 | apply(perm_simp add: abs_perm calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3997 | apply(perm_simp add: alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3998 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 3999 | apply(perm_simp add: alpha fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4000 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4001 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4002 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4003 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4004 | lemma alpha_coname: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4005 | fixes M::"trm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4006 | and a::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4007 | assumes a: "[a].M = [b].N" "c\<sharp>(a,b,M,N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4008 | shows "M = [(a,c)]\<bullet>[(b,c)]\<bullet>N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4009 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4010 | apply(auto simp add: alpha_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4011 | apply(drule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4012 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4013 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4014 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4015 | lemma alpha_name: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4016 | fixes M::"trm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4017 | and x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4018 | assumes a: "[x].M = [y].N" "z\<sharp>(x,y,M,N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4019 | shows "M = [(x,z)]\<bullet>[(y,z)]\<bullet>N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4020 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4021 | apply(auto simp add: alpha_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4022 | apply(drule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4023 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4024 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4025 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4026 | lemma alpha_name_coname: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4027 | fixes M::"trm" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4028 | and x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4029 | and a::"coname" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4030 | assumes a: "[x].[b].M = [y].[c].N" "z\<sharp>(x,y,M,N)" "a\<sharp>(b,c,M,N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4031 | shows "M = [(x,z)]\<bullet>[(b,a)]\<bullet>[(c,a)]\<bullet>[(y,z)]\<bullet>N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4032 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4033 | apply(auto simp add: alpha_fresh fresh_prod fresh_atm | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4034 | abs_supp fin_supp abs_fresh abs_perm fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4035 | apply(drule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4036 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4037 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4038 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4039 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4040 | lemma Cut_l_redu_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4041 | assumes a: "Cut <a>.M (x).N \<longrightarrow>\<^sub>l R" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4042 | shows "(\<exists>b. R = M[a\<turnstile>c>b]) \<or> (\<exists>y. R = N[x\<turnstile>n>y]) \<or> | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4043 | (\<exists>y M' b N'. M = NotR (y).M' a \<and> N = NotL <b>.N' x \<and> R = Cut <b>.N' (y).M' \<and> fic M a \<and> fin N x) \<or> | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4044 | (\<exists>b M1 c M2 y N'. M = AndR <b>.M1 <c>.M2 a \<and> N = AndL1 (y).N' x \<and> R = Cut <b>.M1 (y).N' | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4045 | \<and> fic M a \<and> fin N x) \<or> | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4046 | (\<exists>b M1 c M2 y N'. M = AndR <b>.M1 <c>.M2 a \<and> N = AndL2 (y).N' x \<and> R = Cut <c>.M2 (y).N' | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4047 | \<and> fic M a \<and> fin N x) \<or> | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4048 | (\<exists>b N' z M1 y M2. M = OrR1 <b>.N' a \<and> N = OrL (z).M1 (y).M2 x \<and> R = Cut <b>.N' (z).M1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4049 | \<and> fic M a \<and> fin N x) \<or> | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4050 | (\<exists>b N' z M1 y M2. M = OrR2 <b>.N' a \<and> N = OrL (z).M1 (y).M2 x \<and> R = Cut <b>.N' (y).M2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4051 | \<and> fic M a \<and> fin N x) \<or> | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4052 | (\<exists>z b M' c N1 y N2. M = ImpR (z).<b>.M' a \<and> N = ImpL <c>.N1 (y).N2 x \<and> | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4053 | R = Cut <b>.(Cut <c>.N1 (z).M') (y).N2 \<and> b\<sharp>(c,N1) \<and> fic M a \<and> fin N x)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4054 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4055 | apply(erule_tac l_redu.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4056 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4057 | (* ax case *) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4058 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4059 | apply(rule_tac x="b" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4060 | apply(erule conjE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4061 | apply(simp add: alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4062 | apply(erule disjE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4063 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4064 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4065 | apply(simp add: rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4066 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4067 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4068 | (* ax case *) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4069 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4070 | apply(rule_tac x="y" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4071 | apply(erule conjE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4072 | apply(thin_tac "[a].M = [aa].Ax y aa") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4073 | apply(simp add: alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4074 | apply(erule disjE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4075 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4076 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4077 | apply(simp add: rename_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4078 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4079 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4080 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4081 | (* not case *) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4082 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4083 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4084 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4085 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4086 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4087 | apply(drule_tac c="c" in alpha_coname) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4088 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4089 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4090 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4091 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4092 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4093 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4094 | apply(simp add: calc_atm abs_fresh fresh_prod fresh_atm fresh_left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4095 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4096 | apply(drule_tac z="ca" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4097 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4098 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4099 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4100 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4101 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4102 | apply(auto simp add: calc_atm abs_fresh fresh_left)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4103 | apply(case_tac "y=x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4104 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4105 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4106 | apply(case_tac "aa=a") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4107 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4108 | apply(perm_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4109 | (* and1 case *) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4110 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4111 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4112 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4113 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4114 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4115 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4116 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4117 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4118 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4119 | apply(drule_tac c="c" in alpha_coname) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4120 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4121 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4122 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4123 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4124 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4125 | apply(rule_tac s="a" and t="[(a,c)]\<bullet>[(b,c)]\<bullet>b" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4126 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4127 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4128 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4129 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4130 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4131 | apply(drule_tac z="ca" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4132 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4133 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4134 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4135 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4136 | apply(rule_tac s="x" and t="[(x,ca)]\<bullet>[(y,ca)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4137 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4138 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4139 | apply(auto simp add: fresh_left calc_atm abs_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4140 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4141 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4142 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4143 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4144 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4145 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4146 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4147 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4148 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(y,cb)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4149 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4150 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4151 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4152 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4153 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4154 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4155 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4156 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4157 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4158 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4159 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4160 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4161 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(y,cb)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4162 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4163 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4164 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4165 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4166 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4167 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4168 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4169 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4170 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4171 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4172 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4173 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4174 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(y,cb)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4175 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4176 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4177 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4178 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4179 | (* and2 case *) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4180 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4181 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4182 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4183 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4184 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4185 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4186 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4187 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4188 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4189 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4190 | apply(drule_tac c="c" in alpha_coname) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4191 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4192 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4193 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4194 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4195 | apply(rule_tac s="a" and t="[(a,c)]\<bullet>[(b,c)]\<bullet>b" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4196 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4197 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4198 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4199 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4200 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4201 | apply(drule_tac z="ca" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4202 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4203 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4204 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4205 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4206 | apply(rule_tac s="x" and t="[(x,ca)]\<bullet>[(y,ca)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4207 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4208 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4209 | apply(auto simp add: fresh_left calc_atm abs_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4210 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4211 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4212 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4213 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4214 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4215 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4216 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4217 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4218 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(y,cb)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4219 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4220 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4221 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4222 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4223 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4224 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4225 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4226 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4227 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4228 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4229 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4230 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4231 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(y,cb)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4232 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4233 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4234 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4235 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4236 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4237 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4238 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4239 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4240 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4241 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4242 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4243 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4244 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(y,cb)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4245 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4246 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4247 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4248 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4249 | (* or1 case *) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4250 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4251 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4252 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4253 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4254 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4255 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4256 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4257 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4258 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4259 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4260 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4261 | apply(drule_tac c="c" in alpha_coname) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4262 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4263 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4264 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4265 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4266 | apply(rule_tac s="a" and t="[(a,c)]\<bullet>[(b,c)]\<bullet>b" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4267 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4268 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4269 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4270 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4271 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4272 | apply(drule_tac z="ca" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4273 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4274 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4275 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4276 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4277 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4278 | apply(rule_tac s="x" and t="[(x,ca)]\<bullet>[(y,ca)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4279 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4280 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4281 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4282 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4283 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4284 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4285 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4286 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4287 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4288 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4289 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4290 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4291 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4292 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(y,cb)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4293 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4294 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4295 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4296 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4297 | (* or2 case *) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4298 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4299 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4300 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4301 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4302 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4303 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4304 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4305 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4306 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4307 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4308 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4309 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4310 | apply(drule_tac c="c" in alpha_coname) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4311 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4312 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4313 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4314 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4315 | apply(rule_tac s="a" and t="[(a,c)]\<bullet>[(b,c)]\<bullet>b" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4316 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4317 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4318 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4319 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4320 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4321 | apply(drule_tac z="ca" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4322 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4323 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4324 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4325 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4326 | apply(rule_tac s="x" and t="[(x,ca)]\<bullet>[(y,ca)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4327 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4328 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4329 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4330 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4331 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4332 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4333 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4334 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4335 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4336 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4337 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4338 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4339 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(y,cb)]\<bullet>y" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4340 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4341 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4342 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4343 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4344 | (* imp-case *) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4345 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4346 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4347 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4348 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4349 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4350 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4351 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4352 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4353 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4354 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4355 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4356 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4357 | apply(drule_tac c="ca" in alpha_coname) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4358 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4359 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4360 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4361 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4362 | apply(rule_tac s="a" and t="[(a,ca)]\<bullet>[(b,ca)]\<bullet>b" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4363 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4364 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4365 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4366 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4367 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4368 | apply(drule_tac z="cb" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4369 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4370 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4371 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4372 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4373 | apply(rule_tac s="x" and t="[(x,cb)]\<bullet>[(z,cb)]\<bullet>z" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4374 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4375 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4376 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4377 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4378 | apply(generate_fresh "name") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4379 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4380 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4381 | apply(drule_tac z="cc" in alpha_name) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4382 | apply(simp add: fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4383 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4384 | apply(rule exI)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4385 | apply(rule conjI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4386 | apply(rule_tac s="x" and t="[(x,cc)]\<bullet>[(z,cc)]\<bullet>z" in subst) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4387 | apply(simp add: calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4388 | apply(rule refl) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4389 | apply(auto simp add: fresh_left calc_atm abs_fresh alpha perm_fresh_fresh split: if_splits)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4390 | apply(perm_simp)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4391 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4392 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4393 | inductive | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4394 |   c_redu :: "trm \<Rightarrow> trm \<Rightarrow> bool" ("_ \<longrightarrow>\<^sub>c _" [100,100] 100)
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4395 | where | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4396 |   left[intro]:  "\<lbrakk>\<not>fic M a; a\<sharp>N; x\<sharp>M\<rbrakk> \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>c M{a:=(x).N}"
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4397 | | right[intro]: "\<lbrakk>\<not>fin N x; a\<sharp>N; x\<sharp>M\<rbrakk> \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>c N{x:=<a>.M}"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4398 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4399 | equivariance c_redu | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4400 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4401 | nominal_inductive c_redu | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4402 | by (simp_all add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4403 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4404 | lemma better_left[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4405 |   shows "\<not>fic M a \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>c M{a:=(x).N}"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4406 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4407 | assume not_fic: "\<not>fic M a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4408 | obtain x'::"name" where fs1: "x'\<sharp>(N,M,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4409 | obtain a'::"coname" where fs2: "a'\<sharp>(a,M,N)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4410 | have "Cut <a>.M (x).N = Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4411 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4412 |   also have "\<dots> \<longrightarrow>\<^sub>c ([(a',a)]\<bullet>M){a':=(x').([(x',x)]\<bullet>N)}" using fs1 fs2 not_fic
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4413 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4414 | apply(rule left) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4415 | apply(clarify) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4416 | apply(drule_tac a'="a" in fic_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4417 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4418 | apply(simp add: fresh_left calc_atm)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4419 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4420 |   also have "\<dots> = M{a:=(x).N}" using fs1 fs2
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4421 | by (simp add: subst_rename[symmetric] fresh_atm fresh_prod fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4422 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4423 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4424 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4425 | lemma better_right[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4426 |   shows "\<not>fin N x \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>c N{x:=<a>.M}"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4427 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4428 | assume not_fin: "\<not>fin N x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4429 | obtain x'::"name" where fs1: "x'\<sharp>(N,M,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4430 | obtain a'::"coname" where fs2: "a'\<sharp>(a,M,N)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4431 | have "Cut <a>.M (x).N = Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4432 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4433 |   also have "\<dots> \<longrightarrow>\<^sub>c ([(x',x)]\<bullet>N){x':=<a'>.([(a',a)]\<bullet>M)}" using fs1 fs2 not_fin
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4434 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4435 | apply(rule right) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4436 | apply(clarify) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4437 | apply(drule_tac x'="x" in fin_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4438 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4439 | apply(simp add: fresh_left calc_atm)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4440 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4441 |   also have "\<dots> = N{x:=<a>.M}" using fs1 fs2
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4442 | by (simp add: subst_rename[symmetric] fresh_atm fresh_prod fresh_left calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4443 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4444 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4445 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4446 | lemma fresh_c_redu: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4447 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4448 | and c::"coname" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4449 | shows "M \<longrightarrow>\<^sub>c M' \<Longrightarrow> x\<sharp>M \<Longrightarrow> x\<sharp>M'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4450 | and "M \<longrightarrow>\<^sub>c M' \<Longrightarrow> c\<sharp>M \<Longrightarrow> c\<sharp>M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4451 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4452 | apply(induct rule: c_redu.induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4453 | apply(auto simp add: abs_fresh rename_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4454 | apply(induct rule: c_redu.induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4455 | apply(auto simp add: abs_fresh rename_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4456 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4457 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4458 | inductive | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4459 |   a_redu :: "trm \<Rightarrow> trm \<Rightarrow> bool" ("_ \<longrightarrow>\<^sub>a _" [100,100] 100)
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4460 | where | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4461 | al_redu[intro]: "M\<longrightarrow>\<^sub>l M' \<Longrightarrow> M \<longrightarrow>\<^sub>a M'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4462 | | ac_redu[intro]: "M\<longrightarrow>\<^sub>c M' \<Longrightarrow> M \<longrightarrow>\<^sub>a M'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4463 | | a_Cut_l: "\<lbrakk>a\<sharp>N; x\<sharp>M; M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>a Cut <a>.M' (x).N" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4464 | | a_Cut_r: "\<lbrakk>a\<sharp>N; x\<sharp>M; N\<longrightarrow>\<^sub>a N'\<rbrakk> \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>a Cut <a>.M (x).N'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4465 | | a_NotL[intro]: "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> NotL <a>.M x \<longrightarrow>\<^sub>a NotL <a>.M' x" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4466 | | a_NotR[intro]: "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> NotR (x).M a \<longrightarrow>\<^sub>a NotR (x).M' a" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4467 | | a_AndR_l: "\<lbrakk>a\<sharp>(N,c); b\<sharp>(M,c); b\<noteq>a; M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> AndR <a>.M <b>.N c \<longrightarrow>\<^sub>a AndR <a>.M' <b>.N c" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4468 | | a_AndR_r: "\<lbrakk>a\<sharp>(N,c); b\<sharp>(M,c); b\<noteq>a; N\<longrightarrow>\<^sub>a N'\<rbrakk> \<Longrightarrow> AndR <a>.M <b>.N c \<longrightarrow>\<^sub>a AndR <a>.M <b>.N' c" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4469 | | a_AndL1: "\<lbrakk>x\<sharp>y; M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> AndL1 (x).M y \<longrightarrow>\<^sub>a AndL1 (x).M' y" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4470 | | a_AndL2: "\<lbrakk>x\<sharp>y; M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> AndL2 (x).M y \<longrightarrow>\<^sub>a AndL2 (x).M' y" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4471 | | a_OrL_l: "\<lbrakk>x\<sharp>(N,z); y\<sharp>(M,z); y\<noteq>x; M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> OrL (x).M (y).N z \<longrightarrow>\<^sub>a OrL (x).M' (y).N z" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4472 | | a_OrL_r: "\<lbrakk>x\<sharp>(N,z); y\<sharp>(M,z); y\<noteq>x; N\<longrightarrow>\<^sub>a N'\<rbrakk> \<Longrightarrow> OrL (x).M (y).N z \<longrightarrow>\<^sub>a OrL (x).M (y).N' z" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4473 | | a_OrR1: "\<lbrakk>a\<sharp>b; M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> OrR1 <a>.M b \<longrightarrow>\<^sub>a OrR1 <a>.M' b" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4474 | | a_OrR2: "\<lbrakk>a\<sharp>b; M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> OrR2 <a>.M b \<longrightarrow>\<^sub>a OrR2 <a>.M' b" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4475 | | a_ImpL_l: "\<lbrakk>a\<sharp>N; x\<sharp>(M,y); M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> ImpL <a>.M (x).N y \<longrightarrow>\<^sub>a ImpL <a>.M' (x).N y" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4476 | | a_ImpL_r: "\<lbrakk>a\<sharp>N; x\<sharp>(M,y); N\<longrightarrow>\<^sub>a N'\<rbrakk> \<Longrightarrow> ImpL <a>.M (x).N y \<longrightarrow>\<^sub>a ImpL <a>.M (x).N' y" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4477 | | a_ImpR: "\<lbrakk>a\<sharp>b; M\<longrightarrow>\<^sub>a M'\<rbrakk> \<Longrightarrow> ImpR (x).<a>.M b \<longrightarrow>\<^sub>a ImpR (x).<a>.M' b" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4478 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4479 | lemma fresh_a_redu: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4480 | fixes x::"name" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4481 | and c::"coname" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4482 | shows "M \<longrightarrow>\<^sub>a M' \<Longrightarrow> x\<sharp>M \<Longrightarrow> x\<sharp>M'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4483 | and "M \<longrightarrow>\<^sub>a M' \<Longrightarrow> c\<sharp>M \<Longrightarrow> c\<sharp>M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4484 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4485 | apply(induct rule: a_redu.induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4486 | apply(simp add: fresh_l_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4487 | apply(simp add: fresh_c_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4488 | apply(auto simp add: abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4489 | apply(induct rule: a_redu.induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4490 | apply(simp add: fresh_l_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4491 | apply(simp add: fresh_c_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4492 | apply(auto simp add: abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4493 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4494 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4495 | equivariance a_redu | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4496 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4497 | nominal_inductive a_redu | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4498 | by (simp_all add: abs_fresh fresh_atm fresh_prod abs_supp fin_supp fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4499 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4500 | lemma better_CutL_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4501 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>a Cut <a>.M' (x).N" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4502 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4503 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4504 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4505 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,a)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4506 | have "Cut <a>.M (x).N = Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4507 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4508 | also have "\<dots> \<longrightarrow>\<^sub>a Cut <a'>.([(a',a)]\<bullet>M') (x').([(x',x)]\<bullet>N)" using fs1 fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4509 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4510 | also have "\<dots> = Cut <a>.M' (x).N" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4511 | using fs1 fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4512 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4513 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4514 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4515 | lemma better_CutR_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4516 | shows "N\<longrightarrow>\<^sub>a N' \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>a Cut <a>.M (x).N'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4517 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4518 | assume red: "N\<longrightarrow>\<^sub>a N'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4519 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4520 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,a)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4521 | have "Cut <a>.M (x).N = Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N)" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4522 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4523 | also have "\<dots> \<longrightarrow>\<^sub>a Cut <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N')" using fs1 fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4524 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4525 | also have "\<dots> = Cut <a>.M (x).N'" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4526 | using fs1 fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4527 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4528 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4529 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4530 | lemma better_AndRL_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4531 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> AndR <a>.M <b>.N c \<longrightarrow>\<^sub>a AndR <a>.M' <b>.N c" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4532 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4533 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4534 | obtain b'::"coname" where fs1: "b'\<sharp>(M,N,a,b,c)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4535 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,a,b,c,b')" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4536 | have "AndR <a>.M <b>.N c = AndR <a'>.([(a',a)]\<bullet>M) <b'>.([(b',b)]\<bullet>N) c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4537 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4538 | also have "\<dots> \<longrightarrow>\<^sub>a AndR <a'>.([(a',a)]\<bullet>M') <b'>.([(b',b)]\<bullet>N) c" using fs1 fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4539 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4540 | also have "\<dots> = AndR <a>.M' <b>.N c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4541 | using fs1 fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4542 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4543 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4544 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4545 | lemma better_AndRR_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4546 | shows "N\<longrightarrow>\<^sub>a N' \<Longrightarrow> AndR <a>.M <b>.N c \<longrightarrow>\<^sub>a AndR <a>.M <b>.N' c" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4547 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4548 | assume red: "N\<longrightarrow>\<^sub>a N'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4549 | obtain b'::"coname" where fs1: "b'\<sharp>(M,N,a,b,c)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4550 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,a,b,c,b')" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4551 | have "AndR <a>.M <b>.N c = AndR <a'>.([(a',a)]\<bullet>M) <b'>.([(b',b)]\<bullet>N) c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4552 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4553 | also have "\<dots> \<longrightarrow>\<^sub>a AndR <a'>.([(a',a)]\<bullet>M) <b'>.([(b',b)]\<bullet>N') c" using fs1 fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4554 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4555 | also have "\<dots> = AndR <a>.M <b>.N' c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4556 | using fs1 fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4557 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4558 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4559 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4560 | lemma better_AndL1_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4561 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> AndL1 (x).M y \<longrightarrow>\<^sub>a AndL1 (x).M' y" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4562 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4563 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4564 | obtain x'::"name" where fs1: "x'\<sharp>(M,y,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4565 | have "AndL1 (x).M y = AndL1 (x').([(x',x)]\<bullet>M) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4566 | using fs1 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4567 | also have "\<dots> \<longrightarrow>\<^sub>a AndL1 (x').([(x',x)]\<bullet>M') y" using fs1 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4568 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4569 | also have "\<dots> = AndL1 (x).M' y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4570 | using fs1 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4571 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4572 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4573 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4574 | lemma better_AndL2_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4575 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> AndL2 (x).M y \<longrightarrow>\<^sub>a AndL2 (x).M' y" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4576 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4577 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4578 | obtain x'::"name" where fs1: "x'\<sharp>(M,y,x)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4579 | have "AndL2 (x).M y = AndL2 (x').([(x',x)]\<bullet>M) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4580 | using fs1 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4581 | also have "\<dots> \<longrightarrow>\<^sub>a AndL2 (x').([(x',x)]\<bullet>M') y" using fs1 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4582 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4583 | also have "\<dots> = AndL2 (x).M' y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4584 | using fs1 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4585 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4586 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4587 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4588 | lemma better_OrLL_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4589 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> OrL (x).M (y).N z \<longrightarrow>\<^sub>a OrL (x).M' (y).N z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4590 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4591 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4592 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,x,y,z)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4593 | obtain y'::"name" where fs2: "y'\<sharp>(M,N,x,y,z,x')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4594 | have "OrL (x).M (y).N z = OrL (x').([(x',x)]\<bullet>M) (y').([(y',y)]\<bullet>N) z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4595 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4596 | also have "\<dots> \<longrightarrow>\<^sub>a OrL (x').([(x',x)]\<bullet>M') (y').([(y',y)]\<bullet>N) z" using fs1 fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4597 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4598 | also have "\<dots> = OrL (x).M' (y).N z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4599 | using fs1 fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4600 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4601 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4602 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4603 | lemma better_OrLR_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4604 | shows "N\<longrightarrow>\<^sub>a N' \<Longrightarrow> OrL (x).M (y).N z \<longrightarrow>\<^sub>a OrL (x).M (y).N' z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4605 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4606 | assume red: "N\<longrightarrow>\<^sub>a N'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4607 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,x,y,z)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4608 | obtain y'::"name" where fs2: "y'\<sharp>(M,N,x,y,z,x')" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4609 | have "OrL (x).M (y).N z = OrL (x').([(x',x)]\<bullet>M) (y').([(y',y)]\<bullet>N) z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4610 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4611 | also have "\<dots> \<longrightarrow>\<^sub>a OrL (x').([(x',x)]\<bullet>M) (y').([(y',y)]\<bullet>N') z" using fs1 fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4612 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4613 | also have "\<dots> = OrL (x).M (y).N' z" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4614 | using fs1 fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4615 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4616 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4617 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4618 | lemma better_OrR1_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4619 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> OrR1 <a>.M b \<longrightarrow>\<^sub>a OrR1 <a>.M' b" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4620 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4621 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4622 | obtain a'::"coname" where fs1: "a'\<sharp>(M,b,a)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4623 | have "OrR1 <a>.M b = OrR1 <a'>.([(a',a)]\<bullet>M) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4624 | using fs1 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4625 | also have "\<dots> \<longrightarrow>\<^sub>a OrR1 <a'>.([(a',a)]\<bullet>M') b" using fs1 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4626 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4627 | also have "\<dots> = OrR1 <a>.M' b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4628 | using fs1 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4629 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4630 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4631 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4632 | lemma better_OrR2_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4633 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> OrR2 <a>.M b \<longrightarrow>\<^sub>a OrR2 <a>.M' b" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4634 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4635 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4636 | obtain a'::"coname" where fs1: "a'\<sharp>(M,b,a)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4637 | have "OrR2 <a>.M b = OrR2 <a'>.([(a',a)]\<bullet>M) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4638 | using fs1 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4639 | also have "\<dots> \<longrightarrow>\<^sub>a OrR2 <a'>.([(a',a)]\<bullet>M') b" using fs1 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4640 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4641 | also have "\<dots> = OrR2 <a>.M' b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4642 | using fs1 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4643 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4644 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4645 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4646 | lemma better_ImpLL_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4647 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> ImpL <a>.M (x).N y \<longrightarrow>\<^sub>a ImpL <a>.M' (x).N y" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4648 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4649 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4650 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,x,y)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4651 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,a)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4652 | have "ImpL <a>.M (x).N y = ImpL <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4653 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4654 | also have "\<dots> \<longrightarrow>\<^sub>a ImpL <a'>.([(a',a)]\<bullet>M') (x').([(x',x)]\<bullet>N) y" using fs1 fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4655 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4656 | also have "\<dots> = ImpL <a>.M' (x).N y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4657 | using fs1 fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4658 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4659 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4660 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4661 | lemma better_ImpLR_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4662 | shows "N\<longrightarrow>\<^sub>a N' \<Longrightarrow> ImpL <a>.M (x).N y \<longrightarrow>\<^sub>a ImpL <a>.M (x).N' y" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4663 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4664 | assume red: "N\<longrightarrow>\<^sub>a N'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4665 | obtain x'::"name" where fs1: "x'\<sharp>(M,N,x,y)" by (rule exists_fresh(1), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4666 | obtain a'::"coname" where fs2: "a'\<sharp>(M,N,a)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4667 | have "ImpL <a>.M (x).N y = ImpL <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N) y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4668 | using fs1 fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4669 | also have "\<dots> \<longrightarrow>\<^sub>a ImpL <a'>.([(a',a)]\<bullet>M) (x').([(x',x)]\<bullet>N') y" using fs1 fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4670 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4671 | also have "\<dots> = ImpL <a>.M (x).N' y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4672 | using fs1 fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4673 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4674 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4675 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4676 | lemma better_ImpR_intro[intro]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4677 | shows "M\<longrightarrow>\<^sub>a M' \<Longrightarrow> ImpR (x).<a>.M b \<longrightarrow>\<^sub>a ImpR (x).<a>.M' b" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4678 | proof - | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4679 | assume red: "M\<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4680 | obtain a'::"coname" where fs2: "a'\<sharp>(M,a,b)" by (rule exists_fresh(2), rule fin_supp, blast) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4681 | have "ImpR (x).<a>.M b = ImpR (x).<a'>.([(a',a)]\<bullet>M) b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4682 | using fs2 by (rule_tac sym, auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4683 | also have "\<dots> \<longrightarrow>\<^sub>a ImpR (x).<a'>.([(a',a)]\<bullet>M') b" using fs2 red | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4684 | by (auto intro: a_redu.intros simp add: fresh_left calc_atm a_redu.eqvt fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4685 | also have "\<dots> = ImpR (x).<a>.M' b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4686 | using fs2 red by (auto simp add: trm.inject alpha fresh_atm fresh_prod calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4687 | finally show ?thesis by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4688 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4689 | |
| 63167 | 4690 | text \<open>axioms do not reduce\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4691 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4692 | lemma ax_do_not_l_reduce: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4693 | shows "Ax x a \<longrightarrow>\<^sub>l M \<Longrightarrow> False" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4694 | by (erule_tac l_redu.cases) (simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4695 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4696 | lemma ax_do_not_c_reduce: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4697 | shows "Ax x a \<longrightarrow>\<^sub>c M \<Longrightarrow> False" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4698 | by (erule_tac c_redu.cases) (simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4699 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4700 | lemma ax_do_not_a_reduce: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4701 | shows "Ax x a \<longrightarrow>\<^sub>a M \<Longrightarrow> False" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4702 | apply(erule_tac a_redu.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4703 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4704 | apply(drule ax_do_not_l_reduce) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4705 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4706 | apply(drule ax_do_not_c_reduce) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4707 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4708 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4709 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4710 | lemma a_redu_NotL_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4711 | assumes a: "NotL <a>.M x \<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4712 | shows "\<exists>M'. R = NotL <a>.M' x \<and> M\<longrightarrow>\<^sub>aM'" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 4713 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4714 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4715 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4716 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4717 | apply(auto) | 
| 57492 
74bf65a1910a
Hypsubst preserves equality hypotheses
 Thomas Sewell <thomas.sewell@nicta.com.au> parents: 
56073diff
changeset | 4718 | apply(rotate_tac 2) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4719 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4720 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4721 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4722 | apply(auto simp add: alpha a_redu.eqvt) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4723 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4724 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4725 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4726 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4727 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4728 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4729 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4730 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4731 | lemma a_redu_NotR_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4732 | assumes a: "NotR (x).M a \<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4733 | shows "\<exists>M'. R = NotR (x).M' a \<and> M\<longrightarrow>\<^sub>aM'" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 4734 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4735 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4736 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4737 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4738 | apply(auto) | 
| 57492 
74bf65a1910a
Hypsubst preserves equality hypotheses
 Thomas Sewell <thomas.sewell@nicta.com.au> parents: 
56073diff
changeset | 4739 | apply(rotate_tac 2) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4740 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4741 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4742 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4743 | apply(auto simp add: alpha a_redu.eqvt) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4744 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4745 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4746 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4747 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4748 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4749 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4750 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4751 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4752 | lemma a_redu_AndR_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4753 | assumes a: "AndR <a>.M <b>.N c\<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4754 | shows "(\<exists>M'. R = AndR <a>.M' <b>.N c \<and> M\<longrightarrow>\<^sub>aM') \<or> (\<exists>N'. R = AndR <a>.M <b>.N' c \<and> N\<longrightarrow>\<^sub>aN')" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 4755 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4756 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4757 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4758 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4759 | apply(rotate_tac 6) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4760 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4761 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4762 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4763 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4764 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4765 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4766 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4767 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4768 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4769 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4770 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4771 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4772 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4773 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4774 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4775 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4776 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4777 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4778 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4779 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4780 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4781 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4782 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4783 | apply(rule_tac x="([(b,ba)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4784 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4785 | apply(rule_tac x="([(b,baa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4786 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4787 | apply(rule_tac x="([(b,ba)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4788 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4789 | apply(rule_tac x="([(b,baa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4790 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4791 | apply(rule_tac x="([(b,ba)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4792 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4793 | apply(rule_tac x="([(b,baa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4794 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4795 | apply(rule_tac x="([(b,ba)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4796 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4797 | apply(rule_tac x="([(b,baa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4798 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4799 | apply(rotate_tac 6) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4800 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4801 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4802 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4803 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4804 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4805 | apply(rule_tac x="([(a,aa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4806 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4807 | apply(rule_tac x="([(a,aa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4808 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4809 | apply(rule_tac x="([(a,aa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4810 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4811 | apply(rule_tac x="([(a,aa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4812 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4813 | apply(rule_tac x="([(a,aaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4814 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4815 | apply(rule_tac x="([(a,aaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4816 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4817 | apply(rule_tac x="([(a,aaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4818 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4819 | apply(rule_tac x="([(a,aaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4820 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4821 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4822 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4823 | apply(rule_tac x="([(b,ba)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4824 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4825 | apply(rule_tac x="([(b,ba)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4826 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4827 | apply(rule_tac x="([(b,ba)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4828 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4829 | apply(rule_tac x="([(b,ba)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4830 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4831 | apply(rule_tac x="([(b,baa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4832 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4833 | apply(rule_tac x="([(b,baa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4834 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4835 | apply(rule_tac x="([(b,baa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4836 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4837 | apply(rule_tac x="([(b,baa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4838 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4839 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4840 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4841 | lemma a_redu_AndL1_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4842 | assumes a: "AndL1 (x).M y \<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4843 | shows "\<exists>M'. R = AndL1 (x).M' y \<and> M\<longrightarrow>\<^sub>aM'" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 4844 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4845 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4846 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4847 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4848 | apply(auto) | 
| 57492 
74bf65a1910a
Hypsubst preserves equality hypotheses
 Thomas Sewell <thomas.sewell@nicta.com.au> parents: 
56073diff
changeset | 4849 | apply(rotate_tac 3) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4850 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4851 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4852 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4853 | apply(auto simp add: alpha a_redu.eqvt) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4854 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4855 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4856 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4857 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4858 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4859 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4860 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4861 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4862 | lemma a_redu_AndL2_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4863 | assumes a: "AndL2 (x).M y \<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4864 | shows "\<exists>M'. R = AndL2 (x).M' y \<and> M\<longrightarrow>\<^sub>aM'" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 4865 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4866 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4867 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4868 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4869 | apply(auto) | 
| 57492 
74bf65a1910a
Hypsubst preserves equality hypotheses
 Thomas Sewell <thomas.sewell@nicta.com.au> parents: 
56073diff
changeset | 4870 | apply(rotate_tac 3) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4871 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4872 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4873 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4874 | apply(auto simp add: alpha a_redu.eqvt) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4875 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4876 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4877 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4878 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4879 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4880 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4881 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4882 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4883 | lemma a_redu_OrL_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4884 | assumes a: "OrL (x).M (y).N z\<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4885 | shows "(\<exists>M'. R = OrL (x).M' (y).N z \<and> M\<longrightarrow>\<^sub>aM') \<or> (\<exists>N'. R = OrL (x).M (y).N' z \<and> N\<longrightarrow>\<^sub>aN')" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 4886 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4887 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4888 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4889 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4890 | apply(rotate_tac 6) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4891 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4892 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4893 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4894 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4895 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4896 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4897 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4898 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4899 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4900 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4901 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4902 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4903 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4904 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4905 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4906 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4907 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4908 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4909 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4910 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4911 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4912 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4913 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4914 | apply(rule_tac x="([(y,ya)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4915 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4916 | apply(rule_tac x="([(y,yaa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4917 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4918 | apply(rule_tac x="([(y,ya)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4919 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4920 | apply(rule_tac x="([(y,yaa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4921 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4922 | apply(rule_tac x="([(y,ya)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4923 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4924 | apply(rule_tac x="([(y,yaa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4925 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4926 | apply(rule_tac x="([(y,ya)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4927 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4928 | apply(rule_tac x="([(y,yaa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4929 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4930 | apply(rotate_tac 6) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4931 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4932 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4933 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4934 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4935 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4936 | apply(rule_tac x="([(x,xa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4937 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4938 | apply(rule_tac x="([(x,xa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4939 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4940 | apply(rule_tac x="([(x,xa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4941 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4942 | apply(rule_tac x="([(x,xa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4943 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4944 | apply(rule_tac x="([(x,xaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4945 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4946 | apply(rule_tac x="([(x,xaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4947 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4948 | apply(rule_tac x="([(x,xaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4949 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4950 | apply(rule_tac x="([(x,xaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4951 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4952 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4953 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4954 | apply(rule_tac x="([(y,ya)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4955 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4956 | apply(rule_tac x="([(y,ya)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4957 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4958 | apply(rule_tac x="([(y,ya)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4959 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4960 | apply(rule_tac x="([(y,ya)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4961 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4962 | apply(rule_tac x="([(y,yaa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4963 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4964 | apply(rule_tac x="([(y,yaa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4965 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4966 | apply(rule_tac x="([(y,yaa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4967 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4968 | apply(rule_tac x="([(y,yaa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4969 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4970 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4971 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4972 | lemma a_redu_OrR1_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4973 | assumes a: "OrR1 <a>.M b \<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4974 | shows "\<exists>M'. R = OrR1 <a>.M' b \<and> M\<longrightarrow>\<^sub>aM'" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 4975 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4976 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4977 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4978 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4979 | apply(auto) | 
| 57492 
74bf65a1910a
Hypsubst preserves equality hypotheses
 Thomas Sewell <thomas.sewell@nicta.com.au> parents: 
56073diff
changeset | 4980 | apply(rotate_tac 3) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4981 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4982 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4983 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4984 | apply(auto simp add: alpha a_redu.eqvt) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4985 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4986 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4987 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4988 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4989 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4990 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4991 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4992 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4993 | lemma a_redu_OrR2_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4994 | assumes a: "OrR2 <a>.M b \<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 4995 | shows "\<exists>M'. R = OrR2 <a>.M' b \<and> M\<longrightarrow>\<^sub>aM'" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 4996 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4997 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4998 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 4999 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5000 | apply(auto) | 
| 57492 
74bf65a1910a
Hypsubst preserves equality hypotheses
 Thomas Sewell <thomas.sewell@nicta.com.au> parents: 
56073diff
changeset | 5001 | apply(rotate_tac 3) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5002 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5003 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5004 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5005 | apply(auto simp add: alpha a_redu.eqvt) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5006 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5007 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5008 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5009 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5010 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5011 | apply(simp add: perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5012 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5013 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5014 | lemma a_redu_ImpL_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5015 | assumes a: "ImpL <a>.M (y).N z\<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5016 | shows "(\<exists>M'. R = ImpL <a>.M' (y).N z \<and> M\<longrightarrow>\<^sub>aM') \<or> (\<exists>N'. R = ImpL <a>.M (y).N' z \<and> N\<longrightarrow>\<^sub>aN')" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 5017 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5018 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5019 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5020 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5021 | apply(rotate_tac 5) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5022 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5023 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5024 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5025 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5026 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5027 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5028 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5029 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5030 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5031 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5032 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5033 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5034 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5035 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5036 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5037 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5038 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5039 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5040 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5041 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5042 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5043 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5044 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5045 | apply(rule_tac x="([(y,xa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5046 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5047 | apply(rule_tac x="([(y,xa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5048 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5049 | apply(rule_tac x="([(y,xa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5050 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5051 | apply(rule_tac x="([(y,xa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5052 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5053 | apply(rule_tac x="([(y,xa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5054 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5055 | apply(rule_tac x="([(y,xa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5056 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5057 | apply(rule_tac x="([(y,xa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5058 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5059 | apply(rule_tac x="([(y,xa)]\<bullet>N')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5060 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5061 | apply(rotate_tac 5) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5062 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5063 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5064 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5065 | apply(rule disjI1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5066 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5067 | apply(rule_tac x="([(a,aa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5068 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5069 | apply(rule_tac x="([(a,aa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5070 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5071 | apply(rule_tac x="([(a,aa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5072 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5073 | apply(rule_tac x="([(a,aa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5074 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5075 | apply(rule_tac x="([(a,aaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5076 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5077 | apply(rule_tac x="([(a,aaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5078 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5079 | apply(rule_tac x="([(a,aaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5080 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5081 | apply(rule_tac x="([(a,aaa)]\<bullet>M')" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5082 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5083 | apply(rule disjI2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5084 | apply(auto simp add: alpha a_redu.eqvt)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5085 | apply(rule_tac x="([(y,xa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5086 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5087 | apply(rule_tac x="([(y,xa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5088 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5089 | apply(rule_tac x="([(y,xa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5090 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5091 | apply(rule_tac x="([(y,xa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5092 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5093 | apply(rule_tac x="([(y,xa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5094 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5095 | apply(rule_tac x="([(y,xa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5096 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5097 | apply(rule_tac x="([(y,xa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5098 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5099 | apply(rule_tac x="([(y,xa)]\<bullet>N'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5100 | apply(auto simp add: perm_swap fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5101 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5102 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5103 | lemma a_redu_ImpR_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5104 | assumes a: "ImpR (x).<a>.M b \<longrightarrow>\<^sub>a R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5105 | shows "\<exists>M'. R = ImpR (x).<a>.M' b \<and> M\<longrightarrow>\<^sub>aM'" | 
| 71989 
bad75618fb82
extraction of equations x = t from premises beneath meta-all
 haftmann parents: 
67613diff
changeset | 5106 | using a [[simproc del: defined_all]] | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5107 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5108 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5109 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5110 | apply(auto) | 
| 57492 
74bf65a1910a
Hypsubst preserves equality hypotheses
 Thomas Sewell <thomas.sewell@nicta.com.au> parents: 
56073diff
changeset | 5111 | apply(rotate_tac 3) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5112 | apply(erule_tac a_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5113 | apply(erule_tac l_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5114 | apply(erule_tac c_redu.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5115 | apply(auto simp add: alpha a_redu.eqvt abs_perm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5116 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5117 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5118 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5119 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5120 | apply(rule_tac x="([(a,aa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5121 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5122 | apply(rule_tac x="([(a,aaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5123 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5124 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5125 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5126 | apply(rule_tac x="([(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5127 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5128 | apply(rule_tac x="([(a,aa)]\<bullet>[(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5129 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5130 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5131 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5132 | apply(rule perm_compose) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5133 | apply(simp add: calc_atm perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5134 | apply(rule_tac x="([(a,aaa)]\<bullet>[(x,xa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5135 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5136 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5137 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5138 | apply(rule perm_compose) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5139 | apply(simp add: calc_atm perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5140 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5141 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5142 | apply(rule_tac x="([(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5143 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5144 | apply(rule_tac x="([(a,aa)]\<bullet>[(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5145 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5146 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5147 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5148 | apply(rule perm_compose) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5149 | apply(simp add: calc_atm perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5150 | apply(rule_tac x="([(a,aaa)]\<bullet>[(x,xaa)]\<bullet>M'a)" in exI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5151 | apply(auto simp add: fresh_left alpha a_redu.eqvt calc_atm fresh_a_redu perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5152 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5153 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5154 | apply(rule perm_compose) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5155 | apply(simp add: calc_atm perm_swap) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5156 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5157 | |
| 63167 | 5158 | text \<open>Transitive Closure\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5159 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5160 | abbreviation | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5161 |  a_star_redu :: "trm \<Rightarrow> trm \<Rightarrow> bool" ("_ \<longrightarrow>\<^sub>a* _" [100,100] 100)
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5162 | where | 
| 67613 | 5163 | "M \<longrightarrow>\<^sub>a* M' \<equiv> (a_redu)\<^sup>*\<^sup>* M M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5164 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5165 | lemma a_starI: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5166 | assumes a: "M \<longrightarrow>\<^sub>a M'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5167 | shows "M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5168 | using a by blast | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5169 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5170 | lemma a_starE: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5171 | assumes a: "M \<longrightarrow>\<^sub>a* M'" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5172 | shows "M = M' \<or> (\<exists>N. M \<longrightarrow>\<^sub>a N \<and> N \<longrightarrow>\<^sub>a* M')" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5173 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5174 | by (induct) (auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5175 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5176 | lemma a_star_refl: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5177 | shows "M \<longrightarrow>\<^sub>a* M" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5178 | by blast | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5179 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5180 | lemma a_star_trans[trans]: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5181 | assumes a1: "M1\<longrightarrow>\<^sub>a* M2" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5182 | and a2: "M2\<longrightarrow>\<^sub>a* M3" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5183 | shows "M1 \<longrightarrow>\<^sub>a* M3" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5184 | using a2 a1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5185 | by (induct) (auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5186 | |
| 63167 | 5187 | text \<open>congruence rules for \<open>\<longrightarrow>\<^sub>a*\<close>\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5188 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5189 | lemma ax_do_not_a_star_reduce: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5190 | shows "Ax x a \<longrightarrow>\<^sub>a* M \<Longrightarrow> M = Ax x a" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5191 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5192 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5193 | apply(drule ax_do_not_a_reduce) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5194 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5195 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5196 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5197 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5198 | lemma a_star_CutL: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5199 | "M \<longrightarrow>\<^sub>a* M' \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>a* Cut <a>.M' (x).N" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5200 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5201 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5202 | lemma a_star_CutR: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5203 | "N \<longrightarrow>\<^sub>a* N'\<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>a* Cut <a>.M (x).N'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5204 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5205 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5206 | lemma a_star_Cut: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5207 | "\<lbrakk>M \<longrightarrow>\<^sub>a* M'; N \<longrightarrow>\<^sub>a* N'\<rbrakk> \<Longrightarrow> Cut <a>.M (x).N \<longrightarrow>\<^sub>a* Cut <a>.M' (x).N'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5208 | by (blast intro!: a_star_CutL a_star_CutR intro: rtranclp_trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5209 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5210 | lemma a_star_NotR: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5211 | "M \<longrightarrow>\<^sub>a* M' \<Longrightarrow> NotR (x).M a \<longrightarrow>\<^sub>a* NotR (x).M' a" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5212 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5213 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5214 | lemma a_star_NotL: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5215 | "M \<longrightarrow>\<^sub>a* M' \<Longrightarrow> NotL <a>.M x \<longrightarrow>\<^sub>a* NotL <a>.M' x" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5216 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5217 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5218 | lemma a_star_AndRL: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5219 | "M \<longrightarrow>\<^sub>a* M'\<Longrightarrow> AndR <a>.M <b>.N c \<longrightarrow>\<^sub>a* AndR <a>.M' <b>.N c" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5220 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5221 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5222 | lemma a_star_AndRR: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5223 | "N \<longrightarrow>\<^sub>a* N'\<Longrightarrow> AndR <a>.M <b>.N c \<longrightarrow>\<^sub>a* AndR <a>.M <b>.N' c" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5224 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5225 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5226 | lemma a_star_AndR: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5227 | "\<lbrakk>M \<longrightarrow>\<^sub>a* M'; N \<longrightarrow>\<^sub>a* N'\<rbrakk> \<Longrightarrow> AndR <a>.M <b>.N c \<longrightarrow>\<^sub>a* AndR <a>.M' <b>.N' c" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5228 | by (blast intro!: a_star_AndRL a_star_AndRR intro: rtranclp_trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5229 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5230 | lemma a_star_AndL1: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5231 | "M \<longrightarrow>\<^sub>a* M' \<Longrightarrow> AndL1 (x).M y \<longrightarrow>\<^sub>a* AndL1 (x).M' y" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5232 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5233 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5234 | lemma a_star_AndL2: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5235 | "M \<longrightarrow>\<^sub>a* M' \<Longrightarrow> AndL2 (x).M y \<longrightarrow>\<^sub>a* AndL2 (x).M' y" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5236 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5237 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5238 | lemma a_star_OrLL: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5239 | "M \<longrightarrow>\<^sub>a* M'\<Longrightarrow> OrL (x).M (y).N z \<longrightarrow>\<^sub>a* OrL (x).M' (y).N z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5240 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5241 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5242 | lemma a_star_OrLR: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5243 | "N \<longrightarrow>\<^sub>a* N'\<Longrightarrow> OrL (x).M (y).N z \<longrightarrow>\<^sub>a* OrL (x).M (y).N' z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5244 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5245 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5246 | lemma a_star_OrL: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5247 | "\<lbrakk>M \<longrightarrow>\<^sub>a* M'; N \<longrightarrow>\<^sub>a* N'\<rbrakk> \<Longrightarrow> OrL (x).M (y).N z \<longrightarrow>\<^sub>a* OrL (x).M' (y).N' z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5248 | by (blast intro!: a_star_OrLL a_star_OrLR intro: rtranclp_trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5249 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5250 | lemma a_star_OrR1: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5251 | "M \<longrightarrow>\<^sub>a* M' \<Longrightarrow> OrR1 <a>.M b \<longrightarrow>\<^sub>a* OrR1 <a>.M' b" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5252 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5253 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5254 | lemma a_star_OrR2: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5255 | "M \<longrightarrow>\<^sub>a* M' \<Longrightarrow> OrR2 <a>.M b \<longrightarrow>\<^sub>a* OrR2 <a>.M' b" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5256 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5257 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5258 | lemma a_star_ImpLL: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5259 | "M \<longrightarrow>\<^sub>a* M'\<Longrightarrow> ImpL <a>.M (y).N z \<longrightarrow>\<^sub>a* ImpL <a>.M' (y).N z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5260 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5261 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5262 | lemma a_star_ImpLR: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5263 | "N \<longrightarrow>\<^sub>a* N'\<Longrightarrow> ImpL <a>.M (y).N z \<longrightarrow>\<^sub>a* ImpL <a>.M (y).N' z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5264 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5265 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5266 | lemma a_star_ImpL: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5267 | "\<lbrakk>M \<longrightarrow>\<^sub>a* M'; N \<longrightarrow>\<^sub>a* N'\<rbrakk> \<Longrightarrow> ImpL <a>.M (y).N z \<longrightarrow>\<^sub>a* ImpL <a>.M' (y).N' z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5268 | by (blast intro!: a_star_ImpLL a_star_ImpLR intro: rtranclp_trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5269 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5270 | lemma a_star_ImpR: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5271 | "M \<longrightarrow>\<^sub>a* M' \<Longrightarrow> ImpR (x).<a>.M b \<longrightarrow>\<^sub>a* ImpR (x).<a>.M' b" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5272 | by (induct set: rtranclp) (blast intro: rtranclp.rtrancl_into_rtrancl)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5273 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5274 | lemmas a_star_congs = a_star_Cut a_star_NotR a_star_NotL a_star_AndR a_star_AndL1 a_star_AndL2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5275 | a_star_OrL a_star_OrR1 a_star_OrR2 a_star_ImpL a_star_ImpR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5276 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5277 | lemma a_star_redu_NotL_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5278 | assumes a: "NotL <a>.M x \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5279 | shows "\<exists>M'. R = NotL <a>.M' x \<and> M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5280 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5281 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5282 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5283 | apply(drule a_redu_NotL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5284 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5285 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5286 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5287 | lemma a_star_redu_NotR_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5288 | assumes a: "NotR (x).M a \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5289 | shows "\<exists>M'. R = NotR (x).M' a \<and> M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5290 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5291 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5292 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5293 | apply(drule a_redu_NotR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5294 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5295 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5296 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5297 | lemma a_star_redu_AndR_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5298 | assumes a: "AndR <a>.M <b>.N c\<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5299 | shows "(\<exists>M' N'. R = AndR <a>.M' <b>.N' c \<and> M \<longrightarrow>\<^sub>a* M' \<and> N \<longrightarrow>\<^sub>a* N')" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5300 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5301 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5302 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5303 | apply(drule a_redu_AndR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5304 | apply(auto simp add: alpha trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5305 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5306 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5307 | lemma a_star_redu_AndL1_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5308 | assumes a: "AndL1 (x).M y \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5309 | shows "\<exists>M'. R = AndL1 (x).M' y \<and> M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5310 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5311 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5312 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5313 | apply(drule a_redu_AndL1_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5314 | apply(auto simp add: alpha trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5315 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5316 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5317 | lemma a_star_redu_AndL2_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5318 | assumes a: "AndL2 (x).M y \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5319 | shows "\<exists>M'. R = AndL2 (x).M' y \<and> M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5320 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5321 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5322 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5323 | apply(drule a_redu_AndL2_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5324 | apply(auto simp add: alpha trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5325 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5326 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5327 | lemma a_star_redu_OrL_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5328 | assumes a: "OrL (x).M (y).N z \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5329 | shows "(\<exists>M' N'. R = OrL (x).M' (y).N' z \<and> M \<longrightarrow>\<^sub>a* M' \<and> N \<longrightarrow>\<^sub>a* N')" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5330 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5331 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5332 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5333 | apply(drule a_redu_OrL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5334 | apply(auto simp add: alpha trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5335 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5336 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5337 | lemma a_star_redu_OrR1_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5338 | assumes a: "OrR1 <a>.M y \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5339 | shows "\<exists>M'. R = OrR1 <a>.M' y \<and> M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5340 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5341 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5342 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5343 | apply(drule a_redu_OrR1_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5344 | apply(auto simp add: alpha trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5345 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5346 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5347 | lemma a_star_redu_OrR2_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5348 | assumes a: "OrR2 <a>.M y \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5349 | shows "\<exists>M'. R = OrR2 <a>.M' y \<and> M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5350 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5351 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5352 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5353 | apply(drule a_redu_OrR2_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5354 | apply(auto simp add: alpha trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5355 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5356 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5357 | lemma a_star_redu_ImpR_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5358 | assumes a: "ImpR (x).<a>.M y \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5359 | shows "\<exists>M'. R = ImpR (x).<a>.M' y \<and> M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5360 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5361 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5362 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5363 | apply(drule a_redu_ImpR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5364 | apply(auto simp add: alpha trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5365 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5366 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5367 | lemma a_star_redu_ImpL_elim: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5368 | assumes a: "ImpL <a>.M (y).N z \<longrightarrow>\<^sub>a* R" | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5369 | shows "(\<exists>M' N'. R = ImpL <a>.M' (y).N' z \<and> M \<longrightarrow>\<^sub>a* M' \<and> N \<longrightarrow>\<^sub>a* N')" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5370 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5371 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5372 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5373 | apply(drule a_redu_ImpL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5374 | apply(auto simp add: alpha trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5375 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5376 | |
| 63167 | 5377 | text \<open>Substitution\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5378 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5379 | lemma subst_not_fin1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5380 |   shows "\<not>fin(M{x:=<c>.P}) x"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5381 | apply(nominal_induct M avoiding: x c P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5382 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5383 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5384 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5385 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5386 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5387 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5388 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<c>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5389 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5390 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5391 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5392 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5393 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5394 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5395 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5396 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5397 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5398 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5399 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5400 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5401 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5402 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5403 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5404 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5405 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<c>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5406 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5407 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5408 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5409 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5410 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5411 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5412 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5413 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5414 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5415 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{x:=<c>.P},P,name1,trm2{x:=<c>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5416 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5417 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5418 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5419 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5420 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5421 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5422 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5423 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5424 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<c>.P},P,name1,trm2{name2:=<c>.P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5425 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5426 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5427 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5428 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5429 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5430 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5431 | apply(erule fin.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5432 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5433 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5434 | lemma subst_not_fin2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5435 | assumes a: "\<not>fin M y" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5436 |   shows "\<not>fin(M{c:=(x).P}) y" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5437 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5438 | apply(nominal_induct M avoiding: x c P y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5439 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5440 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5441 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5442 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5443 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5444 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5445 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5446 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5447 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5448 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5449 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5450 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5451 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5452 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5453 | apply(simp add: fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5454 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm1{coname3:=(x).P},P,coname1,trm2{coname3:=(x).P},coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5455 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5456 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5457 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5458 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5459 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5460 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5461 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5462 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5463 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5464 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5465 | apply(simp add: fin.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5466 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5467 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5468 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5469 | apply(simp add: fin.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5470 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5471 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5472 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5473 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5474 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5475 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5476 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5477 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5478 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5479 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5480 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5481 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5482 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5483 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5484 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5485 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5486 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5487 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5488 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5489 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5490 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5491 | apply(simp add: fin.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5492 | apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(trm{coname2:=(x).P},P,coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5493 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5494 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5495 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5496 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5497 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5498 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5499 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5500 | apply(drule fin_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5501 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5502 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5503 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5504 | apply(drule freshn_after_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5505 | apply(simp add: fin.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5506 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5507 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5508 | lemma subst_not_fic1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5509 |   shows "\<not>fic (M{a:=(x).P}) a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5510 | apply(nominal_induct M avoiding: a x P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5511 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5512 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5513 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5514 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5515 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5516 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm{coname:=(x).P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5517 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5518 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5519 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5520 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5521 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5522 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5523 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5524 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5525 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm1{coname3:=(x).P},P,trm2{coname3:=(x).P},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5526 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5527 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5528 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5529 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5530 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5531 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5532 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5533 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5534 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5535 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5536 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5537 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5538 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5539 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5540 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5541 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5542 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5543 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5544 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5545 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5546 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5547 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5548 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5549 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5550 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5551 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5552 | apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(trm{coname2:=(x).P},P,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5553 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5554 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5555 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5556 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5557 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5558 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5559 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5560 | apply(erule fic.cases, simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5561 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5562 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5563 | lemma subst_not_fic2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5564 | assumes a: "\<not>fic M a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5565 |   shows "\<not>fic(M{x:=<b>.P}) a" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5566 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5567 | apply(nominal_induct M avoiding: x a P b rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5568 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5569 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5570 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5571 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5572 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5573 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5574 | apply(simp add: fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5575 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.P},P)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5576 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5577 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5578 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5579 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5580 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5581 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5582 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5583 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5584 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5585 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5586 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5587 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5588 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5589 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5590 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5591 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5592 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5593 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5594 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5595 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5596 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5597 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5598 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5599 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5600 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5601 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5602 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5603 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5604 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5605 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5606 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5607 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5608 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5609 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5610 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5611 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5612 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5613 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{x:=<b>.P},P,name1,trm2{x:=<b>.P},name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5614 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5615 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5616 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5617 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5618 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5619 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5620 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5621 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5622 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5623 | apply(drule freshc_after_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5624 | apply(simp add: fic.intros abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5625 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<b>.P},trm2{name2:=<b>.P},P,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5626 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5627 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5628 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5629 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5630 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5631 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5632 | apply(drule fic_elims, simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5633 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5634 | |
| 63167 | 5635 | text \<open>Reductions\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5636 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5637 | lemma fin_l_reduce: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5638 | assumes a: "fin M x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5639 | and b: "M \<longrightarrow>\<^sub>l M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5640 | shows "fin M' x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5641 | using b a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5642 | apply(induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5643 | apply(erule fin.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5644 | apply(simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5645 | apply(rotate_tac 3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5646 | apply(erule fin.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5647 | apply(simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5648 | apply(erule fin.cases, simp_all add: trm.inject)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5649 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5650 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5651 | lemma fin_c_reduce: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5652 | assumes a: "fin M x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5653 | and b: "M \<longrightarrow>\<^sub>c M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5654 | shows "fin M' x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5655 | using b a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5656 | apply(induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5657 | apply(erule fin.cases, simp_all add: trm.inject)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5658 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5659 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5660 | lemma fin_a_reduce: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5661 | assumes a: "fin M x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5662 | and b: "M \<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5663 | shows "fin M' x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5664 | using a b | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5665 | apply(induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5666 | apply(drule ax_do_not_a_reduce) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5667 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5668 | apply(drule a_redu_NotL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5669 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5670 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5671 | apply(simp add: fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5672 | apply(drule a_redu_AndL1_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5673 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5674 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5675 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5676 | apply(drule a_redu_AndL2_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5677 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5678 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5679 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5680 | apply(drule a_redu_OrL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5681 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5682 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5683 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5684 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5685 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5686 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5687 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5688 | apply(drule a_redu_ImpL_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5689 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5690 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5691 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5692 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5693 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5694 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5695 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5696 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5697 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5698 | lemma fin_a_star_reduce: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5699 | assumes a: "fin M x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5700 | and b: "M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5701 | shows "fin M' x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5702 | using b a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5703 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5704 | apply(auto simp add: fin_a_reduce) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5705 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5706 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5707 | lemma fic_l_reduce: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5708 | assumes a: "fic M x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5709 | and b: "M \<longrightarrow>\<^sub>l M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5710 | shows "fic M' x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5711 | using b a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5712 | apply(induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5713 | apply(erule fic.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5714 | apply(simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5715 | apply(rotate_tac 3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5716 | apply(erule fic.cases) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5717 | apply(simp_all add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5718 | apply(erule fic.cases, simp_all add: trm.inject)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5719 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5720 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5721 | lemma fic_c_reduce: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5722 | assumes a: "fic M x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5723 | and b: "M \<longrightarrow>\<^sub>c M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5724 | shows "fic M' x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5725 | using b a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5726 | apply(induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5727 | apply(erule fic.cases, simp_all add: trm.inject)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5728 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5729 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5730 | lemma fic_a_reduce: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5731 | assumes a: "fic M x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5732 | and b: "M \<longrightarrow>\<^sub>a M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5733 | shows "fic M' x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5734 | using a b | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5735 | apply(induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5736 | apply(drule ax_do_not_a_reduce) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5737 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5738 | apply(drule a_redu_NotR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5739 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5740 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5741 | apply(simp add: fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5742 | apply(drule a_redu_AndR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5743 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5744 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5745 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5746 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5747 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5748 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5749 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5750 | apply(drule a_redu_OrR1_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5751 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5752 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5753 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5754 | apply(drule a_redu_OrR2_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5755 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5756 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5757 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5758 | apply(drule a_redu_ImpR_elim) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5759 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5760 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5761 | apply(force simp add: abs_fresh fresh_a_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5762 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5763 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5764 | lemma fic_a_star_reduce: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5765 | assumes a: "fic M x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5766 | and b: "M \<longrightarrow>\<^sub>a* M'" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5767 | shows "fic M' x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5768 | using b a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5769 | apply(induct set: rtranclp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5770 | apply(auto simp add: fic_a_reduce) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5771 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5772 | |
| 63167 | 5773 | text \<open>substitution properties\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5774 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5775 | lemma subst_with_ax1: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5776 |   shows "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5777 | proof(nominal_induct M avoiding: x a y rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5778 | case (Ax z b x a y) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5779 |   show "(Ax z b){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (Ax z b)[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5780 | proof (cases "z=x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5781 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5782 | assume eq: "z=x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5783 |     have "(Ax z b){x:=<a>.Ax y a} = Cut <a>.Ax y a (x).Ax x b" using eq by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5784 | also have "\<dots> \<longrightarrow>\<^sub>a* (Ax x b)[x\<turnstile>n>y]" by blast | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5785 |     finally show "Ax z b{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (Ax z b)[x\<turnstile>n>y]" using eq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5786 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5787 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5788 | assume neq: "z\<noteq>x" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5789 |     then show "(Ax z b){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (Ax z b)[x\<turnstile>n>y]" using neq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5790 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5791 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5792 | case (Cut b M z N x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5793 | have fs: "b\<sharp>x" "b\<sharp>a" "b\<sharp>y" "b\<sharp>N" "z\<sharp>x" "z\<sharp>a" "z\<sharp>y" "z\<sharp>M" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5794 |   have ih1: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5795 |   have ih2: "N{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* N[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5796 |   show "(Cut <b>.M (z).N){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (Cut <b>.M (z).N)[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5797 | proof (cases "M = Ax x b") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5798 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5799 | assume eq: "M = Ax x b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5800 |     have "(Cut <b>.M (z).N){x:=<a>.Ax y a} = Cut <a>.Ax y a (z).(N{x:=<a>.Ax y a})" using fs eq by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5801 | also have "\<dots> \<longrightarrow>\<^sub>a* Cut <a>.Ax y a (z).(N[x\<turnstile>n>y])" using ih2 a_star_congs by blast | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5802 | also have "\<dots> = Cut <b>.(M[x\<turnstile>n>y]) (z).(N[x\<turnstile>n>y])" using eq | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5803 | by (simp add: trm.inject alpha calc_atm fresh_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5804 |     finally show "(Cut <b>.M (z).N){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (Cut <b>.M (z).N)[x\<turnstile>n>y]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5805 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5806 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5807 | assume neq: "M \<noteq> Ax x b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5808 |     have "(Cut <b>.M (z).N){x:=<a>.Ax y a} = Cut <b>.(M{x:=<a>.Ax y a}) (z).(N{x:=<a>.Ax y a})" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5809 | using fs neq by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5810 | also have "\<dots> \<longrightarrow>\<^sub>a* Cut <b>.(M[x\<turnstile>n>y]) (z).(N[x\<turnstile>n>y])" using ih1 ih2 a_star_congs by blast | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5811 |     finally show "(Cut <b>.M (z).N){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (Cut <b>.M (z).N)[x\<turnstile>n>y]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5812 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5813 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5814 | case (NotR z M b x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5815 | have fs: "z\<sharp>x" "z\<sharp>a" "z\<sharp>y" "z\<sharp>b" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5816 |   have ih: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5817 |   have "(NotR (z).M b){x:=<a>.Ax y a} = NotR (z).(M{x:=<a>.Ax y a}) b" using fs by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5818 | also have "\<dots> \<longrightarrow>\<^sub>a* NotR (z).(M[x\<turnstile>n>y]) b" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5819 |   finally show "(NotR (z).M b){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (NotR (z).M b)[x\<turnstile>n>y]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5820 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5821 | case (NotL b M z x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5822 | have fs: "b\<sharp>x" "b\<sharp>a" "b\<sharp>y" "b\<sharp>z" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5823 |   have ih: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5824 |   show "(NotL <b>.M z){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (NotL <b>.M z)[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5825 | proof(cases "z=x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5826 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5827 | assume eq: "z=x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5828 |     obtain x'::"name" where new: "x'\<sharp>(Ax y a,M{x:=<a>.Ax y a})" by (rule exists_fresh(1)[OF fs_name1])
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5829 |     have "(NotL <b>.M z){x:=<a>.Ax y a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5830 |                         fresh_fun (\<lambda>x'. Cut <a>.Ax y a (x').NotL <b>.(M{x:=<a>.Ax y a}) x')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5831 | using eq fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5832 |     also have "\<dots> = Cut <a>.Ax y a (x').NotL <b>.(M{x:=<a>.Ax y a}) x'" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5833 | using new by (simp add: fresh_fun_simp_NotL fresh_prod) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5834 |     also have "\<dots> \<longrightarrow>\<^sub>a* (NotL <b>.(M{x:=<a>.Ax y a}) x')[x'\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5835 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5836 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5837 | apply(rule al_redu) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5838 | apply(rule better_LAxL_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5839 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5840 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5841 |     also have "\<dots> = NotL <b>.(M{x:=<a>.Ax y a}) y" using new by (simp add: nrename_fresh)
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5842 | also have "\<dots> \<longrightarrow>\<^sub>a* NotL <b>.(M[x\<turnstile>n>y]) y" using ih by (auto intro: a_star_congs) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5843 | also have "\<dots> = (NotL <b>.M z)[x\<turnstile>n>y]" using eq by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5844 |     finally show "(NotL <b>.M z){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (NotL <b>.M z)[x\<turnstile>n>y]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5845 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5846 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5847 | assume neq: "z\<noteq>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5848 |     have "(NotL <b>.M z){x:=<a>.Ax y a} = NotL <b>.(M{x:=<a>.Ax y a}) z" using fs neq by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5849 | also have "\<dots> \<longrightarrow>\<^sub>a* NotL <b>.(M[x\<turnstile>n>y]) z" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5850 |     finally show "(NotL <b>.M z){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (NotL <b>.M z)[x\<turnstile>n>y]" using neq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5851 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5852 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5853 | case (AndR c M d N e x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5854 | have fs: "c\<sharp>x" "c\<sharp>a" "c\<sharp>y" "d\<sharp>x" "d\<sharp>a" "d\<sharp>y" "d\<noteq>c" "c\<sharp>N" "c\<sharp>e" "d\<sharp>M" "d\<sharp>e" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5855 |   have ih1: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5856 |   have ih2: "N{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* N[x\<turnstile>n>y]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5857 |   have "(AndR <c>.M <d>.N e){x:=<a>.Ax y a} = AndR <c>.(M{x:=<a>.Ax y a}) <d>.(N{x:=<a>.Ax y a}) e"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5858 | using fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5859 | also have "\<dots> \<longrightarrow>\<^sub>a* AndR <c>.(M[x\<turnstile>n>y]) <d>.(N[x\<turnstile>n>y]) e" using ih1 ih2 by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5860 |   finally show "(AndR <c>.M <d>.N e){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (AndR <c>.M <d>.N e)[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5861 | using fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5862 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5863 | case (AndL1 u M v x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5864 | have fs: "u\<sharp>x" "u\<sharp>a" "u\<sharp>y" "u\<sharp>v" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5865 |   have ih: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5866 |   show "(AndL1 (u).M v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (AndL1 (u).M v)[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5867 | proof(cases "v=x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5868 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5869 | assume eq: "v=x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5870 |     obtain v'::"name" where new: "v'\<sharp>(Ax y a,M{x:=<a>.Ax y a},u)" by (rule exists_fresh(1)[OF fs_name1])
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5871 |     have "(AndL1 (u).M v){x:=<a>.Ax y a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5872 |                         fresh_fun (\<lambda>v'. Cut <a>.Ax y a (v').AndL1 (u).(M{x:=<a>.Ax y a}) v')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5873 | using eq fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5874 |     also have "\<dots> = Cut <a>.Ax y a (v').AndL1 (u).(M{x:=<a>.Ax y a}) v'" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5875 | using new by (simp add: fresh_fun_simp_AndL1 fresh_prod) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5876 |     also have "\<dots> \<longrightarrow>\<^sub>a* (AndL1 (u).(M{x:=<a>.Ax y a}) v')[v'\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5877 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5878 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5879 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5880 | apply(rule better_LAxL_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5881 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5882 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5883 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5884 |     also have "\<dots> = AndL1 (u).(M{x:=<a>.Ax y a}) y" using fs new
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5885 | by (auto simp add: fresh_prod fresh_atm nrename_fresh) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5886 | also have "\<dots> \<longrightarrow>\<^sub>a* AndL1 (u).(M[x\<turnstile>n>y]) y" using ih by (auto intro: a_star_congs) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5887 | also have "\<dots> = (AndL1 (u).M v)[x\<turnstile>n>y]" using eq fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5888 |     finally show "(AndL1 (u).M v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (AndL1 (u).M v)[x\<turnstile>n>y]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5889 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5890 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5891 | assume neq: "v\<noteq>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5892 |     have "(AndL1 (u).M v){x:=<a>.Ax y a} = AndL1 (u).(M{x:=<a>.Ax y a}) v" using fs neq by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5893 | also have "\<dots> \<longrightarrow>\<^sub>a* AndL1 (u).(M[x\<turnstile>n>y]) v" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5894 |     finally show "(AndL1 (u).M v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (AndL1 (u).M v)[x\<turnstile>n>y]" using fs neq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5895 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5896 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5897 | case (AndL2 u M v x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5898 | have fs: "u\<sharp>x" "u\<sharp>a" "u\<sharp>y" "u\<sharp>v" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5899 |   have ih: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5900 |   show "(AndL2 (u).M v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (AndL2 (u).M v)[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5901 | proof(cases "v=x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5902 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5903 | assume eq: "v=x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5904 |     obtain v'::"name" where new: "v'\<sharp>(Ax y a,M{x:=<a>.Ax y a},u)" by (rule exists_fresh(1)[OF fs_name1])
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5905 |     have "(AndL2 (u).M v){x:=<a>.Ax y a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5906 |                         fresh_fun (\<lambda>v'. Cut <a>.Ax y a (v').AndL2 (u).(M{x:=<a>.Ax y a}) v')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5907 | using eq fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5908 |     also have "\<dots> = Cut <a>.Ax y a (v').AndL2 (u).(M{x:=<a>.Ax y a}) v'" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5909 | using new by (simp add: fresh_fun_simp_AndL2 fresh_prod) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5910 |     also have "\<dots> \<longrightarrow>\<^sub>a* (AndL2 (u).(M{x:=<a>.Ax y a}) v')[v'\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5911 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5912 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5913 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5914 | apply(rule better_LAxL_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5915 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5916 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5917 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5918 |     also have "\<dots> = AndL2 (u).(M{x:=<a>.Ax y a}) y" using fs new
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5919 | by (auto simp add: fresh_prod fresh_atm nrename_fresh) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5920 | also have "\<dots> \<longrightarrow>\<^sub>a* AndL2 (u).(M[x\<turnstile>n>y]) y" using ih by (auto intro: a_star_congs) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5921 | also have "\<dots> = (AndL2 (u).M v)[x\<turnstile>n>y]" using eq fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5922 |     finally show "(AndL2 (u).M v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (AndL2 (u).M v)[x\<turnstile>n>y]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5923 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5924 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5925 | assume neq: "v\<noteq>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5926 |     have "(AndL2 (u).M v){x:=<a>.Ax y a} = AndL2 (u).(M{x:=<a>.Ax y a}) v" using fs neq by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5927 | also have "\<dots> \<longrightarrow>\<^sub>a* AndL2 (u).(M[x\<turnstile>n>y]) v" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5928 |     finally show "(AndL2 (u).M v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (AndL2 (u).M v)[x\<turnstile>n>y]" using fs neq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5929 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5930 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5931 | case (OrR1 c M d x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5932 | have fs: "c\<sharp>x" "c\<sharp>a" "c\<sharp>y" "c\<sharp>d" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5933 |   have ih: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5934 |   have "(OrR1 <c>.M d){x:=<a>.Ax y a} = OrR1 <c>.(M{x:=<a>.Ax y a}) d" using fs by (simp add: fresh_atm)
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5935 | also have "\<dots> \<longrightarrow>\<^sub>a* OrR1 <c>.(M[x\<turnstile>n>y]) d" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5936 |   finally show "(OrR1 <c>.M d){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (OrR1 <c>.M d)[x\<turnstile>n>y]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5937 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5938 | case (OrR2 c M d x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5939 | have fs: "c\<sharp>x" "c\<sharp>a" "c\<sharp>y" "c\<sharp>d" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5940 |   have ih: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5941 |   have "(OrR2 <c>.M d){x:=<a>.Ax y a} = OrR2 <c>.(M{x:=<a>.Ax y a}) d" using fs by (simp add: fresh_atm)
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5942 | also have "\<dots> \<longrightarrow>\<^sub>a* OrR2 <c>.(M[x\<turnstile>n>y]) d" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5943 |   finally show "(OrR2 <c>.M d){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (OrR2 <c>.M d)[x\<turnstile>n>y]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5944 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5945 | case (OrL u M v N z x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5946 | have fs: "u\<sharp>x" "u\<sharp>a" "u\<sharp>y" "v\<sharp>x" "v\<sharp>a" "v\<sharp>y" "v\<noteq>u" "u\<sharp>N" "u\<sharp>z" "v\<sharp>M" "v\<sharp>z" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5947 |   have ih1: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5948 |   have ih2: "N{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* N[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5949 |   show "(OrL (u).M (v).N z){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (OrL (u).M (v).N z)[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5950 | proof(cases "z=x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5951 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5952 | assume eq: "z=x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5953 |     obtain z'::"name" where new: "z'\<sharp>(Ax y a,M{x:=<a>.Ax y a},N{x:=<a>.Ax y a},u,v,y,a)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5954 | by (rule exists_fresh(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5955 |     have "(OrL (u).M (v).N z){x:=<a>.Ax y a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5956 |                  fresh_fun (\<lambda>z'. Cut <a>.Ax y a (z').OrL (u).(M{x:=<a>.Ax y a}) (v).(N{x:=<a>.Ax y a}) z')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5957 | using eq fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5958 |     also have "\<dots> = Cut <a>.Ax y a (z').OrL (u).(M{x:=<a>.Ax y a}) (v).(N{x:=<a>.Ax y a}) z'" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5959 | using new by (simp add: fresh_fun_simp_OrL) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5960 |     also have "\<dots> \<longrightarrow>\<^sub>a* (OrL (u).(M{x:=<a>.Ax y a}) (v).(N{x:=<a>.Ax y a}) z')[z'\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5961 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5962 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5963 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5964 | apply(rule better_LAxL_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5965 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5966 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5967 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5968 |     also have "\<dots> = OrL (u).(M{x:=<a>.Ax y a}) (v).(N{x:=<a>.Ax y a}) y" using fs new
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5969 | by (auto simp add: fresh_prod fresh_atm nrename_fresh subst_fresh) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5970 | also have "\<dots> \<longrightarrow>\<^sub>a* OrL (u).(M[x\<turnstile>n>y]) (v).(N[x\<turnstile>n>y]) y" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5971 | using ih1 ih2 by (auto intro: a_star_congs) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5972 | also have "\<dots> = (OrL (u).M (v).N z)[x\<turnstile>n>y]" using eq fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5973 |     finally show "(OrL (u).M (v).N z){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (OrL (u).M (v).N z)[x\<turnstile>n>y]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5974 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5975 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5976 | assume neq: "z\<noteq>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5977 |     have "(OrL (u).M (v).N z){x:=<a>.Ax y a} = OrL (u).(M{x:=<a>.Ax y a}) (v).(N{x:=<a>.Ax y a}) z" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5978 | using fs neq by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5979 | also have "\<dots> \<longrightarrow>\<^sub>a* OrL (u).(M[x\<turnstile>n>y]) (v).(N[x\<turnstile>n>y]) z" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5980 | using ih1 ih2 by (auto intro: a_star_congs) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5981 |     finally show "(OrL (u).M (v).N z){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (OrL (u).M (v).N z)[x\<turnstile>n>y]" using fs neq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5982 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5983 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5984 | case (ImpR z c M d x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5985 | have fs: "z\<sharp>x" "z\<sharp>a" "z\<sharp>y" "c\<sharp>x" "c\<sharp>a" "c\<sharp>y" "z\<sharp>d" "c\<sharp>d" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5986 |   have ih: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5987 |   have "(ImpR (z).<c>.M d){x:=<a>.Ax y a} = ImpR (z).<c>.(M{x:=<a>.Ax y a}) d" using fs by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5988 | also have "\<dots> \<longrightarrow>\<^sub>a* ImpR (z).<c>.(M[x\<turnstile>n>y]) d" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5989 |   finally show "(ImpR (z).<c>.M d){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (ImpR (z).<c>.M d)[x\<turnstile>n>y]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5990 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5991 | case (ImpL c M u N v x a y) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5992 | have fs: "c\<sharp>x" "c\<sharp>a" "c\<sharp>y" "u\<sharp>x" "u\<sharp>a" "u\<sharp>y" "c\<sharp>N" "c\<sharp>v" "u\<sharp>M" "u\<sharp>v" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5993 |   have ih1: "M{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* M[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5994 |   have ih2: "N{x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* N[x\<turnstile>n>y]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 5995 |   show "(ImpL <c>.M (u).N v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (ImpL <c>.M (u).N v)[x\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5996 | proof(cases "v=x") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5997 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5998 | assume eq: "v=x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 5999 |     obtain v'::"name" where new: "v'\<sharp>(Ax y a,M{x:=<a>.Ax y a},N{x:=<a>.Ax y a},y,a,u)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6000 | by (rule exists_fresh(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6001 |     have "(ImpL <c>.M (u).N v){x:=<a>.Ax y a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6002 |                  fresh_fun (\<lambda>v'. Cut <a>.Ax y a (v').ImpL <c>.(M{x:=<a>.Ax y a}) (u).(N{x:=<a>.Ax y a}) v')"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6003 | using eq fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6004 |     also have "\<dots> = Cut <a>.Ax y a (v').ImpL <c>.(M{x:=<a>.Ax y a}) (u).(N{x:=<a>.Ax y a}) v'" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6005 | using new by (simp add: fresh_fun_simp_ImpL) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6006 |     also have "\<dots> \<longrightarrow>\<^sub>a* (ImpL <c>.(M{x:=<a>.Ax y a}) (u).(N{x:=<a>.Ax y a}) v')[v'\<turnstile>n>y]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6007 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6008 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6009 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6010 | apply(rule better_LAxL_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6011 | apply(rule fin.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6012 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6013 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6014 |     also have "\<dots> = ImpL <c>.(M{x:=<a>.Ax y a}) (u).(N{x:=<a>.Ax y a}) y" using fs new
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6015 | by (auto simp add: fresh_prod subst_fresh fresh_atm trm.inject alpha rename_fresh) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6016 | also have "\<dots> \<longrightarrow>\<^sub>a* ImpL <c>.(M[x\<turnstile>n>y]) (u).(N[x\<turnstile>n>y]) y" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6017 | using ih1 ih2 by (auto intro: a_star_congs) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6018 | also have "\<dots> = (ImpL <c>.M (u).N v)[x\<turnstile>n>y]" using eq fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6019 |     finally show "(ImpL <c>.M (u).N v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (ImpL <c>.M (u).N v)[x\<turnstile>n>y]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6020 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6021 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6022 | assume neq: "v\<noteq>x" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6023 |     have "(ImpL <c>.M (u).N v){x:=<a>.Ax y a} = ImpL <c>.(M{x:=<a>.Ax y a}) (u).(N{x:=<a>.Ax y a}) v" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6024 | using fs neq by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6025 | also have "\<dots> \<longrightarrow>\<^sub>a* ImpL <c>.(M[x\<turnstile>n>y]) (u).(N[x\<turnstile>n>y]) v" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6026 | using ih1 ih2 by (auto intro: a_star_congs) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6027 |     finally show "(ImpL <c>.M (u).N v){x:=<a>.Ax y a} \<longrightarrow>\<^sub>a* (ImpL <c>.M (u).N v)[x\<turnstile>n>y]" 
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6028 | using fs neq by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6029 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6030 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6031 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6032 | lemma subst_with_ax2: | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6033 |   shows "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6034 | proof(nominal_induct M avoiding: b a x rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6035 | case (Ax z c b a x) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6036 |   show "(Ax z c){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (Ax z c)[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6037 | proof (cases "c=b") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6038 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6039 | assume eq: "c=b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6040 |     have "(Ax z c){b:=(x).Ax x a} = Cut <b>.Ax z c (x).Ax x a" using eq by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6041 | also have "\<dots> \<longrightarrow>\<^sub>a* (Ax z c)[b\<turnstile>c>a]" using eq by blast | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6042 |     finally show "(Ax z c){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (Ax z c)[b\<turnstile>c>a]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6043 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6044 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6045 | assume neq: "c\<noteq>b" | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6046 |     then show "(Ax z c){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (Ax z c)[b\<turnstile>c>a]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6047 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6048 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6049 | case (Cut c M z N b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6050 | have fs: "c\<sharp>b" "c\<sharp>a" "c\<sharp>x" "c\<sharp>N" "z\<sharp>b" "z\<sharp>a" "z\<sharp>x" "z\<sharp>M" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6051 |   have ih1: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6052 |   have ih2: "N{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* N[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6053 |   show "(Cut <c>.M (z).N){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (Cut <c>.M (z).N)[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6054 | proof (cases "N = Ax z b") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6055 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6056 | assume eq: "N = Ax z b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6057 |     have "(Cut <c>.M (z).N){b:=(x).Ax x a} = Cut <c>.(M{b:=(x).Ax x a}) (x).Ax x a" using eq fs by simp 
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6058 | also have "\<dots> \<longrightarrow>\<^sub>a* Cut <c>.(M[b\<turnstile>c>a]) (x).Ax x a" using ih1 a_star_congs by blast | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6059 | also have "\<dots> = Cut <c>.(M[b\<turnstile>c>a]) (z).(N[b\<turnstile>c>a])" using eq fs | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6060 | by (simp add: trm.inject alpha calc_atm fresh_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6061 |     finally show "(Cut <c>.M (z).N){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (Cut <c>.M (z).N)[b\<turnstile>c>a]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6062 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6063 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6064 | assume neq: "N \<noteq> Ax z b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6065 |     have "(Cut <c>.M (z).N){b:=(x).Ax x a} = Cut <c>.(M{b:=(x).Ax x a}) (z).(N{b:=(x).Ax x a})" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6066 | using fs neq by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6067 | also have "\<dots> \<longrightarrow>\<^sub>a* Cut <c>.(M[b\<turnstile>c>a]) (z).(N[b\<turnstile>c>a])" using ih1 ih2 a_star_congs by blast | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6068 |     finally show "(Cut <c>.M (z).N){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (Cut <c>.M (z).N)[b\<turnstile>c>a]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6069 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6070 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6071 | case (NotR z M c b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6072 | have fs: "z\<sharp>b" "z\<sharp>a" "z\<sharp>x" "z\<sharp>c" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6073 |   have ih: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6074 |   show "(NotR (z).M c){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (NotR (z).M c)[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6075 | proof (cases "c=b") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6076 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6077 | assume eq: "c=b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6078 |     obtain a'::"coname" where new: "a'\<sharp>(Ax x a,M{b:=(x).Ax x a})" by (rule exists_fresh(2)[OF fs_coname1])
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6079 |     have "(NotR (z).M c){b:=(x).Ax x a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6080 |                         fresh_fun (\<lambda>a'. Cut <a'>.NotR (z).M{b:=(x).Ax x a} a' (x).Ax x a)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6081 | using eq fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6082 |     also have "\<dots> = Cut <a'>.NotR (z).M{b:=(x).Ax x a} a' (x).Ax x a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6083 | using new by (simp add: fresh_fun_simp_NotR fresh_prod) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6084 |     also have "\<dots> \<longrightarrow>\<^sub>a* (NotR (z).(M{b:=(x).Ax x a}) a')[a'\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6085 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6086 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6087 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6088 | apply(rule better_LAxR_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6089 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6090 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6091 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6092 |     also have "\<dots> = NotR (z).(M{b:=(x).Ax x a}) a" using new by (simp add: crename_fresh)
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6093 | also have "\<dots> \<longrightarrow>\<^sub>a* NotR (z).(M[b\<turnstile>c>a]) a" using ih by (auto intro: a_star_congs) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6094 | also have "\<dots> = (NotR (z).M c)[b\<turnstile>c>a]" using eq by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6095 |     finally show "(NotR (z).M c){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (NotR (z).M c)[b\<turnstile>c>a]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6096 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6097 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6098 | assume neq: "c\<noteq>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6099 |     have "(NotR (z).M c){b:=(x).Ax x a} = NotR (z).(M{b:=(x).Ax x a}) c" using fs neq by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6100 | also have "\<dots> \<longrightarrow>\<^sub>a* NotR (z).(M[b\<turnstile>c>a]) c" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6101 |     finally show "(NotR (z).M c){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (NotR (z).M c)[b\<turnstile>c>a]" using neq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6102 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6103 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6104 | case (NotL c M z b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6105 | have fs: "c\<sharp>b" "c\<sharp>a" "c\<sharp>x" "c\<sharp>z" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6106 |   have ih: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6107 |   have "(NotL <c>.M z){b:=(x).Ax x a} = NotL <c>.(M{b:=(x).Ax x a}) z" using fs by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6108 | also have "\<dots> \<longrightarrow>\<^sub>a* NotL <c>.(M[b\<turnstile>c>a]) z" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6109 |   finally show "(NotL <c>.M z){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (NotL <c>.M z)[b\<turnstile>c>a]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6110 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6111 | case (AndR c M d N e b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6112 | have fs: "c\<sharp>b" "c\<sharp>a" "c\<sharp>x" "d\<sharp>b" "d\<sharp>a" "d\<sharp>x" "d\<noteq>c" "c\<sharp>N" "c\<sharp>e" "d\<sharp>M" "d\<sharp>e" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6113 |   have ih1: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6114 |   have ih2: "N{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* N[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6115 |   show "(AndR <c>.M <d>.N e){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (AndR <c>.M <d>.N e)[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6116 | proof(cases "e=b") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6117 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6118 | assume eq: "e=b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6119 |     obtain e'::"coname" where new: "e'\<sharp>(Ax x a,M{b:=(x).Ax x a},N{b:=(x).Ax x a},c,d)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6120 | by (rule exists_fresh(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6121 |     have "(AndR <c>.M <d>.N e){b:=(x).Ax x a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6122 |                fresh_fun (\<lambda>e'. Cut <e'>.AndR <c>.(M{b:=(x).Ax x a}) <d>.(N{b:=(x).Ax x a}) e' (x).Ax x a)"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6123 | using eq fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6124 |     also have "\<dots> = Cut <e'>.AndR <c>.(M{b:=(x).Ax x a}) <d>.(N{b:=(x).Ax x a}) e' (x).Ax x a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6125 | using new by (simp add: fresh_fun_simp_AndR fresh_prod) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6126 |     also have "\<dots> \<longrightarrow>\<^sub>a* (AndR <c>.(M{b:=(x).Ax x a}) <d>.(N{b:=(x).Ax x a}) e')[e'\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6127 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6128 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6129 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6130 | apply(rule better_LAxR_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6131 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6132 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6133 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6134 |     also have "\<dots> = AndR <c>.(M{b:=(x).Ax x a}) <d>.(N{b:=(x).Ax x a}) a" using fs new
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6135 | by (auto simp add: fresh_prod fresh_atm subst_fresh crename_fresh) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6136 | also have "\<dots> \<longrightarrow>\<^sub>a* AndR <c>.(M[b\<turnstile>c>a]) <d>.(N[b\<turnstile>c>a]) a" using ih1 ih2 by (auto intro: a_star_congs) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6137 | also have "\<dots> = (AndR <c>.M <d>.N e)[b\<turnstile>c>a]" using eq fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6138 |     finally show "(AndR <c>.M <d>.N e){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (AndR <c>.M <d>.N e)[b\<turnstile>c>a]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6139 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6140 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6141 | assume neq: "e\<noteq>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6142 |     have "(AndR <c>.M <d>.N e){b:=(x).Ax x a} = AndR <c>.(M{b:=(x).Ax x a}) <d>.(N{b:=(x).Ax x a}) e"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6143 | using fs neq by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6144 | also have "\<dots> \<longrightarrow>\<^sub>a* AndR <c>.(M[b\<turnstile>c>a]) <d>.(N[b\<turnstile>c>a]) e" using ih1 ih2 by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6145 |     finally show "(AndR <c>.M <d>.N e){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (AndR <c>.M <d>.N e)[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6146 | using fs neq by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6147 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6148 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6149 | case (AndL1 u M v b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6150 | have fs: "u\<sharp>b" "u\<sharp>a" "u\<sharp>x" "u\<sharp>v" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6151 |   have ih: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6152 |   have "(AndL1 (u).M v){b:=(x).Ax x a} = AndL1 (u).(M{b:=(x).Ax x a}) v" using fs by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6153 | also have "\<dots> \<longrightarrow>\<^sub>a* AndL1 (u).(M[b\<turnstile>c>a]) v" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6154 |   finally show "(AndL1 (u).M v){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (AndL1 (u).M v)[b\<turnstile>c>a]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6155 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6156 | case (AndL2 u M v b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6157 | have fs: "u\<sharp>b" "u\<sharp>a" "u\<sharp>x" "u\<sharp>v" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6158 |   have ih: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6159 |   have "(AndL2 (u).M v){b:=(x).Ax x a} = AndL2 (u).(M{b:=(x).Ax x a}) v" using fs by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6160 | also have "\<dots> \<longrightarrow>\<^sub>a* AndL2 (u).(M[b\<turnstile>c>a]) v" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6161 |   finally show "(AndL2 (u).M v){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (AndL2 (u).M v)[b\<turnstile>c>a]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6162 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6163 | case (OrR1 c M d b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6164 | have fs: "c\<sharp>b" "c\<sharp>a" "c\<sharp>x" "c\<sharp>d" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6165 |   have ih: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6166 |   show "(OrR1 <c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (OrR1 <c>.M d)[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6167 | proof(cases "d=b") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6168 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6169 | assume eq: "d=b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6170 |     obtain a'::"coname" where new: "a'\<sharp>(Ax x a,M{b:=(x).Ax x a},c,x,a)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6171 | by (rule exists_fresh(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6172 |     have "(OrR1 <c>.M d){b:=(x).Ax x a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6173 |              fresh_fun (\<lambda>a'. Cut <a'>.OrR1 <c>.M{b:=(x).Ax x a} a' (x).Ax x a)" using fs eq by (simp)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6174 |     also have "\<dots> = Cut <a'>.OrR1 <c>.M{b:=(x).Ax x a} a' (x).Ax x a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6175 | using new by (simp add: fresh_fun_simp_OrR1) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6176 |     also have "\<dots> \<longrightarrow>\<^sub>a* (OrR1 <c>.M{b:=(x).Ax x a} a')[a'\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6177 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6178 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6179 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6180 | apply(rule better_LAxR_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6181 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6182 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6183 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6184 |     also have "\<dots> = OrR1 <c>.M{b:=(x).Ax x a} a" using fs new
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6185 | by (auto simp add: fresh_prod fresh_atm crename_fresh subst_fresh) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6186 | also have "\<dots> \<longrightarrow>\<^sub>a* OrR1 <c>.(M[b\<turnstile>c>a]) a" using ih by (auto intro: a_star_congs) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6187 | also have "\<dots> = (OrR1 <c>.M d)[b\<turnstile>c>a]" using eq fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6188 |     finally show "(OrR1 <c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (OrR1 <c>.M d)[b\<turnstile>c>a]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6189 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6190 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6191 | assume neq: "d\<noteq>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6192 |     have "(OrR1 <c>.M d){b:=(x).Ax x a} = OrR1 <c>.(M{b:=(x).Ax x a}) d" using fs neq by (simp)
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6193 | also have "\<dots> \<longrightarrow>\<^sub>a* OrR1 <c>.(M[b\<turnstile>c>a]) d" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6194 |     finally show "(OrR1 <c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (OrR1 <c>.M d)[b\<turnstile>c>a]" using fs neq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6195 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6196 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6197 | case (OrR2 c M d b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6198 | have fs: "c\<sharp>b" "c\<sharp>a" "c\<sharp>x" "c\<sharp>d" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6199 |   have ih: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6200 |   show "(OrR2 <c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (OrR2 <c>.M d)[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6201 | proof(cases "d=b") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6202 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6203 | assume eq: "d=b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6204 |     obtain a'::"coname" where new: "a'\<sharp>(Ax x a,M{b:=(x).Ax x a},c,x,a)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6205 | by (rule exists_fresh(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6206 |     have "(OrR2 <c>.M d){b:=(x).Ax x a} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6207 |              fresh_fun (\<lambda>a'. Cut <a'>.OrR2 <c>.M{b:=(x).Ax x a} a' (x).Ax x a)" using fs eq by (simp)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6208 |     also have "\<dots> = Cut <a'>.OrR2 <c>.M{b:=(x).Ax x a} a' (x).Ax x a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6209 | using new by (simp add: fresh_fun_simp_OrR2) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6210 |     also have "\<dots> \<longrightarrow>\<^sub>a* (OrR2 <c>.M{b:=(x).Ax x a} a')[a'\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6211 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6212 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6213 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6214 | apply(rule better_LAxR_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6215 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6216 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6217 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6218 |     also have "\<dots> = OrR2 <c>.M{b:=(x).Ax x a} a" using fs new
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6219 | by (auto simp add: fresh_prod fresh_atm crename_fresh subst_fresh) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6220 | also have "\<dots> \<longrightarrow>\<^sub>a* OrR2 <c>.(M[b\<turnstile>c>a]) a" using ih by (auto intro: a_star_congs) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6221 | also have "\<dots> = (OrR2 <c>.M d)[b\<turnstile>c>a]" using eq fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6222 |     finally show "(OrR2 <c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (OrR2 <c>.M d)[b\<turnstile>c>a]" by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6223 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6224 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6225 | assume neq: "d\<noteq>b" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6226 |     have "(OrR2 <c>.M d){b:=(x).Ax x a} = OrR2 <c>.(M{b:=(x).Ax x a}) d" using fs neq by (simp)
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6227 | also have "\<dots> \<longrightarrow>\<^sub>a* OrR2 <c>.(M[b\<turnstile>c>a]) d" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6228 |     finally show "(OrR2 <c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (OrR2 <c>.M d)[b\<turnstile>c>a]" using fs neq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6229 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6230 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6231 | case (OrL u M v N z b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6232 | have fs: "u\<sharp>b" "u\<sharp>a" "u\<sharp>x" "v\<sharp>b" "v\<sharp>a" "v\<sharp>x" "v\<noteq>u" "u\<sharp>N" "u\<sharp>z" "v\<sharp>M" "v\<sharp>z" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6233 |   have ih1: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6234 |   have ih2: "N{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* N[b\<turnstile>c>a]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6235 |   have "(OrL (u).M (v).N z){b:=(x).Ax x a} = OrL (u).(M{b:=(x).Ax x a}) (v).(N{b:=(x).Ax x a}) z" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6236 | using fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6237 | also have "\<dots> \<longrightarrow>\<^sub>a* OrL (u).(M[b\<turnstile>c>a]) (v).(N[b\<turnstile>c>a]) z" using ih1 ih2 by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6238 |   finally show "(OrL (u).M (v).N z){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (OrL (u).M (v).N z)[b\<turnstile>c>a]" using fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6239 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6240 | case (ImpR z c M d b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6241 | have fs: "z\<sharp>b" "z\<sharp>a" "z\<sharp>x" "c\<sharp>b" "c\<sharp>a" "c\<sharp>x" "z\<sharp>d" "c\<sharp>d" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6242 |   have ih: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6243 |   show "(ImpR (z).<c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (ImpR (z).<c>.M d)[b\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6244 | proof(cases "b=d") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6245 | case True | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6246 | assume eq: "b=d" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6247 |     obtain a'::"coname" where new: "a'\<sharp>(Ax x a,M{b:=(x).Ax x a},x,a,c)" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6248 | by (rule exists_fresh(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6249 |     have "(ImpR (z).<c>.M d){b:=(x).Ax x a} =
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6250 |                 fresh_fun (\<lambda>a'. Cut <a'>.ImpR z.<c>.M{b:=(x).Ax x a} a' (x).Ax x a)" using fs eq by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6251 |     also have "\<dots> = Cut <a'>.ImpR z.<c>.M{b:=(x).Ax x a} a' (x).Ax x a" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6252 | using new by (simp add: fresh_fun_simp_ImpR) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6253 |     also have "\<dots> \<longrightarrow>\<^sub>a* (ImpR z.<c>.M{b:=(x).Ax x a} a')[a'\<turnstile>c>a]"
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6254 | using new | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6255 | apply(rule_tac a_starI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6256 | apply(rule a_redu.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6257 | apply(rule better_LAxR_intro) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6258 | apply(rule fic.intros) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6259 | apply(simp_all add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6260 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6261 |     also have "\<dots> = ImpR z.<c>.M{b:=(x).Ax x a} a" using fs new
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6262 | by (auto simp add: fresh_prod crename_fresh subst_fresh fresh_atm) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6263 | also have "\<dots> \<longrightarrow>\<^sub>a* ImpR z.<c>.(M[b\<turnstile>c>a]) a" using ih by (auto intro: a_star_congs) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6264 | also have "\<dots> = (ImpR z.<c>.M b)[b\<turnstile>c>a]" using eq fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6265 |     finally show "(ImpR (z).<c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (ImpR (z).<c>.M d)[b\<turnstile>c>a]" using eq by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6266 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6267 | case False | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6268 | assume neq: "b\<noteq>d" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6269 |     have "(ImpR (z).<c>.M d){b:=(x).Ax x a} = ImpR (z).<c>.(M{b:=(x).Ax x a}) d" using fs neq by simp
 | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6270 | also have "\<dots> \<longrightarrow>\<^sub>a* ImpR (z).<c>.(M[b\<turnstile>c>a]) d" using ih by (auto intro: a_star_congs) | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6271 |     finally show "(ImpR (z).<c>.M d){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (ImpR (z).<c>.M d)[b\<turnstile>c>a]" using neq fs by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6272 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6273 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6274 | case (ImpL c M u N v b a x) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6275 | have fs: "c\<sharp>b" "c\<sharp>a" "c\<sharp>x" "u\<sharp>b" "u\<sharp>a" "u\<sharp>x" "c\<sharp>N" "c\<sharp>v" "u\<sharp>M" "u\<sharp>v" by fact+ | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6276 |   have ih1: "M{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* M[b\<turnstile>c>a]" by fact
 | 
| 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6277 |   have ih2: "N{b:=(x).Ax x a} \<longrightarrow>\<^sub>a* N[b\<turnstile>c>a]" by fact
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6278 |   have "(ImpL <c>.M (u).N v){b:=(x).Ax x a} = ImpL <c>.(M{b:=(x).Ax x a}) (u).(N{b:=(x).Ax x a}) v" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6279 | using fs by simp | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6280 | also have "\<dots> \<longrightarrow>\<^sub>a* ImpL <c>.(M[b\<turnstile>c>a]) (u).(N[b\<turnstile>c>a]) v" | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6281 | using ih1 ih2 by (auto intro: a_star_congs) | 
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
48567diff
changeset | 6282 |   finally show "(ImpL <c>.M (u).N v){b:=(x).Ax x a} \<longrightarrow>\<^sub>a* (ImpL <c>.M (u).N v)[b\<turnstile>c>a]" 
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6283 | using fs by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6284 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6285 | |
| 63167 | 6286 | text \<open>substitution lemmas\<close> | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6287 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6288 | lemma not_Ax1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6289 |   shows "\<not>(b\<sharp>M) \<Longrightarrow> M{b:=(y).Q} \<noteq> Ax x a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6290 | apply(nominal_induct M avoiding: b y Q x a rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6291 | apply(auto simp add: fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6292 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(y).Q},Q)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6293 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6294 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6295 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6296 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6297 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6298 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname:=(y).Q},Q)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6299 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6300 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6301 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6302 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6303 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6304 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(y).Q},Q,trm2{coname3:=(y).Q},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6305 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6306 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6307 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6308 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6309 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6310 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(y).Q},Q,trm2{coname3:=(y).Q},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6311 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6312 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6313 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6314 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6315 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6316 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm1{coname3:=(y).Q},Q,trm2{coname3:=(y).Q},coname1,coname2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6317 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6318 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6319 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6320 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6321 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6322 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(y).Q},Q,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6323 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6324 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6325 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6326 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6327 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6328 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(y).Q},Q,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6329 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6330 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6331 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6332 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6333 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6334 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(y).Q},Q,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6335 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6336 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6337 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6338 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6339 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6340 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(y).Q},Q,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6341 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6342 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6343 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6344 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6345 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6346 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(y).Q},Q,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6347 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6348 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6349 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6350 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6351 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6352 | apply(subgoal_tac "\<exists>x'::coname. x'\<sharp>(trm{coname2:=(y).Q},Q,coname1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6353 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6354 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6355 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6356 | apply(simp add: fresh_fun_simp_ImpR abs_fresh abs_supp fin_supp fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6357 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6358 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6359 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6360 | lemma not_Ax2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6361 |   shows "\<not>(x\<sharp>M) \<Longrightarrow> M{x:=<b>.Q} \<noteq> Ax y a"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6362 | apply(nominal_induct M avoiding: b y Q x a rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6363 | apply(auto simp add: fresh_atm abs_fresh abs_supp fin_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6364 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.Q},Q)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6365 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6366 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6367 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6368 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6369 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6370 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.Q},Q)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6371 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6372 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6373 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6374 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6375 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6376 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.Q},Q,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6377 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6378 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6379 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6380 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6381 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6382 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.Q},Q,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6383 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6384 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6385 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6386 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6387 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6388 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.Q},Q,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6389 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6390 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6391 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6392 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6393 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6394 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm{x:=<b>.Q},Q,name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6395 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6396 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6397 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6398 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6399 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6400 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{x:=<b>.Q},Q,trm2{x:=<b>.Q},name1,name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6401 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6402 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6403 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6404 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6405 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6406 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{x:=<b>.Q},Q,trm2{x:=<b>.Q},name1,name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6407 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6408 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6409 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6410 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6411 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6412 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{x:=<b>.Q},Q,trm2{x:=<b>.Q},name1,name2)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6413 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6414 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6415 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6416 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6417 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6418 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<b>.Q},Q,trm2{name2:=<b>.Q},name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6419 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6420 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6421 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6422 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6423 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6424 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<b>.Q},Q,trm2{name2:=<b>.Q},name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6425 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6426 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6427 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6428 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6429 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6430 | apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(trm1{name2:=<b>.Q},Q,trm2{name2:=<b>.Q},name1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6431 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6432 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6433 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6434 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6435 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6436 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6437 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6438 | lemma interesting_subst1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6439 | assumes a: "x\<noteq>y" "x\<sharp>P" "y\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6440 |   shows "N{y:=<c>.P}{x:=<c>.P} = N{x:=<c>.Ax y c}{y:=<c>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6441 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6442 | proof(nominal_induct N avoiding: x y c P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6443 | case Ax | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6444 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6445 | by (auto simp add: abs_fresh fresh_atm forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6446 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6447 | case (Cut d M u M' x' y' c P) | 
| 41893 | 6448 | with assms show ?case | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6449 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6450 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6451 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6452 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6453 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6454 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6455 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6456 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6457 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6458 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6459 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6460 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6461 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6462 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6463 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6464 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6465 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6466 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6467 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6468 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6469 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6470 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6471 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6472 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6473 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6474 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6475 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6476 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6477 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6478 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6479 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6480 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6481 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6482 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6483 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6484 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6485 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6486 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6487 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6488 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6489 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6490 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6491 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6492 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6493 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6494 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6495 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6496 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6497 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6498 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6499 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6500 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6501 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6502 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6503 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6504 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6505 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6506 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6507 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6508 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6509 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6510 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6511 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6512 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6513 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6514 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6515 | apply(case_tac "y'\<sharp>M") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6516 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6517 | apply(simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6518 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6519 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6520 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6521 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6522 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6523 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6524 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6525 | apply(case_tac "x'\<sharp>M") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6526 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6527 | apply(simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6528 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6529 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6530 | case NotR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6531 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6532 | by (auto simp add: abs_fresh fresh_atm forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6533 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6534 | case (NotL d M u) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6535 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6536 | apply (auto simp add: abs_fresh fresh_atm forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6537 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{y:=<c>.P},M{x:=<c>.Ax y c}{y:=<c>.P},y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6538 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6539 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6540 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6541 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6542 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6543 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6544 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6545 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6546 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6547 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6548 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6549 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{x:=<c>.Ax y c},M{x:=<c>.Ax y c}{y:=<c>.P},Ax y c,y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6550 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6551 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6552 | apply(simp only: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6553 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6554 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6555 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6556 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6557 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6558 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6559 | apply(simp add: trm.inject alpha forget subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6560 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6561 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6562 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6563 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6564 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6565 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6566 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6567 | case (AndR d1 M d2 M' d3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6568 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6569 | by (auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6570 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6571 | case (AndL1 u M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6572 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6573 | apply(auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6574 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{y:=<c>.P},M{x:=<c>.Ax y c}{y:=<c>.P},u,y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6575 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6576 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6577 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6578 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6579 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6580 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6581 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6582 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6583 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6584 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6585 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6586 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,Ax y c,M{x:=<c>.Ax y c},M{x:=<c>.Ax y c}{y:=<c>.P},u,y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6587 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6588 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6589 | apply(simp only: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6590 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6591 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6592 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6593 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6594 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6595 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6596 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6597 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6598 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6599 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6600 | case (AndL2 u M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6601 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6602 | apply(auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6603 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{y:=<c>.P},M{x:=<c>.Ax y c}{y:=<c>.P},u,y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6604 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6605 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6606 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6607 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6608 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6609 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6610 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6611 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6612 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6613 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6614 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6615 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,Ax y c,M{x:=<c>.Ax y c},M{x:=<c>.Ax y c}{y:=<c>.P},u,y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6616 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6617 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6618 | apply(simp only: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6619 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6620 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6621 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6622 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6623 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6624 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6625 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6626 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6627 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6628 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6629 | case OrR1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6630 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6631 | by (auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6632 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6633 | case OrR2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6634 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6635 | by (auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6636 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6637 | case (OrL x1 M x2 M' x3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6638 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6639 | apply(auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6640 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{y:=<c>.P},M{x:=<c>.Ax y c}{y:=<c>.P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6641 |                                         M'{y:=<c>.P},M'{x:=<c>.Ax y c}{y:=<c>.P},x1,x2,x3,y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6642 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6643 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6644 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6645 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6646 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6647 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6648 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6649 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6650 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6651 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6652 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6653 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6654 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6655 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6656 | apply(force) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6657 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6658 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6659 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,Ax y c,M{x:=<c>.Ax y c},M{x:=<c>.Ax y c}{y:=<c>.P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6660 |                                         M'{x:=<c>.Ax y c},M'{x:=<c>.Ax y c}{y:=<c>.P},x1,x2,x3,y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6661 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6662 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6663 | apply(simp only: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6664 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6665 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6666 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6667 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6668 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6669 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6670 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6671 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6672 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6673 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6674 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6675 | apply(force) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6676 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6677 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6678 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6679 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6680 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6681 | case ImpR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6682 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6683 | by (auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6684 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6685 | case (ImpL a M x1 M' x2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6686 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6687 | apply(auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6688 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{x2:=<c>.P},M{x:=<c>.Ax x2 c}{x2:=<c>.P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6689 |                                         M'{x2:=<c>.P},M'{x:=<c>.Ax x2 c}{x2:=<c>.P},x1,y,x)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6690 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6691 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6692 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6693 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6694 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6695 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6696 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6697 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6698 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6699 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6700 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6701 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6702 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6703 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6704 | apply(force) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6705 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6706 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,Ax y c,M{x2:=<c>.Ax y c},M{x2:=<c>.Ax y c}{y:=<c>.P},
 | 
| 48567 
3c4d7ff75f01
tuned proofs -- avoid odd situations of polymorphic Frees in goal state;
 wenzelm parents: 
41893diff
changeset | 6707 |                                         M'{x2:=<c>.Ax y c},M'{x2:=<c>.Ax y c}{y:=<c>.P},x1,x2,y,x)")
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6708 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6709 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6710 | apply(simp only: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6711 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6712 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6713 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6714 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6715 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6716 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6717 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6718 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6719 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6720 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6721 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6722 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6723 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6724 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6725 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6726 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6727 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6728 | lemma interesting_subst1': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6729 | assumes a: "x\<noteq>y" "x\<sharp>P" "y\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6730 |   shows "N{y:=<c>.P}{x:=<c>.P} = N{x:=<a>.Ax y a}{y:=<c>.P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6731 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6732 | show ?thesis | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6733 | proof (cases "c=a") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6734 | case True then show ?thesis using a by (simp add: interesting_subst1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6735 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6736 | case False then show ?thesis using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6737 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6738 |       apply(subgoal_tac "N{x:=<a>.Ax y a} = N{x:=<c>.([(c,a)]\<bullet>Ax y a)}") 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6739 | apply(simp add: interesting_subst1 calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6740 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6741 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6742 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6743 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6744 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6745 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6746 | lemma interesting_subst2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6747 | assumes a: "a\<noteq>b" "a\<sharp>P" "b\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6748 |   shows "N{a:=(y).P}{b:=(y).P} = N{b:=(y).Ax y a}{a:=(y).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6749 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6750 | proof(nominal_induct N avoiding: a b y P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6751 | case Ax | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6752 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6753 | by (auto simp add: abs_fresh fresh_atm forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6754 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6755 | case (Cut d M u M' x' y' c P) | 
| 41893 | 6756 | with assms show ?case | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6757 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6758 | apply(auto simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6759 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6760 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6761 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6762 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6763 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6764 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6765 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6766 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6767 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6768 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6769 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6770 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6771 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6772 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6773 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6774 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6775 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6776 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6777 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6778 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6779 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6780 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6781 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6782 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6783 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6784 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6785 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6786 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6787 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6788 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6789 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6790 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6791 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6792 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6793 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6794 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6795 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6796 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6797 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6798 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6799 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6800 | apply(rule impI) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6801 | apply(simp add: fresh_atm trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6802 | apply(case_tac "x'\<sharp>M'") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6803 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6804 | apply(simp add: not_Ax1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6805 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6806 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6807 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6808 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6809 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6810 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6811 | apply(case_tac "y'\<sharp>M'") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6812 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6813 | apply(simp add: not_Ax1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6814 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6815 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6816 | case NotL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6817 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6818 | by (auto simp add: abs_fresh fresh_atm forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6819 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6820 | case (NotR u M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6821 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6822 | apply (auto simp add: abs_fresh fresh_atm forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6823 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(b,P,M{d:=(y).P},M{b:=(y).Ax y d}{d:=(y).P},u,y)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6824 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6825 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6826 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6827 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6828 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6829 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6830 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6831 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6832 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6833 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6834 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6835 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(P,M{d:=(y).Ax y a},M{d:=(y).Ax y a}{a:=(y).P},Ax y a,y,d)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6836 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6837 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6838 | apply(simp only: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6839 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6840 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6841 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6842 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6843 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6844 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6845 | apply(simp add: trm.inject alpha forget subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6846 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6847 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6848 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6849 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6850 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6851 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6852 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6853 | case (AndR d1 M d2 M' d3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6854 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6855 | apply(auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6856 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(P,M{d3:=(y).P},M{b:=(y).Ax y d3}{d3:=(y).P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6857 |                                         M'{d3:=(y).P},M'{b:=(y).Ax y d3}{d3:=(y).P},d1,d2,d3,b,y)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6858 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6859 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6860 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6861 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6862 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6863 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6864 | apply(simp add: abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6865 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6866 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6867 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6868 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6869 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6870 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6871 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6872 | apply(force) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6873 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6874 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6875 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(P,Ax y a,M{d3:=(y).Ax y a},M{d3:=(y).Ax y a}{a:=(y).P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6876 |                                         M'{d3:=(y).Ax y a},M'{d3:=(y).Ax y a}{a:=(y).P},d1,d2,d3,y,b)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6877 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6878 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6879 | apply(simp only: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6880 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6881 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6882 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6883 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6884 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6885 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6886 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6887 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6888 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6889 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6890 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6891 | apply(force) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6892 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6893 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6894 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6895 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6896 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6897 | case (AndL1 u M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6898 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6899 | by (auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6900 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6901 | case (AndL2 u M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6902 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6903 | by (auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6904 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6905 | case (OrR1 d M e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6906 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6907 | apply (auto simp add: abs_fresh fresh_atm forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6908 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(b,P,M{e:=(y).P},M{b:=(y).Ax y e}{e:=(y).P},d,e)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6909 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6910 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6911 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6912 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6913 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6914 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6915 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6916 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6917 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6918 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6919 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6920 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(b,P,Ax y a,M{e:=(y).Ax y a},M{e:=(y).Ax y a}{a:=(y).P},d,e)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6921 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6922 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6923 | apply(simp only: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6924 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6925 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6926 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6927 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6928 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6929 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6930 | apply(simp add: trm.inject alpha forget subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6931 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6932 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6933 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6934 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6935 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6936 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6937 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6938 | case (OrR2 d M e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6939 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6940 | apply (auto simp add: abs_fresh fresh_atm forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6941 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(b,P,M{e:=(y).P},M{b:=(y).Ax y e}{e:=(y).P},d,e)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6942 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6943 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6944 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6945 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6946 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6947 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6948 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6949 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6950 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6951 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6952 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6953 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(b,P,Ax y a,M{e:=(y).Ax y a},M{e:=(y).Ax y a}{a:=(y).P},d,e)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6954 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6955 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6956 | apply(simp only: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6957 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6958 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6959 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6960 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6961 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6962 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6963 | apply(simp add: trm.inject alpha forget subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6964 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6965 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6966 | apply(simp add: abs_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6967 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6968 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6969 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6970 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6971 | case (OrL x1 M x2 M' x3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6972 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6973 | by(auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6974 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6975 | case ImpL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6976 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6977 | by (auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6978 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6979 | case (ImpR u e M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6980 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6981 | apply(auto simp add: abs_fresh fresh_atm forget trm.inject subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6982 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(b,e,d,P,M{d:=(y).P},M{b:=(y).Ax y d}{d:=(y).P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6983 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6984 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6985 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6986 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6987 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6988 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6989 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6990 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6991 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6992 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6993 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6994 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(e,d,P,Ax y a,M{d:=(y).Ax y a},M{d:=(y).Ax y a}{a:=(y).P})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6995 | apply(erule exE, simp only: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6996 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6997 | apply(simp only: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6998 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 6999 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7000 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7001 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7002 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7003 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7004 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7005 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7006 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7007 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7008 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7009 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7010 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7011 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7012 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7013 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7014 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7015 | lemma interesting_subst2': | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7016 | assumes a: "a\<noteq>b" "a\<sharp>P" "b\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7017 |   shows "N{a:=(y).P}{b:=(y).P} = N{b:=(z).Ax z a}{a:=(y).P}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7018 | proof - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7019 | show ?thesis | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7020 | proof (cases "z=y") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7021 | case True then show ?thesis using a by (simp add: interesting_subst2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7022 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7023 | case False then show ?thesis using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7024 | apply - | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7025 |       apply(subgoal_tac "N{b:=(z).Ax z a} = N{b:=(y).([(y,z)]\<bullet>Ax z a)}") 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7026 | apply(simp add: interesting_subst2 calc_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7027 | apply(rule subst_rename) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7028 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7029 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7030 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7031 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7032 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7033 | lemma subst_subst1: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7034 | assumes a: "a\<sharp>(Q,b)" "x\<sharp>(y,P,Q)" "b\<sharp>Q" "y\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7035 |   shows "M{x:=<a>.P}{b:=(y).Q} = M{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7036 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7037 | proof(nominal_induct M avoiding: x a P b y Q rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7038 | case (Ax z c) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7039 | have fs: "a\<sharp>(Q,b)" "x\<sharp>(y,P,Q)" "b\<sharp>Q" "y\<sharp>P" by fact+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7040 |   { assume asm: "z=x \<and> c=b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7041 |     have "(Ax x b){x:=<a>.P}{b:=(y).Q} = (Cut <a>.P (x).Ax x b){b:=(y).Q}" using fs by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7042 |     also have "\<dots> = Cut <a>.(P{b:=(y).Q}) (y).Q"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7043 | using fs by (simp_all add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7044 |     also have "\<dots> = Cut <a>.(P{b:=(y).Q}) (y).(Q{x:=<a>.(P{b:=(y).Q})})" using fs by (simp add: forget)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7045 |     also have "\<dots> = (Cut <b>.Ax x b (y).Q){x:=<a>.(P{b:=(y).Q})}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7046 | using fs asm by (auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7047 |     also have "\<dots> = (Ax x b){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" using fs by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7048 |     finally have "(Ax z c){x:=<a>.P}{b:=(y).Q} = (Ax z c){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7049 | using asm by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7050 | } | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7051 | moreover | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7052 |   { assume asm: "z\<noteq>x \<and> c=b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7053 |     have "(Ax z c){x:=<a>.P}{b:=(y).Q} = (Ax z c){b:=(y).Q}" using asm by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7054 | also have "\<dots> = Cut <b>.Ax z c (y).Q" using fs asm by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7055 |     also have "\<dots> = Cut <b>.(Ax z c{x:=<a>.(P{b:=(y).Q})}) (y).(Q{x:=<a>.(P{b:=(y).Q})})" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7056 | using fs asm by (simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7057 |     also have "\<dots> = (Cut <b>.Ax z c (y).Q){x:=<a>.(P{b:=(y).Q})}" using asm fs
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7058 | by (auto simp add: trm.inject subst_fresh fresh_prod fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7059 |     also have "\<dots> = (Ax z c){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" using asm fs by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7060 |     finally have "(Ax z c){x:=<a>.P}{b:=(y).Q} = (Ax z c){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7061 | } | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7062 | moreover | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7063 |   { assume asm: "z=x \<and> c\<noteq>b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7064 |     have "(Ax z c){x:=<a>.P}{b:=(y).Q} = (Cut <a>.P (x).Ax z c){b:=(y).Q}" using fs asm by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7065 |     also have "\<dots> = Cut <a>.(P{b:=(y).Q}) (x).Ax z c" using fs asm by (auto simp add: trm.inject abs_fresh)
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7066 |     also have "\<dots> = (Ax z c){x:=<a>.(P{b:=(y).Q})}" using fs asm by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7067 |     also have "\<dots> = (Ax z c){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" using asm by auto
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7068 |     finally have "(Ax z c){x:=<a>.P}{b:=(y).Q} = (Ax z c){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7069 | } | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7070 | moreover | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7071 |   { assume asm: "z\<noteq>x \<and> c\<noteq>b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7072 |     have "(Ax z c){x:=<a>.P}{b:=(y).Q} = (Ax z c){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" using asm by auto
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7073 | } | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7074 | ultimately show ?case by blast | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7075 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7076 | case (Cut c M z N) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7077 |   { assume asm: "M = Ax x c \<and> N = Ax z b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7078 |     have "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <a>.P (z).(N{x:=<a>.P})){b:=(y).Q}" 
 | 
| 41893 | 7079 | using Cut asm by simp | 
| 7080 |     also have "\<dots> = (Cut <a>.P (z).N){b:=(y).Q}" using Cut asm by (simp add: fresh_atm)
 | |
| 7081 |     also have "\<dots> = (Cut <a>.(P{b:=(y).Q}) (y).Q)" using Cut asm by (auto simp add: fresh_prod fresh_atm)
 | |
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7082 |     finally have eq1: "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <a>.(P{b:=(y).Q}) (y).Q)" by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7083 |     have "(Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})} = (Cut <c>.M (y).Q){x:=<a>.(P{b:=(y).Q})}"
 | 
| 41893 | 7084 | using Cut asm by (simp add: fresh_atm) | 
| 7085 |     also have "\<dots> = Cut <a>.(P{b:=(y).Q}) (y).(Q{x:=<a>.(P{b:=(y).Q})})" using Cut asm
 | |
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7086 | by (auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 41893 | 7087 |     also have "\<dots> = Cut <a>.(P{b:=(y).Q}) (y).Q" using Cut asm by (simp add: forget)
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7088 |     finally have eq2: "(Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})} = Cut <a>.(P{b:=(y).Q}) (y).Q"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7089 | by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7090 |     have "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7091 | using eq1 eq2 by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7092 | } | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7093 | moreover | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7094 |   { assume asm: "M \<noteq> Ax x c \<and> N = Ax z b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7095 |     have neq: "M{b:=(y).Q} \<noteq> Ax x c"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7096 | proof (cases "b\<sharp>M") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7097 | case True then show ?thesis using asm by (simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7098 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7099 | case False then show ?thesis by (simp add: not_Ax1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7100 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7101 |     have "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <c>.(M{x:=<a>.P}) (z).(N{x:=<a>.P})){b:=(y).Q}"
 | 
| 41893 | 7102 | using Cut asm by simp | 
| 7103 |     also have "\<dots> = (Cut <c>.(M{x:=<a>.P}) (z).N){b:=(y).Q}" using Cut asm by (simp add: fresh_atm)
 | |
| 7104 |     also have "\<dots> = Cut <c>.(M{x:=<a>.P}{b:=(y).Q}) (y).Q" using Cut asm by (simp add: abs_fresh)
 | |
| 7105 |     also have "\<dots> = Cut <c>.(M{b:=(y).Q}{x:=<a>.P{b:=(y).Q}}) (y).Q" using Cut asm by simp
 | |
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7106 | finally | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7107 |     have eq1: "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = Cut <c>.(M{b:=(y).Q}{x:=<a>.P{b:=(y).Q}}) (y).Q" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7108 | by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7109 |     have "(Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})} = 
 | 
| 41893 | 7110 |                (Cut <c>.(M{b:=(y).Q}) (y).Q){x:=<a>.(P{b:=(y).Q})}" using Cut asm by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7111 |     also have "\<dots> = Cut <c>.(M{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}) (y).(Q{x:=<a>.(P{b:=(y).Q})})"
 | 
| 41893 | 7112 | using Cut asm neq by (auto simp add: fresh_prod fresh_atm subst_fresh abs_fresh) | 
| 7113 |     also have "\<dots> = Cut <c>.(M{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}) (y).Q" using Cut asm by (simp add: forget)
 | |
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7114 |     finally have eq2: "(Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})} 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7115 |                                        = Cut <c>.(M{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}) (y).Q" by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7116 |     have "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}" 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7117 | using eq1 eq2 by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7118 | } | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7119 | moreover | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7120 |   { assume asm: "M = Ax x c \<and> N \<noteq> Ax z b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7121 |     have neq: "N{x:=<a>.P} \<noteq> Ax z b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7122 | proof (cases "x\<sharp>N") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7123 | case True then show ?thesis using asm by (simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7124 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7125 | case False then show ?thesis by (simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7126 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7127 |     have "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <a>.P (z).(N{x:=<a>.P})){b:=(y).Q}"
 | 
| 41893 | 7128 | using Cut asm by simp | 
| 7129 |     also have "\<dots> = Cut <a>.(P{b:=(y).Q}) (z).(N{x:=<a>.P}{b:=(y).Q})" using Cut asm neq 
 | |
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7130 | by (simp add: abs_fresh) | 
| 41893 | 7131 |     also have "\<dots> = Cut <a>.(P{b:=(y).Q}) (z).(N{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})})" using Cut asm by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7132 |     finally have eq1: "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7133 |                     = Cut <a>.(P{b:=(y).Q}) (z).(N{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})})" by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7134 |     have "(Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})} 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7135 |                     = (Cut <c>.(M{b:=(y).Q}) (z).(N{b:=(y).Q})){x:=<a>.(P{b:=(y).Q})}"
 | 
| 41893 | 7136 | using Cut asm by auto | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7137 |     also have "\<dots> = (Cut <c>.M (z).(N{b:=(y).Q})){x:=<a>.(P{b:=(y).Q})}"
 | 
| 41893 | 7138 | using Cut asm by (auto simp add: fresh_atm) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7139 |     also have "\<dots> = Cut <a>.(P{b:=(y).Q}) (z).(N{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})})" 
 | 
| 41893 | 7140 | using Cut asm by (simp add: fresh_prod fresh_atm subst_fresh) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7141 | finally | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7142 |     have eq2: "(Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})} 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7143 |          = Cut <a>.(P{b:=(y).Q}) (z).(N{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})})" by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7144 |     have "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7145 | using eq1 eq2 by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7146 | } | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7147 | moreover | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7148 |   { assume asm: "M \<noteq> Ax x c \<and> N \<noteq> Ax z b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7149 |     have neq1: "N{x:=<a>.P} \<noteq> Ax z b"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7150 | proof (cases "x\<sharp>N") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7151 | case True then show ?thesis using asm by (simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7152 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7153 | case False then show ?thesis by (simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7154 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7155 |     have neq2: "M{b:=(y).Q} \<noteq> Ax x c"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7156 | proof (cases "b\<sharp>M") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7157 | case True then show ?thesis using asm by (simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7158 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7159 | case False then show ?thesis by (simp add: not_Ax1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7160 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7161 |     have "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <c>.(M{x:=<a>.P}) (z).(N{x:=<a>.P})){b:=(y).Q}"
 | 
| 41893 | 7162 | using Cut asm by simp | 
| 7163 |     also have "\<dots> = Cut <c>.(M{x:=<a>.P}{b:=(y).Q}) (z).(N{x:=<a>.P}{b:=(y).Q})" using Cut asm neq1
 | |
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7164 | by (simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7165 |     also have "\<dots> = Cut <c>.(M{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}) (z).(N{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})})"
 | 
| 41893 | 7166 | using Cut asm by simp | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7167 |     finally have eq1: "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q}
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7168 |              = Cut <c>.(M{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}) (z).(N{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})})" by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7169 |     have "(Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})} = 
 | 
| 41893 | 7170 |                 (Cut <c>.(M{b:=(y).Q}) (z).(N{b:=(y).Q})){x:=<a>.(P{b:=(y).Q})}" using Cut asm neq1 by simp
 | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7171 |     also have "\<dots> = Cut <c>.(M{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}) (z).(N{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})})"
 | 
| 41893 | 7172 | using Cut asm neq2 by (simp add: fresh_prod fresh_atm subst_fresh) | 
| 36277 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7173 |     finally have eq2: "(Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})} = 
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7174 |            Cut <c>.(M{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}) (z).(N{b:=(y).Q}{x:=<a>.(P{b:=(y).Q})})" by simp
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7175 |     have "(Cut <c>.M (z).N){x:=<a>.P}{b:=(y).Q} = (Cut <c>.M (z).N){b:=(y).Q}{x:=<a>.(P{b:=(y).Q})}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7176 | using eq1 eq2 by simp | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7177 | } | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7178 | ultimately show ?case by blast | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7179 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7180 | case (NotR z M c) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7181 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7182 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7183 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(M{c:=(y).Q},M{c:=(y).Q}{x:=<a>.P{c:=(y).Q}},Q,a,P,c,y)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7184 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7185 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7186 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7187 | apply(simp add: fresh_fun_simp_NotR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7188 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7189 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7190 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7191 | apply(simp add: fresh_prod fresh_atm subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7192 | apply(simp add: fresh_prod fresh_atm subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7193 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7194 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7195 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7196 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7197 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7198 | case (NotL c M z) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7199 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7200 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7201 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{x:=<a>.P},P{b:=(y).Q},M{b:=(y).Q}{x:=<a>.P{b:=(y).Q}},y,Q)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7202 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7203 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7204 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7205 | apply(simp add: fresh_fun_simp_NotL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7206 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7207 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7208 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7209 | case (AndR c1 M c2 N c3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7210 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7211 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7212 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(Q,M{c3:=(y).Q},M{c3:=(y).Q}{x:=<a>.P{c3:=(y).Q}},c2,c3,a,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7213 |                                      P{c3:=(y).Q},N{c3:=(y).Q},N{c3:=(y).Q}{x:=<a>.P{c3:=(y).Q}},c1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7214 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7215 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7216 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7217 | apply(simp add: fresh_fun_simp_AndR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7218 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7219 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7220 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7221 | apply(simp_all add: fresh_atm abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7222 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7223 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7224 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7225 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7226 | case (AndL1 z1 M z2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7227 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7228 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7229 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{x:=<a>.P},P{b:=(y).Q},z1,y,Q,M{b:=(y).Q}{x:=<a>.P{b:=(y).Q}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7230 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7231 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7232 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7233 | apply(simp add: fresh_fun_simp_AndL1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7234 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7235 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7236 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7237 | case (AndL2 z1 M z2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7238 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7239 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7240 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{x:=<a>.P},P{b:=(y).Q},z1,y,Q,M{b:=(y).Q}{x:=<a>.P{b:=(y).Q}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7241 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7242 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7243 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7244 | apply(simp add: fresh_fun_simp_AndL2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7245 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7246 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7247 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7248 | case (OrL z1 M z2 N z3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7249 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7250 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7251 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,M{x:=<a>.P},M{b:=(y).Q}{x:=<a>.P{b:=(y).Q}},z2,z3,a,y,Q,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7252 |                                      P{b:=(y).Q},N{x:=<a>.P},N{b:=(y).Q}{x:=<a>.P{b:=(y).Q}},z1)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7253 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7254 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7255 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7256 | apply(simp add: fresh_fun_simp_OrL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7257 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7258 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7259 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7260 | apply(simp_all add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7261 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7262 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7263 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7264 | case (OrR1 c1 M c2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7265 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7266 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7267 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(Q,M{c2:=(y).Q},a,P{c2:=(y).Q},c1,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7268 |                                                      M{c2:=(y).Q}{x:=<a>.P{c2:=(y).Q}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7269 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7270 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7271 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7272 | apply(simp add: fresh_fun_simp_OrR1 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7273 | apply(simp_all add: fresh_atm subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7274 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7275 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7276 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7277 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7278 | case (OrR2 c1 M c2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7279 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7280 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7281 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(Q,M{c2:=(y).Q},a,P{c2:=(y).Q},c1,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7282 |                                                      M{c2:=(y).Q}{x:=<a>.P{c2:=(y).Q}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7283 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7284 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7285 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7286 | apply(simp add: fresh_fun_simp_OrR2 abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7287 | apply(simp_all add: fresh_atm subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7288 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7289 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7290 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7291 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7292 | case (ImpR z c M d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7293 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7294 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7295 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(Q,M{d:=(y).Q},a,P{d:=(y).Q},c,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7296 |                                                      M{d:=(y).Q}{x:=<a>.P{d:=(y).Q}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7297 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7298 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7299 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7300 | apply(simp add: fresh_fun_simp_ImpR abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7301 | apply(simp_all add: fresh_atm subst_fresh forget abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7302 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7303 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7304 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7305 | case (ImpL c M z N u) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7306 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7307 | apply(auto simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7308 |     apply(subgoal_tac "\<exists>z'::name. z'\<sharp>(P,P{b:=(y).Q},M{u:=<a>.P},N{u:=<a>.P},y,Q,
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7309 |                         M{b:=(y).Q}{u:=<a>.P{b:=(y).Q}},N{b:=(y).Q}{u:=<a>.P{b:=(y).Q}},z)")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7310 | apply(erule exE) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7311 | apply(simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7312 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7313 | apply(simp add: fresh_fun_simp_ImpL abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7314 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7315 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7316 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7317 | apply(simp_all add: fresh_atm subst_fresh forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7318 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7319 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7320 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7321 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7322 | lemma subst_subst2: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7323 | assumes a: "a\<sharp>(b,P,N)" "x\<sharp>(y,P,M)" "b\<sharp>(M,N)" "y\<sharp>P" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7324 |   shows "M{a:=(x).N}{y:=<b>.P} = M{y:=<b>.P}{a:=(x).N{y:=<b>.P}}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7325 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7326 | proof(nominal_induct M avoiding: a x N y b P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7327 | case (Ax z c) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7328 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7329 | by (auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7330 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7331 | case (Cut d M' u M'') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7332 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7333 | apply(simp add: fresh_atm fresh_prod trm.inject abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7334 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7335 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7336 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7337 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7338 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7339 | apply(simp add: abs_fresh subst_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7340 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7341 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7342 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7343 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7344 | apply(case_tac "a\<sharp>M'") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7345 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7346 | apply(simp add: not_Ax1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7347 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7348 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7349 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7350 | apply(simp add: abs_fresh subst_fresh fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7351 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7352 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7353 | apply(case_tac "y\<sharp>M''") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7354 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7355 | apply(simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7356 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7357 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7358 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7359 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7360 | apply(simp add: subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7361 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7362 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7363 | apply(case_tac "y\<sharp>M''") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7364 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7365 | apply(simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7366 | apply(case_tac "a\<sharp>M'") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7367 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7368 | apply(simp add: not_Ax1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7369 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7370 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7371 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7372 | apply(simp add: subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7373 | apply(simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7374 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7375 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7376 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7377 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7378 | apply(simp add: subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7379 | apply(simp add: subst_fresh abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7380 | apply(auto)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7381 | apply(case_tac "y\<sharp>M''") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7382 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7383 | apply(simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7384 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7385 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7386 | case (NotR z M' d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7387 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7388 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7389 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(y,P,N,N{y:=<b>.P},M'{d:=(x).N},M'{y:=<b>.P}{d:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7390 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7391 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7392 | apply(simp add: fresh_fun_simp_NotR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7393 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7394 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7395 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7396 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7397 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7398 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7399 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7400 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7401 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7402 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7403 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7404 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7405 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7406 | case (NotL d M' z) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7407 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7408 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7409 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(z,y,P,N,N{y:=<b>.P},M'{y:=<b>.P},M'{y:=<b>.P}{a:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7410 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7411 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7412 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7413 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7414 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7415 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7416 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7417 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7418 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7419 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7420 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7421 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7422 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7423 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7424 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7425 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7426 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7427 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7428 | case (AndR d M' e M'' f) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7429 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7430 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7431 |     apply(subgoal_tac "\<exists>a'::coname. a'\<sharp>(P,b,d,e,N,N{y:=<b>.P},M'{f:=(x).N},M''{f:=(x).N},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7432 |                   M'{y:=<b>.P}{f:=(x).N{y:=<b>.P}},M''{y:=<b>.P}{f:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7433 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7434 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7435 | apply(simp add: fresh_fun_simp_AndR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7436 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7437 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7438 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7439 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7440 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7441 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7442 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7443 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7444 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7445 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7446 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7447 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7448 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7449 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7450 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7451 | case (AndL1 z M' u) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7452 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7453 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7454 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,b,z,u,x,N,M'{y:=<b>.P},M'{y:=<b>.P}{a:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7455 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7456 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7457 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7458 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7459 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7460 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7461 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7462 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7463 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7464 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7465 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7466 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7467 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7468 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7469 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7470 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7471 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7472 | case (AndL2 z M' u) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7473 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7474 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7475 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(P,b,z,u,x,N,M'{y:=<b>.P},M'{y:=<b>.P}{a:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7476 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7477 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7478 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7479 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7480 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7481 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7482 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7483 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7484 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7485 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7486 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7487 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7488 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7489 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7490 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7491 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7492 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7493 | case (OrL u M' v M'' w) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7494 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7495 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7496 |     apply(subgoal_tac "\<exists>z'::name. z'\<sharp>(P,b,u,w,v,N,N{y:=<b>.P},M'{y:=<b>.P},M''{y:=<b>.P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7497 |                   M'{y:=<b>.P}{a:=(x).N{y:=<b>.P}},M''{y:=<b>.P}{a:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7498 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7499 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7500 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7501 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7502 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7503 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7504 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7505 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7506 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7507 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7508 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7509 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7510 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7511 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7512 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7513 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7514 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7515 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7516 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7517 | case (OrR1 e M' f) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7518 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7519 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7520 |     apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(P,b,e,f,x,N,N{y:=<b>.P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7521 |                                         M'{f:=(x).N},M'{y:=<b>.P}{f:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7522 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7523 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7524 | apply(simp add: fresh_fun_simp_OrR1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7525 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7526 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7527 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7528 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7529 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7530 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7531 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7532 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7533 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7534 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7535 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7536 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7537 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7538 | case (OrR2 e M' f) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7539 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7540 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7541 |     apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(P,b,e,f,x,N,N{y:=<b>.P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7542 |                                         M'{f:=(x).N},M'{y:=<b>.P}{f:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7543 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7544 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7545 | apply(simp add: fresh_fun_simp_OrR2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7546 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7547 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7548 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7549 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7550 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7551 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7552 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7553 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7554 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7555 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7556 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7557 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7558 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7559 | case (ImpR x e M' f) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7560 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7561 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7562 |     apply(subgoal_tac "\<exists>c'::coname. c'\<sharp>(P,b,e,f,x,N,N{y:=<b>.P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7563 |                                         M'{f:=(x).N},M'{y:=<b>.P}{f:=(x).N{y:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7564 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7565 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7566 | apply(simp add: fresh_fun_simp_ImpR) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7567 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7568 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7569 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7570 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7571 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7572 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7573 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7574 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7575 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7576 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7577 | apply(simp add: fresh_atm trm.inject alpha abs_fresh fin_supp abs_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7578 | apply(rule exists_fresh'(2)[OF fs_coname1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7579 | apply(simp add: fresh_atm trm.inject alpha abs_fresh fin_supp abs_supp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7580 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7581 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7582 | case (ImpL e M' v M'' w) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7583 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7584 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7585 |     apply(subgoal_tac "\<exists>z'::name. z'\<sharp>(P,b,e,w,v,N,N{y:=<b>.P},M'{w:=<b>.P},M''{w:=<b>.P},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7586 |                   M'{w:=<b>.P}{a:=(x).N{w:=<b>.P}},M''{w:=<b>.P}{a:=(x).N{w:=<b>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7587 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7588 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7589 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7590 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7591 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7592 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7593 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7594 | apply(simp add: fresh_prod subst_fresh fresh_atm abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7595 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7596 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7597 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7598 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7599 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7600 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7601 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7602 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7603 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7604 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7605 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7606 | lemma subst_subst3: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7607 | assumes a: "a\<sharp>(P,N,c)" "c\<sharp>(M,N)" "x\<sharp>(y,P,M)" "y\<sharp>(P,x)" "M\<noteq>Ax y a" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7608 |   shows "N{x:=<a>.M}{y:=<c>.P} = N{y:=<c>.P}{x:=<a>.(M{y:=<c>.P})}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7609 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7610 | proof(nominal_induct N avoiding: x y a c M P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7611 | case (Ax z c) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7612 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7613 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7614 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7615 | case (Cut d M' u M'') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7616 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7617 | apply(simp add: fresh_atm fresh_prod trm.inject abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7618 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7619 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7620 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7621 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7622 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7623 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7624 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7625 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7626 | apply(subgoal_tac "P \<noteq> Ax x c") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7627 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7628 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7629 | apply(clarify) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7630 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7631 | apply(case_tac "x\<sharp>M'") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7632 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7633 | apply(simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7634 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7635 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7636 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7637 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7638 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7639 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7640 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7641 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7642 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7643 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7644 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7645 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7646 | apply(case_tac "y\<sharp>M'") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7647 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7648 | apply(simp add: not_Ax2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7649 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7650 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7651 | case NotR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7652 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7653 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7654 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7655 | case (NotL d M' u) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7656 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7657 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7658 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(y,P,M,M{y:=<c>.P},M'{x:=<a>.M},M'{y:=<c>.P}{x:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7659 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7660 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7661 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7662 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7663 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7664 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7665 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7666 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7667 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7668 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7669 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7670 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7671 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7672 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7673 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(x,y,P,M,M'{y:=<c>.P},M'{y:=<c>.P}{x:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7674 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7675 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7676 | apply(simp add: fresh_fun_simp_NotL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7677 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7678 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7679 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7680 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7681 | apply(simp add: fresh_atm subst_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7682 | apply(subgoal_tac "P \<noteq> Ax x c") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7683 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7684 | apply(simp add: forget trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7685 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7686 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7687 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7688 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7689 | apply(clarify) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7690 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7691 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7692 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7693 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7694 | case AndR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7695 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7696 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7697 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7698 | case (AndL1 u M' v) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7699 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7700 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7701 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(u,y,v,P,M,M{y:=<c>.P},M'{x:=<a>.M},M'{y:=<c>.P}{x:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7702 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7703 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7704 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7705 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7706 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7707 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7708 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7709 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7710 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7711 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7712 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7713 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7714 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7715 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7716 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(x,y,u,v,P,M,M'{y:=<c>.P},M'{y:=<c>.P}{x:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7717 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7718 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7719 | apply(simp add: fresh_fun_simp_AndL1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7720 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7721 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7722 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7723 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7724 | apply(simp add: fresh_atm subst_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7725 | apply(subgoal_tac "P \<noteq> Ax x c") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7726 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7727 | apply(simp add: forget trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7728 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7729 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7730 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7731 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7732 | apply(clarify) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7733 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7734 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7735 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7736 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7737 | case (AndL2 u M' v) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7738 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7739 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7740 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(u,y,v,P,M,M{y:=<c>.P},M'{x:=<a>.M},M'{y:=<c>.P}{x:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7741 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7742 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7743 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7744 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7745 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7746 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7747 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7748 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7749 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7750 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7751 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7752 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7753 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7754 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7755 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(x,y,u,v,P,M,M'{y:=<c>.P},M'{y:=<c>.P}{x:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7756 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7757 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7758 | apply(simp add: fresh_fun_simp_AndL2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7759 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7760 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7761 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7762 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7763 | apply(simp add: fresh_atm subst_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7764 | apply(subgoal_tac "P \<noteq> Ax x c") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7765 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7766 | apply(simp add: forget trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7767 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7768 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7769 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7770 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7771 | apply(clarify) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7772 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7773 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7774 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7775 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7776 | case OrR1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7777 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7778 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7779 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7780 | case OrR2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7781 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7782 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7783 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7784 | case (OrL x1 M' x2 M'' x3) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7785 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7786 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7787 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(y,P,M,M{y:=<c>.P},M'{x:=<a>.M},M'{y:=<c>.P}{x:=<a>.M{y:=<c>.P}},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7788 |                                       x1,x2,x3,M''{x:=<a>.M},M''{y:=<c>.P}{x:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7789 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7790 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7791 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7792 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7793 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7794 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7795 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7796 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7797 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7798 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7799 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7800 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7801 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7802 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7803 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7804 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7805 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(x,y,P,M,M'{y:=<c>.P},M'{y:=<c>.P}{x:=<a>.M{y:=<c>.P}},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7806 |                                       x1,x2,x3,M''{y:=<c>.P},M''{y:=<c>.P}{x:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7807 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7808 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7809 | apply(simp add: fresh_fun_simp_OrL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7810 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7811 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7812 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7813 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7814 | apply(simp add: fresh_atm subst_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7815 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7816 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7817 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7818 | apply(simp add: forget trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7819 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7820 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7821 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7822 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7823 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7824 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7825 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7826 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7827 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7828 | case ImpR | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7829 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7830 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7831 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7832 | case (ImpL d M' x1 M'' x2) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7833 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7834 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7835 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(y,P,M,M{y:=<c>.P},M'{x2:=<a>.M},M'{y:=<c>.P}{x2:=<a>.M{y:=<c>.P}},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7836 |                                       x1,x2,M''{x2:=<a>.M},M''{y:=<c>.P}{x2:=<a>.M{y:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7837 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7838 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7839 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7840 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7841 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7842 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7843 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7844 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7845 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7846 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7847 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7848 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7849 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7850 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7851 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7852 |     apply(subgoal_tac "\<exists>x'::name. x'\<sharp>(x,y,P,M,M'{x2:=<c>.P},M'{x2:=<c>.P}{x:=<a>.M{x2:=<c>.P}},
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7853 |                                       x1,x2,M''{x2:=<c>.P},M''{x2:=<c>.P}{x:=<a>.M{x2:=<c>.P}})")
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7854 | apply(erule exE, simp add: fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7855 | apply(erule conjE)+ | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7856 | apply(simp add: fresh_fun_simp_ImpL) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7857 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7858 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7859 | apply(rule better_Cut_substn) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7860 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7861 | apply(simp add: fresh_atm subst_fresh fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7862 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7863 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7864 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7865 | apply(simp add: forget trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7866 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7867 | apply(rule substn.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7868 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7869 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7870 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7871 | apply(rule exists_fresh'(1)[OF fs_name1]) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7872 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7873 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7874 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7875 | lemma subst_subst4: | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7876 | assumes a: "x\<sharp>(P,N,y)" "y\<sharp>(M,N)" "a\<sharp>(c,P,M)" "c\<sharp>(P,a)" "M\<noteq>Ax x c" | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7877 |   shows "N{a:=(x).M}{c:=(y).P} = N{c:=(y).P}{a:=(x).(M{c:=(y).P})}"
 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7878 | using a | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7879 | proof(nominal_induct N avoiding: x y a c M P rule: trm.strong_induct) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7880 | case (Ax z c) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7881 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7882 | by (auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7883 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7884 | case (Cut d M' u M'') | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7885 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7886 | apply(simp add: fresh_atm fresh_prod trm.inject abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7887 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7888 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7889 | apply(simp add: trm.inject) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7890 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7891 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7892 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7893 | apply(simp add: abs_fresh subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7894 | apply(simp add: fresh_prod subst_fresh abs_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7895 | apply(subgoal_tac "P \<noteq> Ax y a") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7896 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7897 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7898 | apply(clarify) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7899 | apply(simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7900 | apply(case_tac "a\<sharp>M''") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7901 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7902 | apply(simp add: not_Ax1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7903 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7904 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7905 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7906 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7907 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7908 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7909 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7910 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7911 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7912 | apply(simp add: fresh_prod subst_fresh fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7913 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7914 | apply(auto) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7915 | apply(case_tac "c\<sharp>M''") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7916 | apply(simp add: forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7917 | apply(simp add: not_Ax1) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7918 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7919 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7920 | case NotL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7921 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7922 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7923 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7924 | case (NotR u M' d) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7925 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7926 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7927 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7928 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7929 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7930 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7931 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7932 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7933 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7934 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7935 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7936 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7937 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7938 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7939 | apply(simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7940 | apply(auto simp add: fresh_atm fresh_prod)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7941 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7942 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7943 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7944 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7945 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7946 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7947 | apply(simp add: fresh_prod fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7948 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7949 | apply(auto simp add: fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7950 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7951 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7952 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7953 | apply(simp add: fresh_atm subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7954 | apply(auto simp add: fresh_prod fresh_atm) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7955 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7956 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7957 | case AndL1 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7958 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7959 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7960 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7961 | case AndL2 | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7962 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7963 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7964 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7965 | case (AndR d M e M' f) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7966 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7967 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7968 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7969 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7970 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7971 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7972 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7973 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7974 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7975 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7976 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7977 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7978 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7979 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7980 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7981 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7982 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7983 | apply(auto simp add: fresh_atm fresh_prod)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7984 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7985 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7986 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7987 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7988 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7989 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7990 | apply(simp add: subst_fresh fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7991 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7992 | apply(auto simp add: fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7993 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7994 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7995 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7996 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7997 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7998 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 7999 | apply(auto simp add: fresh_atm fresh_prod)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8000 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8001 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8002 | case OrL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8003 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8004 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8005 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8006 | case (OrR1 d M' e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8007 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8008 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8009 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8010 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8011 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8012 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8013 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8014 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8015 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8016 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8017 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8018 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8019 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8020 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8021 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8022 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8023 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8024 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8025 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8026 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8027 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8028 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8029 | apply(simp add: subst_fresh fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8030 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8031 | apply(auto simp add: fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8032 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8033 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8034 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8035 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8036 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8037 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8038 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8039 | case (OrR2 d M' e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8040 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8041 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8042 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8043 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8044 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8045 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8046 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8047 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8048 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8049 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8050 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8051 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8052 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8053 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8054 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8055 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8056 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8057 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8058 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8059 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8060 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8061 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8062 | apply(simp add: subst_fresh fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8063 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8064 | apply(auto simp add: fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8065 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8066 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8067 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8068 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8069 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8070 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8071 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8072 | case ImpL | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8073 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8074 | by(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8075 | next | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8076 | case (ImpR u d M' e) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8077 | then show ?case | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8078 | apply(auto simp add: subst_fresh abs_fresh fresh_atm fresh_prod forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8079 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8080 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8081 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8082 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8083 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8084 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8085 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8086 | apply(simp add: abs_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8087 | apply(simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8088 | apply(simp add: trm.inject alpha) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8089 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8090 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8091 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8092 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8093 | apply(auto simp add: fresh_prod fresh_atm subst_fresh abs_fresh abs_supp fin_supp)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8094 | apply(generate_fresh "coname") | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8095 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8096 | apply(fresh_fun_simp) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8097 | apply(rule sym) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8098 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8099 | apply(rule better_Cut_substc) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8100 | apply(simp add: subst_fresh fresh_atm fresh_prod) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8101 | apply(simp add: abs_fresh subst_fresh) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8102 | apply(auto simp add: fresh_atm)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8103 | apply(simp add: trm.inject alpha forget) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8104 | apply(rule trans) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8105 | apply(rule substc.simps) | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8106 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8107 | apply(auto simp add: fresh_prod fresh_atm subst_fresh)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8108 | apply(auto simp add: fresh_prod fresh_atm subst_fresh abs_fresh abs_supp fin_supp)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8109 | apply(auto simp add: fresh_prod fresh_atm subst_fresh abs_fresh abs_supp fin_supp)[1] | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8110 | done | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8111 | qed | 
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8112 | |
| 
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
 wenzelm parents: diff
changeset | 8113 | end |