summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/1905.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/shouldsucceed/1905.v')
-rw-r--r--test-suite/bugs/closed/shouldsucceed/1905.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/1905.v b/test-suite/bugs/closed/shouldsucceed/1905.v
new file mode 100644
index 00000000..bd7fd796
--- /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