X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fground_2%2Frelocation%2Frtmap_uni.ma;h=fa8cf7ebfa3d955e47ad2e36d40c00f214feb4d8;hb=bd53c4e895203eb049e75434f638f26b5a161a2b;hp=247311b3ed0359a5f159effbfa052172383b960d;hpb=75f395f0febd02de8e0f881d918a8812b1425c8d;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_uni.ma b/matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_uni.ma index 247311b3e..fa8cf7ebf 100644 --- a/matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_uni.ma +++ b/matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_uni.ma @@ -20,7 +20,7 @@ include "ground_2/relocation/rtmap_isuni.ma". rec definition uni (n:nat) on n: rtmap ≝ match n with [ O ⇒ 𝐈𝐝 -| S n ⇒ ⫯(uni n) +| S n ⇒ ↑(uni n) ]. interpretation "uniform relocation (rtmap)" @@ -28,74 +28,74 @@ interpretation "uniform relocation (rtmap)" (* Basic properties *********************************************************) -lemma uni_zero: 𝐈𝐝 = 𝐔❴0❵. +lemma uni_zero: 𝐈𝐝 = 𝐔❨0❩. // qed. -lemma uni_succ: ∀n. ⫯𝐔❴n❵ = 𝐔❴⫯n❵. +lemma uni_succ: ∀n. ↑𝐔❨n❩ = 𝐔❨↑n❩. // qed. (* Basic inversion lemmas ***************************************************) -lemma uni_inv_push_dx: ∀f,n. 𝐔❴n❵ ≗ ↑f → 0 = n ∧ 𝐈𝐝 ≗ f. +lemma uni_inv_push_dx: ∀f,n. 𝐔❨n❩ ≡ ⫯f → 0 = n ∧ 𝐈𝐝 ≡ f. #f * /3 width=5 by eq_inv_pp, conj/ #n