X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Frelocation%2Fdrops_vector.ma;h=66bfbcfd6979924f7085810a0873fe90e40018a9;hb=e9da8e091898b6e67a2f270581bdc5cdbe80e9b0;hp=f76942c5d911328a6f7f5d287cd070d87b13ecae;hpb=3a430d712f9d87185e9271b7b0c5188c5f311e4b;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2/relocation/drops_vector.ma b/matita/matita/contribs/lambdadelta/basic_2/relocation/drops_vector.ma index f76942c5d..66bfbcfd6 100644 --- a/matita/matita/contribs/lambdadelta/basic_2/relocation/drops_vector.ma +++ b/matita/matita/contribs/lambdadelta/basic_2/relocation/drops_vector.ma @@ -18,14 +18,14 @@ include "basic_2/relocation/drops.ma". (* GENERIC SLICING FOR LOCAL ENVIRONMENTS ***********************************) definition d_liftable1_all: relation2 lenv term → predicate bool ≝ - λR,c. ∀L,K,f. ⬇*[c, f] L ≡ K → + λR,b. ∀f,L,K. ⬇*[b, f] L ≡ K → ∀Ts,Us. ⬆*[f] Ts ≡ Us → all … (R K) Ts → all … (R L) Us. (* Properties with generic relocation for term vectors **********************) (* Basic_2A1: was: d1_liftables_liftables_all *) -lemma d1_liftable_liftable_all: ∀R,c. d_liftable1 R c → d_liftable1_all R c. -#R #c #HR #L #K #f #HLK #Ts #Us #H elim H -Ts -Us normalize // +lemma d1_liftable_liftable_all: ∀R,b. d_liftable1 R b → d_liftable1_all R b. +#R #b #HR #f #L #K #HLK #Ts #Us #H elim H -Ts -Us normalize // #Ts #Us #T #U #HTU #_ #IHTUs * /3 width=7 by conj/ qed.