From: Ferruccio Guidi Date: Wed, 10 Aug 2011 11:13:18 +0000 (+0000) Subject: some refactoring X-Git-Tag: make_still_working~2339 X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=commitdiff_plain;ds=sidebyside;h=14fef03bcc79583593a129bf9c68bdf690a10eb7;p=helm.git some refactoring --- diff --git a/matita/matita/lib/lambda-delta/ground.ma b/matita/matita/lib/lambda-delta/ground.ma index e09e7d47a..ed5876107 100644 --- a/matita/matita/lib/lambda-delta/ground.ma +++ b/matita/matita/lib/lambda-delta/ground.ma @@ -144,6 +144,9 @@ lemma arith_h1: ∀a1,a2,b,c1. c1 ≤ a1 → c1 ≤ b → #a1 #a2 #b #c1 #H1 #H2 arith6 // #HU2 - @pr_delta [4,5,6: /2/ |1,2,3: skip ] (**) (* /2/ *) -| #L #i #d #e #Hdei #X #HX - lapply (lift_inv_lref1_ge … HX ?) -HX /2/ #HX destruct -X; - >arith7 /2/ -| #L #I #V1 #V2 #T1 #T2 #d #e #_ #_ #IHV12 #IHT12 #X #HX - elim (lift_inv_bind1 … HX) -HX #V #T #HV2 #HT2 #HX destruct -X /3/ -| #L #I #V1 #V2 #T1 #T2 #d #e #_ #_ #IHV12 #IHT12 #X #HX - elim (lift_inv_flat1 … HX) -HX #V #T #HV2 #HT2 #HX destruct -X /3/ -] -qed. -(* -lemma pr_subst_pr: ∀L,T1,T. L ⊢ T1 ⇒ T → ∀d,e,U. L ⊢ ↓[d,e] T ≡ U → - ∀T2. ↑[d,e] U ≡ T2 → L ⊢ T1 ⇒ T2. -#L #T1 #T #H elim H -H L T1 T -[ /2 width=5/ -| /2 width=5/ -| #L #I #V1 #V2 #T1 #T2 #HV12 #HT12 #IHV12 #IHT12 #d #e #X2 #HX2 #X1 #HX1 - elim (subst_inv_bind1 … HX2) -HX2 #V3 #T3 #HV23 #HT23 #H destruct -X2; - elim (lift_inv_bind1 … HX1) -HX1 #V4 #T4 #HV34 #HT34 #H destruct -X1; - @pr_bind /2 width=5/ @IHT12 -| #L #I #V1 #V2 #T1 #T2 #_ #_ #IHV12 #IHT12 #d #e #X2 #HX2 #X1 #HX1 - elim (subst_inv_flat1 … HX2) -HX2 #V3 #T3 #HV23 #HT23 #H destruct -X2; - elim (lift_inv_flat1 … HX1) -HX1 #V4 #T4 #HV34 #HT34 #H destruct -X1; - /3 width=5/ -| #L #V1 #V2 #W #T1 #T2 #_ #_ #IHV12 #IHT12 #d #e #X2 #HX2 #X1 #HX1 - elim (subst_inv_bind1 … HX2) -HX2 #V3 #T3 #HV23 #HT23 #H destruct -X2; - elim (lift_inv_bind1 … HX1) -HX1 #V4 #T4 #HV34 #HT34 #H destruct -X1; - @pr_beta /2 width=5/ @IHT12 -| #L #K #V1 #V2 #V #i #HLK #HV12 #HV2 #IHV12 #d #e #U #HVU #U0 #HU0 - lapply (lift_free … HU0 0 (i + 1 + e) ? ? ?) // - - - @pr_delta [4: // |1,2: skip |6: -*) diff --git a/matita/matita/lib/lambda-delta/substitution/tps_tps.ma b/matita/matita/lib/lambda-delta/substitution/tps_tps.ma index 8d801d50e..c1faa23f4 100644 --- a/matita/matita/lib/lambda-delta/substitution/tps_tps.ma +++ b/matita/matita/lib/lambda-delta/substitution/tps_tps.ma @@ -11,9 +11,6 @@ include "lambda-delta/substitution/tps_split.ma". -lemma arith_i2: ∀a,c1,c2. c1 + c2 ≤ a → c1 + c2 + (a - c1 - c2) = a. -/2/ qed. - (* PARTIAL SUBSTITUTION ON TERMS ********************************************) (* Main properties **********************************************************)