aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-08 11:17:14 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-08 11:17:14 +0100
commit76058420ec0ea037504adf0af213d0542bd7c1c3 (patch)
tree37282697132f0b7db4f560b5503f7ec2dba11029 /test-suite/bugs
parent1f5699d57e9d4950b43d6c5f5259c3cf15564b31 (diff)
parent34babfdb5f45a04e89f671a21cc632ad127a26d4 (diff)
Merge PR #6899: [compat] Remove "Standard Proposition Elimination"
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/2378.v2
-rw-r--r--test-suite/bugs/opened/1596.v1
2 files changed, 0 insertions, 3 deletions
diff --git a/test-suite/bugs/closed/2378.v b/test-suite/bugs/closed/2378.v
index 85ad41d1c..23a58501f 100644
--- a/test-suite/bugs/closed/2378.v
+++ b/test-suite/bugs/closed/2378.v
@@ -505,8 +505,6 @@ Qed.
Require Export Coq.Logic.FunctionalExtensionality.
Print PLanguage.
-Unset Standard Proposition Elimination Names.
-
Program Definition PTransfo l1 l2 (tr: Transformation l1 l2) (h: isSharedTransfo l1 l2 tr):
Transformation (PLanguage l1) (PLanguage l2) :=
mkTransformation (PLanguage l1) (PLanguage l2)
diff --git a/test-suite/bugs/opened/1596.v b/test-suite/bugs/opened/1596.v
index 0b576db6b..820022d99 100644
--- a/test-suite/bugs/opened/1596.v
+++ b/test-suite/bugs/opened/1596.v
@@ -2,7 +2,6 @@ Require Import Relations.
Require Import FSets.
Require Import Arith.
Require Import Omega.
-Unset Standard Proposition Elimination Names.
Set Keyed Unification.