diff options
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/bugs/closed/2001.v | 2 | ||||
-rw-r--r-- | test-suite/bugs/closed/3320.v | 2 | ||||
-rw-r--r-- | test-suite/bugs/closed/3350.v | 2 | ||||
-rw-r--r-- | test-suite/success/ShowExtraction.v | 2 | ||||
-rw-r--r-- | test-suite/success/name_mangling.v | 3 |
5 files changed, 5 insertions, 6 deletions
diff --git a/test-suite/bugs/closed/2001.v b/test-suite/bugs/closed/2001.v index d0b3bf173..652c65706 100644 --- a/test-suite/bugs/closed/2001.v +++ b/test-suite/bugs/closed/2001.v @@ -7,7 +7,7 @@ Inductive T : Set := | v : T. Definition f (s:nat) (t:T) : nat. -fix 2. +fix f 2. intros s t. refine match t with diff --git a/test-suite/bugs/closed/3320.v b/test-suite/bugs/closed/3320.v index 0aac3c1b0..a5c243d8e 100644 --- a/test-suite/bugs/closed/3320.v +++ b/test-suite/bugs/closed/3320.v @@ -1,5 +1,5 @@ Goal forall x : nat, True. - fix 1. + fix goal 1. assumption. Fail Qed. Undo. diff --git a/test-suite/bugs/closed/3350.v b/test-suite/bugs/closed/3350.v index c041c401f..c1ff292b3 100644 --- a/test-suite/bugs/closed/3350.v +++ b/test-suite/bugs/closed/3350.v @@ -55,7 +55,7 @@ Lemma lower_ind (P: forall n (p i:Fin.t (S n)), option (Fin.t n) -> Prop) P (S n) (Fin.FS p) (Fin.FS i) None) : forall n (p i:Fin.t (S n)), P n p i (lower p i). Proof. - fix 2. intros n p. + fix lower_ind 2. intros n p. refine (match p as p1 in Fin.t (S n1) return forall (i1:Fin.t (S n1)), P n1 p1 i1 (lower p1 i1) with diff --git a/test-suite/success/ShowExtraction.v b/test-suite/success/ShowExtraction.v index e34c240c5..a4a35003d 100644 --- a/test-suite/success/ShowExtraction.v +++ b/test-suite/success/ShowExtraction.v @@ -12,7 +12,7 @@ Fail Show Extraction. Lemma decListA : forall (xs ys : list A), {xs=ys}+{xs<>ys}. Proof. Show Extraction. -fix 1. +fix decListA 1. destruct xs as [|x xs], ys as [|y ys]. Show Extraction. - now left. diff --git a/test-suite/success/name_mangling.v b/test-suite/success/name_mangling.v index 571dde880..e98241420 100644 --- a/test-suite/success/name_mangling.v +++ b/test-suite/success/name_mangling.v @@ -122,8 +122,7 @@ Lemma a : forall n, n = 0. Proof. fix a 1. Check a. -fix 1. -Fail Check a0. +Fail fix a 1. Abort. (* Test stability of "induction" *) |