]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/dynamic/lsubsv_lsubd.ma
some renaming and some typos corrected ...
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / dynamic / lsubsv_lsubd.ma
index 86007b1f5cdbe9e32ec3947f3617005f8ded70e1..b7eac381af2b3c2a55ba02b3100e4f6e8aefe05c 100644 (file)
@@ -19,6 +19,6 @@ include "basic_2/dynamic/lsubsv.ma".
 
 (* Forward lemmas on lenv refinement for degree assignment ******************)
 
-lemma lsubsv_fwd_lsubd: ∀h,g,G,L1,L2. G ⊢ L1 ¡⫃[h, g] L2 → G ⊢ L1 ▪⫃[h, g] L2.
+lemma lsubsv_fwd_lsubd: ∀h,g,G,L1,L2. G ⊢ L1 ⫃¡[h, g] L2 → G ⊢ L1 ⫃▪[h, g] L2.
 #h #g #G #L1 #L2 #H elim H -L1 -L2 // /2 width=1/ /2 width=3/
 qed-.