X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambda_delta%2FBasic_2%2Fcomputation%2Fcsn_vector.ma;fp=matita%2Fmatita%2Fcontribs%2Flambda_delta%2FBasic_2%2Fcomputation%2Fcsn_vector.ma;h=0000000000000000000000000000000000000000;hb=eb918fc784eacd2094e3986ba321ef47690d9983;hp=bddaaa89de3028d51c17d46f3910054d6a18c488;hpb=011cf6478141e69822a5b40933f2444d0522532f;p=helm.git diff --git a/matita/matita/contribs/lambda_delta/Basic_2/computation/csn_vector.ma b/matita/matita/contribs/lambda_delta/Basic_2/computation/csn_vector.ma deleted file mode 100644 index bddaaa89d..000000000 --- a/matita/matita/contribs/lambda_delta/Basic_2/computation/csn_vector.ma +++ /dev/null @@ -1,50 +0,0 @@ -(**************************************************************************) -(* ___ *) -(* ||M|| *) -(* ||A|| A project by Andrea Asperti *) -(* ||T|| *) -(* ||I|| Developers: *) -(* ||T|| The HELM team. *) -(* ||A|| http://helm.cs.unibo.it *) -(* \ / *) -(* \ / This file is distributed under the terms of the *) -(* v GNU General Public License Version 2 *) -(* *) -(**************************************************************************) - -include "Basic_2/grammar/term_vector.ma". -include "Basic_2/computation/csn.ma". - -(* CONTEXT-SENSITIVE STRONGLY NORMALIZING TERM VECTORS **********************) - -inductive csnv (L:lenv): predicate (list term) ≝ -| csnv_nil: csnv L ◊ -| csn_cons: ∀Ts,T. L ⊢ ⬇* T → csnv L Ts → csnv L (T :: Ts) -. - -interpretation - "context-sensitive strong normalization (term vector)" - 'SN L Ts = (csnv L Ts). - -(* Basic inversion lemmas ***************************************************) - -fact csnv_inv_cons_aux: ∀L,Ts. L ⊢ ⬇* Ts → ∀U,Us. Ts = U :: Us → - L ⊢ ⬇* U ∧ L ⊢ ⬇* Us. -#L #Ts * -Ts -[ #U #Us #H destruct -| #Ts #T #HT #HTs #U #Us #H destruct /2 width=1/ -] -qed. - -lemma csnv_inv_cons: ∀L,T,Ts. L ⊢ ⬇* T :: Ts → L ⊢ ⬇* T ∧ L ⊢ ⬇* Ts. -/2 width=3/ qed-. - -include "Basic_2/computation/csn_cpr.ma". - -lemma csn_fwd_applv: ∀L,T,Vs. L ⊢ ⬇* Ⓐ Vs. T → L ⊢ ⬇* Vs ∧ L ⊢ ⬇* T. -#L #T #Vs elim Vs -Vs /2 width=1/ -#V #Vs #IHVs #HVs -lapply (csn_fwd_pair_sn … HVs) #HV -lapply (csn_fwd_flat_dx … HVs) -HVs #HVs -elim (IHVs HVs) -IHVs -HVs /3 width=1/ -qed-.