X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambda_delta%2Fbasic_2%2Fgrammar%2Fcl_weight.ma;h=478911825ae6aa046b402a77ba6f4f3c3cc42cca;hb=53f874fba5b9c39a788085515a4fefe5d29281da;hp=40a364a44124ccf03c9f38d01074936252ec3465;hpb=f7386d0b74f935f07ede4be46d0489a233d68b85;p=helm.git diff --git a/matita/matita/contribs/lambda_delta/basic_2/grammar/cl_weight.ma b/matita/matita/contribs/lambda_delta/basic_2/grammar/cl_weight.ma index 40a364a44..478911825 100644 --- a/matita/matita/contribs/lambda_delta/basic_2/grammar/cl_weight.ma +++ b/matita/matita/contribs/lambda_delta/basic_2/grammar/cl_weight.ma @@ -17,21 +17,21 @@ include "basic_2/grammar/cl_shift.ma". (* WEIGHT OF A CLOSURE ******************************************************) -definition cw: lenv → term → ? ≝ λL,T. #{L} + #{T}. +definition fw: lenv → term → ? ≝ λL,T. #{L} + #{T}. -interpretation "weight (closure)" 'Weight L T = (cw L T). +interpretation "weight (closure)" 'Weight L T = (fw L T). (* Basic properties *********************************************************) (* Basic_1: was: flt_wf__q_ind *) (* Basic_1: was: flt_wf_ind *) -axiom cw_wf_ind: ∀R:lenv→predicate term. - (∀L2,T2. (∀L1,T1. #{L1,T1} < #{L2,T2} → R L1 T1) → R L2 T2) → - ∀L,T. R L T. +axiom fw_ind: ∀R:relation2 lenv term. + (∀L2,T2. (∀L1,T1. #{L1,T1} < #{L2,T2} → R L1 T1) → R L2 T2) → + ∀L,T. R L T. (* Basic_1: was: flt_shift *) -lemma cw_shift: ∀a,K,I,V,T. #{K. ⓑ{I} V, T} < #{K, ⓑ{a,I} V. T}. +lemma fw_shift: ∀a,K,I,V,T. #{K. ⓑ{I} V, T} < #{K, ⓑ{a,I} V. T}. normalize // qed. @@ -41,19 +41,19 @@ lemma tw_shift: ∀L,T. #{L, T} ≤ #{L @@ T}. @transitive_le [3: @IHL |2: /2 width=2/ | skip ] qed. -lemma cw_tpair_sn: ∀I,L,V,T. #{L, V} < #{L, ②{I}V.T}. +lemma fw_tpair_sn: ∀I,L,V,T. #{L, V} < #{L, ②{I}V.T}. #I #L #V #T normalize in ⊢ (? % %); // qed. -lemma cw_tpair_dx: ∀I,L,V,T. #{L, T} < #{L, ②{I}V.T}. +lemma fw_tpair_dx: ∀I,L,V,T. #{L, T} < #{L, ②{I}V.T}. #I #L #V #T normalize in ⊢ (? % %); // qed. -lemma cw_tpair_dx_sn: ∀I1,I2,L,V1,V2,T. #{L, V2} < #{L, ②{I1}V1.②{I2}V2.T}. +lemma fw_tpair_dx_sn: ∀I1,I2,L,V1,V2,T. #{L, V2} < #{L, ②{I1}V1.②{I2}V2.T}. #I1 #I2 #L #V1 #V2 #T normalize in ⊢ (? % %); /2 width=1/ qed. -lemma cw_tpair_dx_sn_shift: ∀a2,I1,I2,L,V1,V2,T. +lemma fw_tpair_dx_sn_shift: ∀a2,I1,I2,L,V1,V2,T. #{L.ⓑ{I2}V2, T} < #{L, ②{I1}V1.ⓑ{a2,I2}V2.T}. #a2 #I1 #I2 #L #V1 #V2 #T normalize in ⊢ (? % %); /2 width=1/ qed.