X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matitaB%2Fmatita%2Fcontribs%2FRELATIONAL%2FZEq%2Fsetoid.ma;fp=matitaB%2Fmatita%2Fcontribs%2FRELATIONAL%2FZEq%2Fsetoid.ma;h=0000000000000000000000000000000000000000;hb=da0775e27b362e91ea1453a800bc403781cc2ca3;hp=03075bb75818909371091eaeec06d4178d59eafc;hpb=d9824956d9132109ed5f23380a0a1f9c5181d18a;p=helm.git diff --git a/matitaB/matita/contribs/RELATIONAL/ZEq/setoid.ma b/matitaB/matita/contribs/RELATIONAL/ZEq/setoid.ma deleted file mode 100644 index 03075bb75..000000000 --- a/matitaB/matita/contribs/RELATIONAL/ZEq/setoid.ma +++ /dev/null @@ -1,37 +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 "NPlus/fun.ma". -include "ZEq/defs.ma". - -theorem zeq_refl: ∀z. z ≈ z. - intros; elim z. clear z. - lapply (nplus_total a b); decompose; - autobatch. -qed. - -theorem zeq_sym: ∀z1,z2. z1 ≈ z2 → z2 ≈ z1. - intros; elim H; clear H z1 z2; autobatch. -qed. -(* -theorem zeq_trans: \forall z1,z2. z1 = z2 \to - \forall z3. z2 = z3 \to z1 = z3. - intros 3. elim H. clear H z1 z2. - inversion H3. clear H3. intros. destruct. - lapply (nplus_total n5 n6). decompose. - lapply (nplus_total n4 n9). decompose. - apply zeq. -*)