]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/reduction/cpr.ma
- lsubr moved down one component
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / reduction / cpr.ma
index 28b040bf8dd9f5f63736d2868063e7b0e1a4f74d..3c0514a3c7a876b4ca2c0f1a305b54d837e3f621 100644 (file)
@@ -16,7 +16,7 @@ include "basic_2/notation/relations/pred_4.ma".
 include "basic_2/grammar/genv.ma".
 include "basic_2/grammar/cl_shift.ma".
 include "basic_2/relocation/ldrop_append.ma".
-include "basic_2/substitution/lsubr.ma".
+include "basic_2/relocation/lsubr.ma".
 
 (* CONTEXT-SENSITIVE PARALLEL REDUCTION FOR TERMS ***************************)
 
@@ -286,7 +286,7 @@ lemma cpr_fwd_bind1_minus: ∀I,G,L,V1,T1,T. ⦃G, L⦄ ⊢ -ⓑ{I}V1.T1 ➡ T 
 #I #G #L #V1 #T1 #T #H #b
 elim (cpr_inv_bind1 … H) -H *
 [ #V2 #T2 #HV12 #HT12 #H destruct /3 width=4/
-| #T2 #_ #_ #H destruct 
+| #T2 #_ #_ #H destruct
 ]
 qed-.