]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/static_2/static/reqx.ma
update in static_2
[helm.git] / matita / matita / contribs / lambdadelta / static_2 / static / reqx.ma
index 251814a3bd8f62debf0669a18e147b7e92c73c29..8b7badaf9b849fb39ce500bf5425d9b8cb9ddbd5 100644 (file)
 (*                                                                        *)
 (**************************************************************************)
 
-include "static_2/notation/relations/stareqsn_3.ma".
+include "static_2/notation/relations/approxeqsn_3.ma".
 include "static_2/syntax/teqx_ext.ma".
-include "static_2/static/rex.ma".
+include "static_2/static/reqg.ma".
 
 (* SORT-IRRELEVANT EQUIVALENCE FOR LOCAL ENVIRONMENTS ON REFERRED ENTRIES ***)
-
+(*
 definition reqx: relation3 â€Ķ â‰
-           rex cdeq.
-
+           reqg sfull.
+*)
 interpretation
   "sort-irrelevant equivalence on referred entries (local environment)"
-  'StarEqSn T L1 L2 = (reqx T L1 L2).
+  'ApproxEqSn T L1 L2 = (reqg sfull T L1 L2).
 
 interpretation
   "sort-irrelevant ranged equivalence (local environment)"
-  'StarEqSn f L1 L2 = (sex cdeq_ext cfull f L1 L2).
+  'StarEqSn f L1 L2 = (sex ceqx_ext cfull f L1 L2).
 
 (* Basic properties ***********************************************************)
-
+(*
 lemma frees_teqx_conf_reqx:
       âˆ€f,L1,T1. L1 âŠĒ ð…+❊T1âŦ â‰˜ f â†’ âˆ€T2. T1 â‰› T2 â†’
       âˆ€L2. L1 â‰›[f] L2 â†’ L2 âŠĒ ð…+❊T2âŦ â‰˜ f.
@@ -128,7 +128,11 @@ lemma reqx_bind_repl_dx:
       âˆ€I,I1,L1,L2.∀T:term. L1.ⓘ[I] â‰›[T] L2.ⓘ[I1] â†’
       âˆ€I2. I â‰› I2 â†’ L1.ⓘ[I] â‰›[T] L2.ⓘ[I2].
 /2 width=2 by rex_bind_repl_dx/ qed-.
-
+*)
+lemma reqg_reqx (S) (T):
+      âˆ€L1,L2. L1 â‰›[S,T] L2 â†’ L1 â‰…[T] L2.
+/2 width=3 by reqg_co/ qed.
+(*
 (* Basic inversion lemmas ***************************************************)
 
 lemma reqx_inv_atom_sn:
@@ -215,3 +219,4 @@ lemma reqx_fwd_dx:
       âˆ€I2,L1,K2. âˆ€T:term. L1 â‰›[T] K2.ⓘ[I2] â†’
       âˆƒâˆƒI1,K1. L1 = K1.ⓘ[I1].
 /2 width=5 by rex_fwd_dx/ qed-.
+*)