X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fdelayed_updating%2Fsyntax%2Fprototerm_equivalence.ma;fp=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fdelayed_updating%2Fsyntax%2Fprototerm_equivalence.ma;h=0000000000000000000000000000000000000000;hb=6c52017b15171aa20ddfd01c1bbf3cc22a86c81c;hp=414c47d27e78313401b538d7c36a6c854d46ba02;hpb=4ac2becfaa45abb18acb2bdf3db5d2587cadb6d4;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/delayed_updating/syntax/prototerm_equivalence.ma b/matita/matita/contribs/lambdadelta/delayed_updating/syntax/prototerm_equivalence.ma deleted file mode 100644 index 414c47d27..000000000 --- a/matita/matita/contribs/lambdadelta/delayed_updating/syntax/prototerm_equivalence.ma +++ /dev/null @@ -1,32 +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 "ground/lib/subset_equivalence.ma". -include "delayed_updating/syntax/prototerm.ma". - -(* EQUIVALENCE FOR PROTOTERM ************************************************) - -(* Constructions with prototerm_root ****************************************) - -lemma prototerm_root_incl_repl: - ∀t1,t2. t1 ⊆ t2 → ▵t1 ⊆ ▵t2. -#t1 #t2 #Ht #p * #q #Hq -/3 width=2 by ex_intro/ -qed. - -lemma prototerm_root_eq_repl: - ∀t1,t2. t1 ⇔ t2 → ▵t1 ⇔ ▵t2. -#t1 #t2 * #H1 #H2 -/3 width=3 by conj, prototerm_root_incl_repl/ -qed.