]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/basic_2/static/lsuba_aaa.ma
- we introduced the pointer_step rc in the perspective of proving
[helm.git] / matita / matita / contribs / lambda_delta / basic_2 / static / lsuba_aaa.ma
index a6a9c3fae26656c3c8fc963b26b0b888915ee2d1..66e802aaed6e8348ef63c69c2deba38a170b267a 100644 (file)
 (*                                                                        *)
 (**************************************************************************)
 
-include "Basic_2/static/aaa_aaa.ma".
-include "Basic_2/static/lsuba_ldrop.ma".
+include "basic_2/static/aaa_aaa.ma".
+include "basic_2/static/lsuba_ldrop.ma".
 
 (* LOCAL ENVIRONMENT REFINEMENT FOR ATOMIC ARITY ASSIGNMENT *****************)
 
 (* Properties concerning atomic arity assignment ****************************)
 
-lemma lsuba_aaa_conf: ∀L1,V,A. L1 ⊢ V ÷ A → ∀L2. L1 ÷⊑ L2 → L2 ⊢ V ÷ A.
+lemma lsuba_aaa_conf: ∀L1,V,A. L1 ⊢ V ⁝ A → ∀L2. L1 ⁝⊑ L2 → L2 ⊢ V ⁝ A.
 #L1 #V #A #H elim H -L1 -V -A
 [ //
 | #I #L1 #K1 #V1 #B #i #HLK1 #HV1B #IHV1 #L2 #HL12
@@ -36,7 +36,7 @@ lemma lsuba_aaa_conf: ∀L1,V,A. L1 ⊢ V ÷ A → ∀L2. L1 ÷⊑ L2 → L2 ⊢
 ]
 qed.
 
-lemma lsuba_aaa_trans: ∀L2,V,A. L2 ⊢ V ÷ A → ∀L1. L1 ÷⊑ L2 → L1 ⊢ V ÷ A.
+lemma lsuba_aaa_trans: ∀L2,V,A. L2 ⊢ V ⁝ A → ∀L1. L1 ⁝⊑ L2 → L1 ⊢ V ⁝ A.
 #L2 #V #A #H elim H -L2 -V -A
 [ //
 | #I #L2 #K2 #V2 #B #i #HLK2 #HV2B #IHV2 #L1 #HL12