]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_tls.ma
frees_drops completed!
[helm.git] / matita / matita / contribs / lambdadelta / ground_2 / relocation / rtmap_tls.ma
index 11a0c9092b8799ca03c5e9db7cc930fac6dc54c8..dc277016d988cc390f35a700322d37d2dfd8f4c3 100644 (file)
@@ -13,6 +13,7 @@
 (**************************************************************************)
 
 include "ground_2/notation/functions/droppreds_2.ma".
+include "ground_2/relocation/rtmap_pushs.ma".
 include "ground_2/relocation/rtmap_tl.ma".
 
 (* RELOCATION MAP ***********************************************************)
@@ -24,18 +25,25 @@ interpretation "tls (rtmap)" 'DropPreds n f = (tls f n).
 
 (* Basic properties *********************************************************)
 
-lemma tls_rew_O: ∀f. f = ⫱*[0] f.
+lemma tls_O: ∀f. f = ⫱*[0] f.
 // qed.
 
-lemma tls_rew_S: ∀f,n. ⫱ ⫱*[n] f = ⫱*[⫯n] f.
+lemma tls_S: ∀f,n. ⫱ ⫱*[n] f = ⫱*[⫯n] f.
 // qed.
 
 lemma tls_eq_repl: ∀n. eq_repl (λf1,f2. ⫱*[n] f1 ≗ ⫱*[n] f2).
 #n elim n -n /3 width=1 by tl_eq_repl/
 qed.
 
-(* Advancedd properties *****************************************************)
+(* Advanced properties ******************************************************)
 
 lemma tls_xn: ∀n,f. ⫱*[n] ⫱f = ⫱*[⫯n] f.
 #n elim n -n //
 qed.
+
+(* Properties with pushs ****************************************************)
+
+lemma tls_pushs: ∀n,f. f = ⫱*[n] ↑*[n] f.
+#n elim n -n //
+#n #IH #f <tls_xn //
+qed.