aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-22 14:44:15 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-22 14:44:15 +0000
commitee07024b3b3265c2764e2d6b26036a69c280cb70 (patch)
treedffb61c75ab62f9b4556c39645cd6bf264727980
parentfef54f7bae3342686e8005879ed89253ea19c3aa (diff)
Add test-suite file for bug# 1905 and minor fix in Program/Equality.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11245 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--test-suite/bugs/closed/shouldsucceed/1905.v13
-rw-r--r--theories/Program/Equality.v2
2 files changed, 14 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/1905.v b/test-suite/bugs/closed/shouldsucceed/1905.v
new file mode 100644
index 000000000..bd7fd7967
--- /dev/null
+++ b/test-suite/bugs/closed/shouldsucceed/1905.v
@@ -0,0 +1,13 @@
+
+Require Import Setoid.
+
+Axiom t : Set.
+Axiom In : nat -> t -> Prop.
+Axiom InE : forall (x : nat) (s:t), impl (In x s) True.
+
+Goal forall a s,
+ In a s -> False.
+Proof.
+ intros a s Ia.
+ rewrite InE in Ia.
+Admitted. \ No newline at end of file
diff --git a/theories/Program/Equality.v b/theories/Program/Equality.v
index bb1ffbd2b..89e44c9bc 100644
--- a/theories/Program/Equality.v
+++ b/theories/Program/Equality.v
@@ -82,7 +82,7 @@ Ltac simpl_uip :=
(** Simplify equalities appearing in the context and goal. *)
-Ltac simpl_eq := simpl ; repeat (elim_eq_rect ; simpl) ; repeat (simpl_uip ; simpl).
+Ltac simpl_eq := simpl ; unfold eq_rec_r, eq_rec ; repeat (elim_eq_rect ; simpl) ; repeat (simpl_uip ; simpl).
(** Try to abstract a proof of equality, if no proof of the same equality is present in the context. *)