]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/computation/dxprs_lift.ma
- lambdadelta: last recursive part of preservation finally proved!
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / computation / dxprs_lift.ma
index 628563cf416aa2cb160d9bc1bb5d3c0befb36ddc..eaa73f3454ae812e86b324c09d2523e9c1ac739b 100644 (file)
@@ -30,7 +30,7 @@ qed-.
 
 (* Advanced properties ******************************************************)
 
-lemma ssta_cprs_dxprs: ∀h,g,L,T1,T,T2,l. ⦃h, L⦄ ⊢ T1 •[g, l+1] T →
+lemma ssta_cprs_dxprs: ∀h,g,L,T1,T,T2,l. ⦃h, L⦄ ⊢ T1 •[g] ⦃l+1, T⦄ →
                        L ⊢ T ➡* T2 → ⦃h, L⦄ ⊢ T1 •*➡*[g] T2.
 /3 width=3/ qed.