X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambda_delta%2FBasic_2%2Freducibility%2Fltpr.ma;h=8e834b2dadaae3d79d6c4ce3961ddcae716fcb85;hb=48b202cd4ccd3ffc10f9a134314f747fdee30d36;hp=2208557a7c188c950b6d651008fe637a8f36d0a0;hpb=04cd2181640b3828b3d193a8e819c849ef574236;p=helm.git diff --git a/matita/matita/contribs/lambda_delta/Basic_2/reducibility/ltpr.ma b/matita/matita/contribs/lambda_delta/Basic_2/reducibility/ltpr.ma index 2208557a7..8e834b2da 100644 --- a/matita/matita/contribs/lambda_delta/Basic_2/reducibility/ltpr.ma +++ b/matita/matita/contribs/lambda_delta/Basic_2/reducibility/ltpr.ma @@ -19,7 +19,7 @@ include "Basic_2/reducibility/tpr.ma". inductive ltpr: relation lenv ≝ | ltpr_stom: ltpr (⋆) (⋆) | ltpr_pair: ∀K1,K2,I,V1,V2. - ltpr K1 K2 → V1 ⇒ V2 → ltpr (K1. 𝕓{I} V1) (K2. 𝕓{I} V2) (*𝕓*) + ltpr K1 K2 → V1 ➡ V2 → ltpr (K1. ⓑ{I} V1) (K2. ⓑ{I} V2) (*ⓑ*) . interpretation @@ -28,13 +28,13 @@ interpretation (* Basic properties *********************************************************) -lemma ltpr_refl: ∀L:lenv. L ⇒ L. +lemma ltpr_refl: ∀L:lenv. L ➡ L. #L elim L -L // /2 width=1/ qed. (* Basic inversion lemmas ***************************************************) -fact ltpr_inv_atom1_aux: ∀L1,L2. L1 ⇒ L2 → L1 = ⋆ → L2 = ⋆. +fact ltpr_inv_atom1_aux: ∀L1,L2. L1 ➡ L2 → L1 = ⋆ → L2 = ⋆. #L1 #L2 * -L1 -L2 [ // | #K1 #K2 #I #V1 #V2 #_ #_ #H destruct @@ -42,11 +42,11 @@ fact ltpr_inv_atom1_aux: ∀L1,L2. L1 ⇒ L2 → L1 = ⋆ → L2 = ⋆. qed. (* Basic_1: was: wcpr0_gen_sort *) -lemma ltpr_inv_atom1: ∀L2. ⋆ ⇒ L2 → L2 = ⋆. +lemma ltpr_inv_atom1: ∀L2. ⋆ ➡ L2 → L2 = ⋆. /2 width=3/ qed-. -fact ltpr_inv_pair1_aux: ∀L1,L2. L1 ⇒ L2 → ∀K1,I,V1. L1 = K1. 𝕓{I} V1 → - ∃∃K2,V2. K1 ⇒ K2 & V1 ⇒ V2 & L2 = K2. 𝕓{I} V2. +fact ltpr_inv_pair1_aux: ∀L1,L2. L1 ➡ L2 → ∀K1,I,V1. L1 = K1. ⓑ{I} V1 → + ∃∃K2,V2. K1 ➡ K2 & V1 ➡ V2 & L2 = K2. ⓑ{I} V2. #L1 #L2 * -L1 -L2 [ #K1 #I #V1 #H destruct | #K1 #K2 #I #V1 #V2 #HK12 #HV12 #L #J #W #H destruct /2 width=5/ @@ -54,35 +54,35 @@ fact ltpr_inv_pair1_aux: ∀L1,L2. L1 ⇒ L2 → ∀K1,I,V1. L1 = K1. 𝕓{I} V1 qed. (* Basic_1: was: wcpr0_gen_head *) -lemma ltpr_inv_pair1: ∀K1,I,V1,L2. K1. 𝕓{I} V1 ⇒ L2 → - ∃∃K2,V2. K1 ⇒ K2 & V1 ⇒ V2 & L2 = K2. 𝕓{I} V2. +lemma ltpr_inv_pair1: ∀K1,I,V1,L2. K1. ⓑ{I} V1 ➡ L2 → + ∃∃K2,V2. K1 ➡ K2 & V1 ➡ V2 & L2 = K2. ⓑ{I} V2. /2 width=3/ qed-. -fact ltpr_inv_atom2_aux: ∀L1,L2. L1 ⇒ L2 → L2 = ⋆ → L1 = ⋆. +fact ltpr_inv_atom2_aux: ∀L1,L2. L1 ➡ L2 → L2 = ⋆ → L1 = ⋆. #L1 #L2 * -L1 -L2 [ // | #K1 #K2 #I #V1 #V2 #_ #_ #H destruct ] qed. -lemma ltpr_inv_atom2: ∀L1. L1 ⇒ ⋆ → L1 = ⋆. +lemma ltpr_inv_atom2: ∀L1. L1 ➡ ⋆ → L1 = ⋆. /2 width=3/ qed-. -fact ltpr_inv_pair2_aux: ∀L1,L2. L1 ⇒ L2 → ∀K2,I,V2. L2 = K2. 𝕓{I} V2 → - ∃∃K1,V1. K1 ⇒ K2 & V1 ⇒ V2 & L1 = K1. 𝕓{I} V1. +fact ltpr_inv_pair2_aux: ∀L1,L2. L1 ➡ L2 → ∀K2,I,V2. L2 = K2. ⓑ{I} V2 → + ∃∃K1,V1. K1 ➡ K2 & V1 ➡ V2 & L1 = K1. ⓑ{I} V1. #L1 #L2 * -L1 -L2 [ #K2 #I #V2 #H destruct | #K1 #K2 #I #V1 #V2 #HK12 #HV12 #K #J #W #H destruct /2 width=5/ ] qed. -lemma ltpr_inv_pair2: ∀L1,K2,I,V2. L1 ⇒ K2. 𝕓{I} V2 → - ∃∃K1,V1. K1 ⇒ K2 & V1 ⇒ V2 & L1 = K1. 𝕓{I} V1. +lemma ltpr_inv_pair2: ∀L1,K2,I,V2. L1 ➡ K2. ⓑ{I} V2 → + ∃∃K1,V1. K1 ➡ K2 & V1 ➡ V2 & L1 = K1. ⓑ{I} V1. /2 width=3/ qed-. (* Basic forward lemmas *****************************************************) -lemma ltpr_fwd_length: ∀L1,L2. L1 ⇒ L2 → |L1| = |L2|. +lemma ltpr_fwd_length: ∀L1,L2. L1 ➡ L2 → |L1| = |L2|. #L1 #L2 #H elim H -L1 -L2 normalize // qed-.