aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-09 15:11:52 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-09 15:11:52 +0100
commit0b3a458ecf2cfbe8cd2905d28f2459bd16240a18 (patch)
treee49f0cb970aad0ba8dd22088bf51d7d75ce2b8b8 /test-suite
parentd04f262f4c27a086b9ddfef1931586ef1062614d (diff)
parent67091e1d155be19333c5e5bd2cc306792ca630d3 (diff)
Merge PR #6895: [compat] Remove "Refolding Reduction" option.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/opened/3424.v (renamed from test-suite/bugs/closed/3424.v)4
-rw-r--r--test-suite/output/inference.out2
-rw-r--r--test-suite/output/inference.v6
3 files changed, 2 insertions, 10 deletions
diff --git a/test-suite/bugs/closed/3424.v b/test-suite/bugs/opened/3424.v
index ee8cabf17..d1c5bb68f 100644
--- a/test-suite/bugs/closed/3424.v
+++ b/test-suite/bugs/opened/3424.v
@@ -13,12 +13,12 @@ Notation "0" := (trunc_S minus_one) : trunc_scope.
Class IsTrunc (n : trunc_index) (A : Type) : Type := Trunc_is_trunc : IsTrunc_internal n A.
Notation IsHProp := (IsTrunc minus_one).
Notation IsHSet := (IsTrunc 0).
-Set Refolding Reduction.
Goal forall (A : Type) (a b : A) (H' : IsHSet A), { x : Type & IsHProp x }.
Proof.
intros.
eexists.
(* exact (H' a b). *)
(* Undo. *)
-apply (H' a b).
+Fail apply (H' a b).
+exact (H' a b).
Qed.
diff --git a/test-suite/output/inference.out b/test-suite/output/inference.out
index 5e9eff048..f7ffd1959 100644
--- a/test-suite/output/inference.out
+++ b/test-suite/output/inference.out
@@ -4,8 +4,6 @@ fun e : option L => match e with
| None => None
end
: option L -> option L
-fun (m n p : nat) (H : S m <= S n + p) => le_S_n m (n + p) H
- : forall m n p : nat, S m <= S n + p -> m <= n + p
fun n : nat => let y : T n := A n in ?t ?x : T n
: forall n : nat, T n
where
diff --git a/test-suite/output/inference.v b/test-suite/output/inference.v
index 73169dae6..57a4739e9 100644
--- a/test-suite/output/inference.v
+++ b/test-suite/output/inference.v
@@ -13,12 +13,6 @@ Definition P (e:option L) :=
Print P.
-(* Check that plus is folded even if reduction is involved *)
-Set Warnings Append "-deprecated-option".
-Set Refolding Reduction.
-Check (fun m n p (H : S m <= (S n) + p) => le_S_n _ _ H).
-
-
(* Check that the heuristic to solve constraints is not artificially
dependent on the presence of a let-in, and in particular that the
second [_] below is not inferred to be n, as if obtained by