]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/unfold/sstas_aaa.ma
partial commit: just the components before "static" ...
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / unfold / sstas_aaa.ma
index 36951ce083cc0c41f15897ffe5ba7b10533debe3..b369caa723559093d5bc85d777db561d8331bf4c 100644 (file)
@@ -19,7 +19,7 @@ include "basic_2/unfold/sstas.ma".
 
 (* Properties on atomic arity assignment for terms **************************)
 
-lemma sstas_aaa: ∀h,g,L,T,U. ⦃h, L⦄ ⊢ T •*[g] U →
-                 ∀A. L ⊢ T ⁝ A → L ⊢ U ⁝ A.
+lemma sstas_aaa: ∀h,g,L,T,U. ⦃G, L⦄ ⊢ T •*[h, g] U →
+                 ∀A. ⦃G, L⦄ ⊢ T ⁝ A → ⦃G, L⦄ ⊢ U ⁝ A.
 #h #g #L #T #U #H @(sstas_ind_dx … H) -T // /3 width=6/
 qed.