X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=helm%2Fsoftware%2Fmatita%2Ftests%2Fsubsumption.ma;fp=helm%2Fsoftware%2Fmatita%2Ftests%2Fsubsumption.ma;h=333afdc5c881a1cde21e8f7f2c141abe615aebbb;hb=a023ee84b0efd8febff8bdd3cf7d92aa0317f12a;hp=0000000000000000000000000000000000000000;hpb=2701c980f48541dd5e8317b5a5661b439ced8b29;p=helm.git diff --git a/helm/software/matita/tests/subsumption.ma b/helm/software/matita/tests/subsumption.ma new file mode 100644 index 000000000..333afdc5c --- /dev/null +++ b/helm/software/matita/tests/subsumption.ma @@ -0,0 +1,54 @@ +(**************************************************************************) +(* ___ *) +(* ||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 "logic/equality.ma". + +ntheorem foo : + ∀U : Type. + ∀a : U. + ∀b : U. + ∀f : U → U → U. + ∀g : U → U → U. + ∀H : ∀x.g x a = g a x. + ∃y,z. f (g y b) y = f (g z a) a. +#U. #a. #b. #f. #g. #H. +napply (ex_intro ????); +##[ ##2: napply (ex_intro ????); + ##[ ##2: nauto by H. ##| ##skip ##] ##| ##skip ##] nqed. + +ntheorem foo1 : + ∀U : Type. + ∀a : U. + ∀b : U. + ∀f : U → U → U. + ∀g : U → U → U. + ∀H : ∀x.g x a = g a x. + ∃y,z. f y (g y b) = f a (g z a). +#U. #a. #b. #f. #g. #H. +napply (ex_intro ????); +##[ ##2: napply (ex_intro ????); + ##[ ##2: nauto by H. ##| ##skip ##] ##| ##skip ##] nqed. + +ntheorem foo2 : + ∀U : Type. + ∀a : U. + ∀b : U. + ∀f : U → U → U. + ∀g : U → U → U. + ∀H : ∀x.g x a = g a x. + ∃y,z. f (g z a) (g y b) = f (g y b) (g z a). +#U. #a. #b. #f. #g. #H. +napply (ex_intro ????); +##[ ##2: napply (ex_intro ????); + ##[ ##2: nauto by H. ##| ##skip ##] ##| ##skip ##] nqed. + \ No newline at end of file