From 246909f2c587ed798bc42b65fb90c7b77dfa52b7 Mon Sep 17 00:00:00 2001 From: herbelin Date: Fri, 13 Jul 2007 14:55:03 +0000 Subject: Répertoire Numbers poursuit l'objectif entamé en syntaxe V7 dans le répertoire Num. Suppression de ce dernier de l'archive courante. MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9995 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Num/LtProps.v | 82 -------------------------------------------------- 1 file changed, 82 deletions(-) delete mode 100644 theories/Num/LtProps.v (limited to 'theories/Num/LtProps.v') diff --git a/theories/Num/LtProps.v b/theories/Num/LtProps.v deleted file mode 100644 index 79f0f3303..000000000 --- a/theories/Num/LtProps.v +++ /dev/null @@ -1,82 +0,0 @@ -(************************************************************************) -(* v * The Coq Proof Assistant / The Coq Development Team *) -(* ~(y~(x(x<(S y)). -EAuto with num. -Qed. -Hints Resolve eq_lt_x_Sy : num. - -Lemma lt_lt_x_Sy : (x,y:N)(x(x<(S y)). -EAuto with num. -Qed. -Hints Immediate lt_lt_x_Sy : num. - -Lemma lt_Sx_y_lt : (x,y:N)((S x)(x(x<>y). -Red; Intros x y lt1 eq1; Apply (lt_anti_refl x); EAuto with num. -Qed. -Hints Immediate lt_neq : num. - -Lemma lt_neq_sym : (x,y:N)(y(x<>y). -Intros x y lt1 ; Apply neq_sym; Auto with num. -Qed. -Hints Immediate lt_neq_sym : num. - -(** Application to inequalities properties *) - -Lemma neq_x_Sx : (x:N)x<>(S x). -Auto with num. -Qed. -Hints Resolve neq_x_Sx : num. - -Lemma neq_0_1 : zero<>one. -Auto with num. -Qed. -Hints Resolve neq_0_1 : num. - -(** Relating [<] and [+] *) - -Lemma lt_add_compat_r : (x,y,z:N)(x((z+x)<(z+y)). -Intros x y z H; Apply lt_eq_compat with (x+z) (y+z); Auto with num. -Qed. -Hints Resolve lt_add_compat_r : num. - -Lemma lt_add_compat : (x1,x2,y1,y2:N)(x1(y1((x1+y1)<(x2+y2)). -Intros; Apply lt_trans with (x1+y2); Auto with num. -Qed. -Hints Immediate lt_add_compat : num. - -- cgit v1.2.3