diff options
author | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2014-09-30 09:50:07 +0200 |
---|---|---|
committer | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2014-09-30 10:02:47 +0200 |
commit | a1be9ce30ed0c59d3cd8651ff0c624a24a6d3fc9 (patch) | |
tree | a2d0ce66634899dd71d5abb8e525cf1a7ebad7cb /test-suite/success | |
parent | 538b77dbb3b7799dc4d2e18033fc4fbf2eb26f7f (diff) |
Seeing IntroWildcard as an action intro pattern rather than as a naming pattern
(the action is "clear").
Added subst_intropattern which was missing since the introduction of
ApplyOn intro patterns.
Still to do: make "intros _ ?id" working without interferences when
"id" is precisely the internal name used for hypotheses to discard.
Diffstat (limited to 'test-suite/success')
-rw-r--r-- | test-suite/success/intros.v | 5 |
1 files changed, 5 insertions, 0 deletions
diff --git a/test-suite/success/intros.v b/test-suite/success/intros.v index bb9fc0c50..9443d01e3 100644 --- a/test-suite/success/intros.v +++ b/test-suite/success/intros.v @@ -28,3 +28,8 @@ Goal forall n p, n + p = 0. intros [|*]; intro p. Abort. +(* Check non-interference of "_" with name generation *) +Goal True -> True -> True. +intros _ ?. +exact H. +Qed. |