]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/apps_2/models/deq.ma
some restyling ...
[helm.git] / matita / matita / contribs / lambdadelta / apps_2 / models / deq.ma
index 8de93a606782d76b8c6afbbca2ab9c7c204dc201..849ad9dd43ef0e834c3846791737526bafdae80b 100644 (file)
 (**************************************************************************)
 
 include "apps_2/notation/models/ringeq_5.ma".
-include "apps_2/models/model_gi.ma".
-include "apps_2/models/model_li.ma".
-include "apps_2/models/model_props.ma".
+include "apps_2/models/li.ma".
+include "static_2/syntax/genv.ma".
 
 (* DENOTATIONAL EQUIVALENCE  ************************************************)
 
 definition deq (M): relation4 genv lenv term term ≝
-                    λG,L,T1,T2. ∀gv,lv. lv ϵ ⟦L⟧[gv] → ⟦T1⟧[gv, lv] ≗{M} ⟦T2⟧[gv, lv].
+                    λG,L,T1,T2. ∀gv,lv. lv ϵ ⟦L⟧[gv] → ⟦T1⟧[gv,lv] ≗{M} ⟦T2⟧[gv,lv].
 
 interpretation "denotational equivalence (model)"
    'RingEq M G L T1 T2 = (deq M G L T1 T2).
@@ -29,7 +28,7 @@ interpretation "denotational equivalence (model)"
 
 lemma deq_refl (M): is_model M →
                     ∀G,L. reflexive … (deq M G L).
-/2 width=1 by mq/ qed.
+/2 width=1 by mr/ qed.
 (*
 lemma veq_sym: ∀M. symmetric … (veq M).
 // qed-.