]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/etc/lsx/lsx.etc
partial commit in basic_2
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / etc / lsx / lsx.etc
index b5407abdf26155c986321c697494929cb1775229..f09dc1da874da7a1eb8cb2d688b18167e716797b 100644 (file)
@@ -6,7 +6,7 @@ lemma lsx_lreq_conf: ∀h,o,G,L1,T,l. G ⊢ ⬊*[h, o, T, l] L1 →
 #L0 #HL03 #HL10 #H elim (H T) -H /4 width=4 by/
 qed-.
 
-(* these two are better expressed with the binder \chi *)
+(* this is better expressed with the binder \chi *)
 
 lemma lsx_fwd_bind_dx: ∀h,o,a,I,G,L,V,T,l. G ⊢ ⬈*[h, o, ⓑ{a,I}V.T, l] L →
                        G ⊢ ⬈*[h, o, T, ⫯l] L.ⓑ{I}V.
@@ -19,7 +19,3 @@ lemma lsx_fwd_bind_dx: ∀h,o,a,I,G,L,V,T,l. G ⊢ ⬈*[h, o, ⓑ{a,I}V.T, l] L
 @(lleq_lreq_trans … (L2.ⓑ{I}V1))
 /2 width=2 by lleq_fwd_bind_dx, lreq_succ/
 qed-.
-
-lemma lsx_inv_bind: ∀h,o,a,I,G,L,V,T,l. G ⊢ ⬈*[h, o, ⓑ{a, I}V.T, l] L →
-                    G ⊢ ⬈*[h, o, V, l] L ∧ G ⊢ ⬈*[h, o, T, ⫯l] L.ⓑ{I}V.
-/3 width=4 by lsx_fwd_bind_sn, lsx_fwd_bind_dx, conj/ qed-.