X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fground%2Fetc%2Frelocation%2Fpstream.etc;h=8827703c5f62b3c7daed862894aa89a697cd6323;hb=61bc42e04598a9f5e489c3867af72e700c7fda04;hp=90626a1d5ab6237a9fa742283abef67fcaafe7c6;hpb=11093619476326238c2ef9d2dfe9150b8c9bc920;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/ground/etc/relocation/pstream.etc b/matita/matita/contribs/lambdadelta/ground/etc/relocation/pstream.etc index 90626a1d5..8827703c5 100644 --- a/matita/matita/contribs/lambdadelta/ground/etc/relocation/pstream.etc +++ b/matita/matita/contribs/lambdadelta/ground/etc/relocation/pstream.etc @@ -18,24 +18,6 @@ include "ground/arith/pnat.ma". (* RELOCATION P-STREAM ******************************************************) -definition gr_push: gr_map → gr_map ≝ λf. 𝟏⨮f. - -interpretation "push (pstream)" 'UpSpoon f = (gr_push f). - -definition gr_next: gr_map → gr_map. -* #p #f @(↑p⨮f) -defined. - -interpretation "next (pstream)" 'UpArrow f = (gr_next f). - -(* Basic properties *********************************************************) - -lemma gr_push_unfold: ∀f. 𝟏⨮f = ⫯f. -// qed. - -lemma gr_next_unfold: ∀f,p. (↑p)⨮f = ↑(p⨮f). -// qed. - (* Basic inversion lemmas ***************************************************) lemma eq_inv_gr_push_bi: injective ? ? gr_push. @@ -54,22 +36,6 @@ lemma eq_inv_gr_next_bi: injective ? ? gr_next. * #p1 #f1 * #p2 #f2