diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2006-01-21 15:25:41 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2006-01-21 15:25:41 +0000 |
commit | 5ec47cbb80137eb2542d665056d1f1d2a5a82c9f (patch) | |
tree | 16222109dd02afdbdf10c08f82afecfe33b977ed | |
parent | 642e522429e6f5faa381aaf26cd530a939b5a601 (diff) |
Backtrack commit précédent: la préservation de l'énoncé exact Acc_ind est incompatible avec la préservation du type de Acc_intro (par uniformité de notations, x est finalement préféré)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@7912 85f007b7-540e-0410-9357-904b9bb8a0f7
-rwxr-xr-x | theories/Init/Wf.v | 4 |
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Init/Wf.v b/theories/Init/Wf.v index 3d4d0efba..5a05f7b65 100755 --- a/theories/Init/Wf.v +++ b/theories/Init/Wf.v @@ -29,8 +29,8 @@ Section Well_founded. (** The accessibility predicate is defined to be non-informative *) - Inductive Acc (a: A) : Prop := - Acc_intro : (forall y:A, R y a -> Acc y) -> Acc a. + Inductive Acc (x: A) : Prop := + Acc_intro : (forall y:A, R y x -> Acc y) -> Acc x. Lemma Acc_inv : forall x:A, Acc x -> forall y:A, R y x -> Acc y. destruct 1; trivial. |