From 3675bac6c38e0a26516e434be08bc100865b339b Mon Sep 17 00:00:00 2001 From: barras Date: Mon, 15 Dec 2003 19:48:24 +0000 Subject: modif existentielle (exists | --> exists ,) + bug d'affichage des pt fixes git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5099 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Wellfounded/Inverse_Image.v | 2 +- theories/Wellfounded/Lexicographic_Exponentiation.v | 4 ++-- theories/Wellfounded/Union.v | 2 +- 3 files changed, 4 insertions(+), 4 deletions(-) (limited to 'theories/Wellfounded') diff --git a/theories/Wellfounded/Inverse_Image.v b/theories/Wellfounded/Inverse_Image.v index 66a7f5b5b..b11c8c635 100644 --- a/theories/Wellfounded/Inverse_Image.v +++ b/theories/Wellfounded/Inverse_Image.v @@ -35,7 +35,7 @@ Section Inverse_Image. Variable F : A -> B -> Prop. Let RoF (x y:A) : Prop := - exists2 b : B | F x b & (forall c:B, F y c -> R b c). + exists2 b : B, F x b & (forall c:B, F y c -> R b c). Lemma Acc_inverse_rel : forall b:B, Acc R b -> forall x:A, F x b -> Acc RoF x. induction 1 as [x _ IHAcc]; intros x0 H2. diff --git a/theories/Wellfounded/Lexicographic_Exponentiation.v b/theories/Wellfounded/Lexicographic_Exponentiation.v index e8203c399..3daf09a97 100644 --- a/theories/Wellfounded/Lexicographic_Exponentiation.v +++ b/theories/Wellfounded/Lexicographic_Exponentiation.v @@ -54,7 +54,7 @@ Qed. Lemma right_prefix : forall x y z:List, - ltl x (y ++ z) -> ltl x y \/ ( exists y' : List | x = y ++ y' /\ ltl y' z). + ltl x (y ++ z) -> ltl x y \/ (exists y' : List, x = y ++ y' /\ ltl y' z). Proof. intros x y; generalize x. elim y; simpl in |- *. @@ -371,4 +371,4 @@ Proof. Qed. -End Wf_Lexicographic_Exponentiation. \ No newline at end of file +End Wf_Lexicographic_Exponentiation. diff --git a/theories/Wellfounded/Union.v b/theories/Wellfounded/Union.v index d7f241dd0..6a6a9882f 100644 --- a/theories/Wellfounded/Union.v +++ b/theories/Wellfounded/Union.v @@ -26,7 +26,7 @@ Remark strip_commut : commut A R1 R2 -> forall x y:A, clos_trans A R1 y x -> - forall z:A, R2 z y -> exists2 y' : A | R2 y' x & clos_trans A R1 z y'. + forall z:A, R2 z y -> exists2 y' : A, R2 y' x & clos_trans A R1 z y'. Proof. induction 2 as [x y| x y z H0 IH1 H1 IH2]; intros. elim H with y x z; auto with sets; intros x0 H2 H3. -- cgit v1.2.3