]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/delayed_updating/syntax/preterm_constructors.ma
update in delayed updating
[helm.git] / matita / matita / contribs / lambdadelta / delayed_updating / syntax / preterm_constructors.ma
index 03394c5bf6349fe99c6ab14b648259bea5fe8334..852fa0a59f204028bec097b7d212fbb0c51e8568 100644 (file)
@@ -21,15 +21,15 @@ include "delayed_updating/notation/functions/at_2.ma".
 (* CONSTRUCTORS FOR PRETERM *************************************************)
 
 definition preterm_node_0 (l): preterm ā‰
-           Ī»p. l;šž = p.
+           Ī»p. lā——šž = p.
 
 definition preterm_node_1 (l): preterm ā†’ preterm ā‰
-           Ī»t,p. āˆƒāˆƒq. q Ļµā¬¦ t & l;q = p.
+           Ī»t,p. āˆƒāˆƒq. q Ļµ t & lā——q = p.
 
 definition preterm_node_2 (l1) (l2): preterm ā†’ preterm ā†’ preterm ā‰
            Ī»t1,t2,p.
-           āˆØāˆØ āˆƒāˆƒq. q Ļµā¬¦ t1 & l1;q = p
-            | āˆƒāˆƒq. q Ļµā¬¦ t2 & l2;q = p.
+           āˆØāˆØ āˆƒāˆƒq. q Ļµ t1 & l1ā——q = p
+            | āˆƒāˆƒq. q Ļµ t2 & l2ā——q = p.
 
 interpretation
   "outer variable reference by depth (preterm)"
@@ -50,8 +50,8 @@ interpretation
 (* Basic Inversions *********************************************************)
 
 lemma preterm_in_root_inv_lcons_oref:
-      āˆ€p,l,n. l;p Ļµā–µ #n ā†’
-      āˆ§āˆ§ š—±āØnā© = l & šž = p.
+      āˆ€p,l,n. lā——p Ļµ ā–µ#n ā†’
+      āˆ§āˆ§ š—±n = l & šž = p.
 #p #l #n * #q
 <list_append_lcons_sn #H0 destruct -H0
 elim (eq_inv_list_empty_append ā€¦ e0) -e0 #H0 #_
@@ -59,25 +59,25 @@ elim (eq_inv_list_empty_append ā€¦ e0) -e0 #H0 #_
 qed-.
 
 lemma preterm_in_root_inv_lcons_iref:
-      āˆ€t,p,l,n. l;p Ļµā–µ š›—n.t ā†’
-      āˆ§āˆ§ š—±āØnā© = l & p Ļµā–µ t.
+      āˆ€t,p,l,n. lā——p Ļµ ā–µš›—n.t ā†’
+      āˆ§āˆ§ š—±n = l & p Ļµ ā–µt.
 #t #p #l #n * #q
 <list_append_lcons_sn * #r #Hr #H0 destruct
 /3 width=2 by ex_intro, conj/
 qed-.
 
 lemma preterm_in_root_inv_lcons_abst:
-      āˆ€t,p,l. l;p Ļµā–µ š›Œ.t ā†’
-      āˆ§āˆ§ š—Ÿ = l & p Ļµā–µ t.
+      āˆ€t,p,l. lā——p Ļµ ā–µš›Œ.t ā†’
+      āˆ§āˆ§ š—Ÿ = l & p Ļµ ā–µt.
 #t #p #l * #q
 <list_append_lcons_sn * #r #Hr #H0 destruct
 /3 width=2 by ex_intro, conj/
 qed-.
 
 lemma preterm_in_root_inv_lcons_appl:
-      āˆ€u,t,p,l. l;p Ļµā–µ @u.t ā†’
-      āˆØāˆØ āˆ§āˆ§ š—¦ = l & p Ļµā–µ u
-       | āˆ§āˆ§ š—” = l & p Ļµā–µ t.
+      āˆ€u,t,p,l. lā——p Ļµ ā–µ@u.t ā†’
+      āˆØāˆØ āˆ§āˆ§ š—¦ = l & p Ļµ ā–µu
+       | āˆ§āˆ§ š—” = l & p Ļµ ā–µt.
 #u #t #p #l * #q
 <list_append_lcons_sn * * #r #Hr #H0 destruct
 /4 width=2 by ex_intro, or_introl, or_intror, conj/