diff options
author | glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-12-23 19:28:45 +0000 |
---|---|---|
committer | glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2010-12-23 19:28:45 +0000 |
commit | b26dcdc37705c2e0d5f7d4322f5dc26fb6b7984a (patch) | |
tree | b3f7bb2f56c18a452d6a4972d84d1475c7a3b219 /test-suite/success | |
parent | 4dc1e6db7c6742e098b2f710613afd14fdff3987 (diff) |
Remove the two-argument variant of "decide equality"
This variant was ignoring its second argument, and didn't exactly
respect its documented specification. This is fixed by removing the
variant altogether.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13746 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r-- | test-suite/success/eqdecide.v | 7 |
1 files changed, 1 insertions, 6 deletions
diff --git a/test-suite/success/eqdecide.v b/test-suite/success/eqdecide.v index 5f2d0f395..8c00583ed 100644 --- a/test-suite/success/eqdecide.v +++ b/test-suite/success/eqdecide.v @@ -16,12 +16,7 @@ Qed. Lemma lem2 : forall x y : T, {x = y} + {x <> y}. intros x y. - decide equality x y. -Qed. - -Lemma lem3 : forall x y : T, {x = y} + {x <> y}. -intros x y. - decide equality y x. + decide equality. Qed. Lemma lem4 : forall x y : T, {x = y} + {x <> y}. |