X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambda-delta%2FBasic-2%2Freduction%2Fcpr_cpr.ma;h=08620900765d54f2097db20b105bd7d17ae9a78f;hb=95fe49b9bd546ee4f0d27dce7267d7285eb81b01;hp=d544918acc0e6dc2267619da5a948581b3a4c9fd;hpb=b4240d93f7fd4c3e60d3495dc558edfc0e0f48e7;p=helm.git diff --git a/matita/matita/contribs/lambda-delta/Basic-2/reduction/cpr_cpr.ma b/matita/matita/contribs/lambda-delta/Basic-2/reduction/cpr_cpr.ma index d544918ac..086209007 100644 --- a/matita/matita/contribs/lambda-delta/Basic-2/reduction/cpr_cpr.ma +++ b/matita/matita/contribs/lambda-delta/Basic-2/reduction/cpr_cpr.ma @@ -17,12 +17,42 @@ include "Basic-2/reduction/cpr.ma". (* CONTEXT-SENSITIVE PARALLEL REDUCTION ON TERMS ****************************) +(* Advanced properties ******************************************************) + +lemma cpr_bind_sn: ∀I,L,V1,V2,T1,T2. L ⊢ V1 ⇒ V2 → T1 ⇒ T2 → + L ⊢ 𝕓{I} V1. T1 ⇒ 𝕓{I} V2. T2. +#I #L #V1 #V2 #T1 #T2 * #V #HV1 #HV2 #HT12 +@ex2_1_intro [2: @(tpr_delta … HV1 HT12) | skip ] /2/ (* /3 width=5/ is too slow *) +qed. + +(* Basic-1: was only: pr2_gen_cbind *) +lemma cpr_bind_dx: ∀I,L,V1,V2,T1,T2. V1 ⇒ V2 → L. 𝕓{I} V2 ⊢ T1 ⇒ T2 → + L ⊢ 𝕓{I} V1. T1 ⇒ 𝕓{I} V2. T2. +#I #L #V1 #V2 #T1 #T2 #HV12 * #T #HT1 normalize #HT2 +elim (tpss_split_up … HT2 1 ? ?) -HT2 // #T0