aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Cases.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-11-10 18:43:07 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-11-10 19:00:00 +0100
commitf0ff590f380fb3d9fac6ebfdd6cfd7bf6874658e (patch)
treee67a26401e465a9ab75d029b8ee680868fa36c6a /test-suite/output/Cases.v
parente67760138af866b788db7b43a8e93c5f65a9a84e (diff)
Updating test-suite after Bracketing Last Introduction Pattern set by
default. Interestingly, there is an example where it makes the rest of the proof less natural. Goal forall x y:Z, ... intros [y|p1[|p2|p2]|p1[|p2|p2]]. where case analysis on y is not only in the 2nd and 3rd case, is not anymore easy to do. Still, I find the bracketing of intro-patterns a natural property, and its generalization in all situations a natural expectation for uniformity. So, what to do? The following is e.g. not as compact and "one-shot": intros [|p1|p1]; [intros y|intros [|p2|p2] ..].
Diffstat (limited to 'test-suite/output/Cases.v')
-rw-r--r--test-suite/output/Cases.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/output/Cases.v b/test-suite/output/Cases.v
index 4116a5ebc..a95b085ac 100644
--- a/test-suite/output/Cases.v
+++ b/test-suite/output/Cases.v
@@ -73,7 +73,7 @@ Definition f : B -> True.
Proof.
intros [].
-destruct b as [|] ; intros _ ; exact Logic.I.
+destruct b as [|] ; exact Logic.I.
Defined.
Print f.