]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/Basic_2/substitution/ltps.ma
- the relocation properties of cpr are closed!
[helm.git] / matita / matita / contribs / lambda_delta / Basic_2 / substitution / ltps.ma
index 3982ed2f9be3b96431bc73d64afc64584f808bf4..06201e8e521564f74ea5f617a06b41a3deeb6c77 100644 (file)
 (*                                                                        *)
 (**************************************************************************)
 
-include "Basic-2/substitution/tps.ma".
+include "Basic_2/substitution/tps.ma".
 
 (* PARALLEL SUBSTITUTION ON LOCAL ENVIRONMENTS ******************************)
 
-(* Basic-1: includes: csubst1_bind *)
+(* Basic_1: includes: csubst1_bind *)
 inductive ltps: nat → nat → relation lenv ≝
 | ltps_atom: ∀d,e. ltps d e (⋆) (⋆)
 | ltps_pair: ∀L,I,V. ltps 0 0 (L. 𝕓{I} V) (L. 𝕓{I} V)
@@ -47,7 +47,7 @@ lemma ltps_tps1_lt: ∀L1,L2,I,V1,V2,d,e.
 >(plus_minus_m_m d 1) /2/
 qed.
 
-(* Basic-1: was by definition: csubst1_refl *)
+(* Basic_1: was by definition: csubst1_refl *)
 lemma ltps_refl: ∀L,d,e. L [d, e] ≫ L.
 #L elim L -L //
 #L #I #V #IHL * /2/ * /2/
@@ -169,10 +169,10 @@ lemma ltps_inv_tps12: ∀L1,K2,I,V2,d,e. L1 [d, e] ≫ K2. 𝕓{I} V2 → 0 < d
                                   L1 = K1. 𝕓{I} V1.
 /2/ qed.
 
-(* Basic-1: removed theorems 27:
-            csubst0_clear_O csubst0_drop_lt csubst0_drop_gt csubst0_drop_eq
+(* Basic_1: removed theorems 27:
+            csubst0_clear_O csubst0_ldrop_lt csubst0_ldrop_gt csubst0_ldrop_eq
             csubst0_clear_O_back csubst0_clear_S csubst0_clear_trans
-            csubst0_drop_gt_back csubst0_drop_eq_back csubst0_drop_lt_back
+            csubst0_ldrop_gt_back csubst0_ldrop_eq_back csubst0_ldrop_lt_back
             csubst0_gen_sort csubst0_gen_head csubst0_getl_ge csubst0_getl_lt
             csubst0_gen_S_bind_2 csubst0_getl_ge_back csubst0_getl_lt_back
             csubst0_snd_bind csubst0_fst_bind csubst0_both_bind