X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambda_delta%2Fbasic_2%2Fcomputation%2Flcprs.ma;fp=matita%2Fmatita%2Fcontribs%2Flambda_delta%2Fbasic_2%2Fcomputation%2Flcprs.ma;h=0000000000000000000000000000000000000000;hb=7bedf1797ba168f0742194b2add69575e5d4a5cd;hp=7661358dc1083a8afc8eac93d38ff3bbd673ed5c;hpb=3ca25660341410dd0f8694e6863c7c16f4e912a7;p=helm.git diff --git a/matita/matita/contribs/lambda_delta/basic_2/computation/lcprs.ma b/matita/matita/contribs/lambda_delta/basic_2/computation/lcprs.ma deleted file mode 100644 index 7661358dc..000000000 --- a/matita/matita/contribs/lambda_delta/basic_2/computation/lcprs.ma +++ /dev/null @@ -1,52 +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/reducibility/lcpr.ma". - -(* CONTEXT-SENSITIVE PARALLEL COMPUTATION ON LOCAL ENVIRONMENTS *************) - -definition lcprs: relation lenv ≝ TC … lcpr. - -interpretation - "context-sensitive parallel computation (environment)" - 'CPRedStar L1 L2 = (lcprs L1 L2). - -(* Basic eliminators ********************************************************) - -lemma lcprs_ind: ∀L1. ∀R:predicate lenv. R L1 → - (∀L,L2. L1 ⊢ ➡* L → L ⊢ ➡ L2 → R L → R L2) → - ∀L2. L1 ⊢ ➡* L2 → R L2. -#L1 #R #HL1 #IHL1 #L2 #HL12 -@(TC_star_ind … HL1 IHL1 … HL12) // -qed-. - -lemma lcprs_ind_dx: ∀L2. ∀R:predicate lenv. R L2 → - (∀L1,L. L1 ⊢ ➡ L → L ⊢ ➡* L2 → R L → R L1) → - ∀L1. L1 ⊢ ➡* L2 → R L1. -#L2 #R #HL2 #IHL2 #L1 #HL12 -@(TC_star_ind_dx … HL2 IHL2 … HL12) // -qed-. - -(* Basic properties *********************************************************) - -lemma lcprs_refl: ∀L. L ⊢ ➡* L. -/2 width=1/ qed. - -lemma lcprs_strap1: ∀L1,L,L2. - L1 ⊢ ➡* L → L ⊢ ➡ L2 → L1 ⊢ ➡* L2. -/2 width=3/ qed. - -lemma lcprs_strap2: ∀L1,L,L2. - L1 ⊢ ➡ L → L ⊢ ➡* L2 → L1 ⊢ ➡* L2. -/2 width=3/ qed.