diff options
author | Emilio Jesus Gallego Arias <e+git@x80.org> | 2018-04-09 01:33:31 +0200 |
---|---|---|
committer | Emilio Jesus Gallego Arias <e+git@x80.org> | 2018-04-13 12:13:48 +0200 |
commit | 2243c25c79ab19876ad74452c9cecc7dcc88c67c (patch) | |
tree | f32573eb7d7c4dbdb4493e186bed87c80e61a747 /test-suite/bugs/closed | |
parent | b68e0b4f9ba37d1c2fa5921e1d934b4b38bfdfe7 (diff) |
[ltac] Deprecate nameless fix/cofix.
LTAC's `fix` and `cofix` do require access to the proof object inside
the tactic monad when used without a name. This is a bit inconvenient
as we aim to make the handling of the proof object purely functional.
Alternatives have been discussed in #7196, and it seems that
deprecating the nameless forms may have the best cost/benefit ratio,
so opening this PR for discussion.
See also #6171.
Diffstat (limited to 'test-suite/bugs/closed')
-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 |
3 files changed, 3 insertions, 3 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 |