]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/dynamic/lsubsv_lsuba.ma
lambdadelta
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / dynamic / lsubsv_lsuba.ma
index d19d320e4fcad2b510c1d2987ebbee0e8cc85fb1..d542b686bfe2c51d7eb2271e671dad3b0351bf9d 100644 (file)
@@ -18,8 +18,8 @@ include "basic_2/dynamic/lsubsv.ma".
 (* LOCAL ENVIRONMENT REFINEMENT FOR STRATIFIED NATIVE VALIDITY **************)
 
 (* Properties on local environment refinement for atomic arity assignment ***)
-
-lemma lsubsv_fwd_lsuba: ∀h,g,L1,L2. h ⊢ L1 ¡⊑[g] L2 → L1 ⁝⊑ L2.
+(*
+lamma lsubsv_fwd_lsuba: ∀h,g,L1,L2. h ⊢ L1 ¡⊑[g] L2 → L1 ⁝⊑ L2.
 #h #g #L1 #L2 #H elim H -L1 -L2 // /2 width=1/
 #L1 #L2 #V1 #V2 #W1 #W2 #l #HV1 #HVW1 #HW12 #HW2 #_ #_ #HL12
 elim (snv_fwd_aaa … HV1) -HV1 #A #HV1
@@ -28,3 +28,4 @@ lapply (ssta_aaa … HV1 … HVW1) -HVW1 #H1
 lapply (lsuba_aaa_trans … HW2 … HL12) #H2
 lapply (aaa_cpcs_mono … HW12 … H1 … H2) -W1 -H2 #H destruct /2 width=3/
 qed-.
+*)