X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;ds=sidebyside;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Fetc_new%2Fllor%2Fllor.etc;fp=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Fetc_new%2Fllor%2Fllor.etc;h=0000000000000000000000000000000000000000;hb=50997cb3042073d58c2a16885ef0c82217367e63;hp=a2d1e61a7e32b2a810ccb59d69c64d48fb2270e2;hpb=560e9f41516968588e97bb6ff2049f85a425ac0a;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2/etc_new/llor/llor.etc b/matita/matita/contribs/lambdadelta/basic_2/etc_new/llor/llor.etc deleted file mode 100644 index a2d1e61a7..000000000 --- a/matita/matita/contribs/lambdadelta/basic_2/etc_new/llor/llor.etc +++ /dev/null @@ -1,40 +0,0 @@ -(**************************************************************************) -(* ___ *) -(* ||M|| *) -(* ||A|| A project by Andrea Asperti *) -(* ||T|| *) -(* ||I|| Developers: *) -(* ||T|| The HELM team. *) -(* ||A|| http://helm.cs.unibo.it *) -(* \ / *) -(* \ / This file is distributed under the terms of the *) -(* v GNU General Public License Version 2 *) -(* *) -(**************************************************************************) - -include "basic_2/notation/relations/lazyor_5.ma". -include "basic_2/multiple/frees.ma". - -(* POINTWISE UNION FOR LOCAL ENVIRONMENTS ***********************************) - -definition llor: ynat → relation4 term lenv lenv lenv ≝ λl,T,L2,L1,L. - ∧∧ |L1| = |L2| & |L1| = |L| - & (∀I1,I2,I,K1,K2,K,V1,V2,V,i. - ⬇[i] L1 ≡ K1.ⓑ{I1}V1 → ⬇[i] L2 ≡ K2.ⓑ{I2}V2 → ⬇[i] L ≡ K.ⓑ{I}V → ∨∨ - (∧∧ yinj i < l & I1 = I & V1 = V) | - (∧∧ (L1 ⊢ i ϵ 𝐅*[l]⦃T⦄ → ⊥) & I1 = I & V1 = V) | - (∧∧ l ≤ yinj i & L1 ⊢ i ϵ 𝐅*[l]⦃T⦄ & I2 = I & V2 = V) - ). - -interpretation - "lazy union (local environment)" - 'LazyOr L1 T l L2 L = (llor l T L2 L1 L). - -(* Basic properties *********************************************************) - -(* Note: this can be proved by llor_skip *) -lemma llor_atom: ∀T,l. ⋆ ⋓[T, l] ⋆ ≡ ⋆. -#T #l @and3_intro // -#I1 #I2 #I #K1 #K2 #K #V1 #V2 #V #i #HLK1 -elim (drop_inv_atom1 … HLK1) -HLK1 #H destruct -qed.