From 3ef7797ef6fc605dfafb32523261fe1b023aeecb Mon Sep 17 00:00:00 2001 From: Samuel Mimram Date: Fri, 28 Apr 2006 14:59:16 +0000 Subject: Imported Upstream version 8.0pl3+8.1alpha --- theories/Logic/Classical_Pred_Set.v | 47 ++++++++++--------------------------- 1 file changed, 12 insertions(+), 35 deletions(-) mode change 100755 => 100644 theories/Logic/Classical_Pred_Set.v (limited to 'theories/Logic/Classical_Pred_Set.v') diff --git a/theories/Logic/Classical_Pred_Set.v b/theories/Logic/Classical_Pred_Set.v old mode 100755 new mode 100644 index c8f87fe8..2a5f03ec --- a/theories/Logic/Classical_Pred_Set.v +++ b/theories/Logic/Classical_Pred_Set.v @@ -6,11 +6,14 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -(*i $Id: Classical_Pred_Set.v,v 1.6.2.1 2004/07/16 19:31:06 herbelin Exp $ i*) +(*i $Id: Classical_Pred_Set.v 8642 2006-03-17 10:09:02Z notin $ i*) + +(** This file is obsolete, use Classical_Pred_Type.v via Classical.v +instead *) (** Classical Predicate Logic on Set*) -Require Import Classical_Prop. +Require Import Classical_Pred_Type. Section Generic. Variable U : Set. @@ -19,52 +22,26 @@ Variable U : Set. Lemma not_all_ex_not : forall P:U -> Prop, ~ (forall n:U, P n) -> exists n : U, ~ P n. -Proof. -unfold not in |- *; intros P notall. -apply NNPP; unfold not in |- *. -intro abs. -cut (forall n:U, P n); auto. -intro n; apply NNPP. -unfold not in |- *; intros. -apply abs; exists n; trivial. -Qed. +Proof (Classical_Pred_Type.not_all_ex_not U). Lemma not_all_not_ex : forall P:U -> Prop, ~ (forall n:U, ~ P n) -> exists n : U, P n. -Proof. -intros P H. -elim (not_all_ex_not (fun n:U => ~ P n) H); intros n Pn; exists n. -apply NNPP; trivial. -Qed. +Proof (Classical_Pred_Type.not_all_not_ex U). Lemma not_ex_all_not : forall P:U -> Prop, ~ (exists n : U, P n) -> forall n:U, ~ P n. -Proof. -unfold not in |- *; intros P notex n abs. -apply notex. -exists n; trivial. -Qed. +Proof (Classical_Pred_Type.not_ex_all_not U). Lemma not_ex_not_all : forall P:U -> Prop, ~ (exists n : U, ~ P n) -> forall n:U, P n. -Proof. -intros P H n. -apply NNPP. -red in |- *; intro K; apply H; exists n; trivial. -Qed. +Proof (Classical_Pred_Type.not_ex_not_all U). Lemma ex_not_not_all : forall P:U -> Prop, (exists n : U, ~ P n) -> ~ (forall n:U, P n). -Proof. -unfold not in |- *; intros P exnot allP. -elim exnot; auto. -Qed. +Proof (Classical_Pred_Type.ex_not_not_all U). Lemma all_not_not_ex : forall P:U -> Prop, (forall n:U, ~ P n) -> ~ (exists n : U, P n). -Proof. -unfold not in |- *; intros P allnot exP; elim exP; intros n p. -apply allnot with n; auto. -Qed. +Proof (Classical_Pred_Type.all_not_not_ex U). -End Generic. \ No newline at end of file +End Generic. -- cgit v1.2.3