aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authormsozeau2009-11-13 00:38:28 +0000
committermsozeau2009-11-13 00:38:28 +0000
commitc242a71f206dfbafff457a1229b6322172d64f55 (patch)
tree9248af1dfe5b8cd8dfafd37aa31043ea840aa2fb
parent0024fe475225340d652d15e68d1e4f657d76cc08 (diff)
Fix test-suite scripts: [Generalizable Variables] and small
changes in obligations. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12514 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--test-suite/bugs/closed/shouldsucceed/1784.v4
-rw-r--r--test-suite/bugs/closed/shouldsucceed/2083.v4
-rw-r--r--test-suite/bugs/closed/shouldsucceed/2139.v2
-rw-r--r--test-suite/success/AdvancedTypeClasses.v2
-rw-r--r--test-suite/success/Generalization.v1
-rw-r--r--test-suite/success/ProgramWf.v5
-rw-r--r--test-suite/success/dependentind.v4
7 files changed, 16 insertions, 6 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/1784.v b/test-suite/bugs/closed/shouldsucceed/1784.v
index 8c2e50e07d..51d5ca728a 100644
--- a/test-suite/bugs/closed/shouldsucceed/1784.v
+++ b/test-suite/bugs/closed/shouldsucceed/1784.v
@@ -93,9 +93,9 @@ Next Obligation.
intro H1; contradict H. inversion H1; subst. assumption.
contradict H0; assumption. Defined.
Next Obligation.
- intro H1; contradict H0. inversion H1; subst. assumption. Defined.
+ intro H1; contradict H. inversion H1; subst. assumption. Defined.
Next Obligation.
- intro H0; contradict H. inversion H0; subst. assumption. Defined.
+ intro H1; contradict H0. inversion H1; subst. assumption. Defined.
Next Obligation.
intro H0; contradict H. inversion H0; subst; auto. Defined.
diff --git a/test-suite/bugs/closed/shouldsucceed/2083.v b/test-suite/bugs/closed/shouldsucceed/2083.v
index 6fc046495c..a6ce4de0f6 100644
--- a/test-suite/bugs/closed/shouldsucceed/2083.v
+++ b/test-suite/bugs/closed/shouldsucceed/2083.v
@@ -15,11 +15,13 @@ Program Fixpoint check_n (n : nat) (P : { i | i < n } -> bool) (p : nat)
Require Import Omega.
+Solve Obligations using program_simpl ; auto with *; try omega.
+
Next Obligation.
apply H. simpl. omega.
Defined.
-Next Obligation.
+Next Obligation.
case (le_lt_dec p i) ; intros. assert(i = p) by omega. subst.
revert H0. clear_subset_proofs. auto.
apply H. simpl. assumption. Defined.
diff --git a/test-suite/bugs/closed/shouldsucceed/2139.v b/test-suite/bugs/closed/shouldsucceed/2139.v
index 415a1b27dd..a7f3550888 100644
--- a/test-suite/bugs/closed/shouldsucceed/2139.v
+++ b/test-suite/bugs/closed/shouldsucceed/2139.v
@@ -1,4 +1,5 @@
(* Call of apply on <-> failed because of evars in elimination predicate *)
+Generalizable Variables patch.
Class Patch (patch : Type) := {
commute : patch -> patch -> Prop
@@ -21,4 +22,3 @@ apply flip in H.
type of (@flip _ _ _ _) itself had non-normalized evars *)
(* By the way, is the check necessary ? *)
-
diff --git a/test-suite/success/AdvancedTypeClasses.v b/test-suite/success/AdvancedTypeClasses.v
index 219a8a7551..a6f1e299b1 100644
--- a/test-suite/success/AdvancedTypeClasses.v
+++ b/test-suite/success/AdvancedTypeClasses.v
@@ -1,3 +1,5 @@
+Generalizable Variables all.
+
Open Scope type_scope.
Section type_reification.
diff --git a/test-suite/success/Generalization.v b/test-suite/success/Generalization.v
index 6b503e95ae..4ec0a79ba1 100644
--- a/test-suite/success/Generalization.v
+++ b/test-suite/success/Generalization.v
@@ -1,3 +1,4 @@
+Generalizable Variables all.
Check `(a = 0).
Check `(a = 0)%type.
diff --git a/test-suite/success/ProgramWf.v b/test-suite/success/ProgramWf.v
index 18111f07c5..81bdbc29f0 100644
--- a/test-suite/success/ProgramWf.v
+++ b/test-suite/success/ProgramWf.v
@@ -56,7 +56,10 @@ Lemma merge_unfold n m : merge n m =
| 0 => 0
| S n' => merge n' m
end.
-Proof. intros. unfold_sub merge (merge n m). simpl. destruct n ; reflexivity. Qed.
+Proof. intros. unfold merge at 1. unfold merge_func.
+ unfold_sub merge (merge n m).
+ simpl. destruct n ; reflexivity.
+Qed.
Print merge.
diff --git a/test-suite/success/dependentind.v b/test-suite/success/dependentind.v
index f308bdfd9b..a19515d06c 100644
--- a/test-suite/success/dependentind.v
+++ b/test-suite/success/dependentind.v
@@ -1,4 +1,4 @@
-Require Import Coq.Program.Program Coq.Program.Equations.
+Require Import Coq.Program.Program Coq.Program.Equality.
Variable A : Set.
@@ -50,6 +50,8 @@ Notation " Γ ; Δ " := (conc Δ Γ) (at level 25, left associativity) : contex
Reserved Notation " Γ ⊢ τ " (at level 30, no associativity).
+Generalizable Variables all.
+
Inductive term : ctx -> type -> Type :=
| ax : `(Γ, τ ⊢ τ)
| weak : `{Γ ⊢ τ -> Γ, τ' ⊢ τ}