summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/1962.v
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <gareuselesinge@debian.org>2015-01-25 14:42:51 +0100
committerGravatar Enrico Tassi <gareuselesinge@debian.org>2015-01-25 14:42:51 +0100
commit7cfc4e5146be5666419451bdd516f1f3f264d24a (patch)
treee4197645da03dc3c7cc84e434cc31d0a0cca7056 /test-suite/bugs/closed/shouldsucceed/1962.v
parent420f78b2caeaaddc6fe484565b2d0e49c66888e5 (diff)
Imported Upstream version 8.5~beta1+dfsg
Diffstat (limited to 'test-suite/bugs/closed/shouldsucceed/1962.v')
-rw-r--r--test-suite/bugs/closed/shouldsucceed/1962.v55
1 files changed, 0 insertions, 55 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/1962.v b/test-suite/bugs/closed/shouldsucceed/1962.v
deleted file mode 100644
index a6b0fee5..00000000
--- a/test-suite/bugs/closed/shouldsucceed/1962.v
+++ /dev/null
@@ -1,55 +0,0 @@
-(* Bug 1962.v
-
-Bonjour,
-
-J'ai un exemple de lemme que j'arrivais à prouver avec fsetdec avec la 8.2beta3
-avec la beta4 et la version svn 11447 branche 8.2 çà diverge.
-
-Voici l'exemple en question, l'exmple test2 marche bien dans les deux version,
-test en revanche pose probleme:
-
-*)
-
-Require Export FSets.
-
-(** This module takes a decidable type and
-build finite sets of this type, tactics and defs *)
-
-Module BuildFSets (DecPoints: UsualDecidableType).
-
-Module Export FiniteSetsOfPoints := FSetWeakList.Make DecPoints.
-Module Export FiniteSetsOfPointsProperties :=
- WProperties FiniteSetsOfPoints.
-Module Export Dec := WDecide FiniteSetsOfPoints.
-Module Export FM := Dec.F.
-
-Definition set_of_points := t.
-Definition Point := DecPoints.t.
-
-Definition couple(x y :Point) : set_of_points :=
-add x (add y empty).
-
-Definition triple(x y t :Point): set_of_points :=
-add x (add y (add t empty)).
-
-Lemma test : forall P A B C A' B' C',
-Equal
-(union (singleton P) (union (triple A B C) (triple A' B' C')))
-(union (triple P B B') (union (couple P A) (triple C A' C'))).
-Proof.
-intros.
-unfold triple, couple.
-Time fsetdec. (* works in 8.2 beta 3, not in beta 4 and final 8.2 *)
- (* appears to works again in 8.3 and trunk, take 4-6 seconds *)
-Qed.
-
-Lemma test2 : forall A B C,
-Equal
- (union (singleton C) (couple A B)) (triple A B C).
-Proof.
-intros.
-unfold triple, couple.
-Time fsetdec.
-Qed.
-
-End BuildFSets. \ No newline at end of file