aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Cases.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-04-27 16:04:07 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-04-28 09:40:46 +0200
commit9eaf502657ae63f6b184d527eaf1c3b40be90a79 (patch)
tree876aeebf7ccfee4837acc91a4f4acd95bf26e7b9 /test-suite/output/Cases.v
parent5eb53b5bc8d765ed75e965f43f1084e18efc8790 (diff)
Fixing #3293 (eta-expansion at "match" printing time was failing
because of let-in's interpreted as being part of the expansion).
Diffstat (limited to 'test-suite/output/Cases.v')
-rw-r--r--test-suite/output/Cases.v14
1 files changed, 14 insertions, 0 deletions
diff --git a/test-suite/output/Cases.v b/test-suite/output/Cases.v
index 505418b14..30ef8778d 100644
--- a/test-suite/output/Cases.v
+++ b/test-suite/output/Cases.v
@@ -58,3 +58,17 @@ Definition foo' :=
Print foo'.
+(* Was bug #3293 (eta-expansion at "match" printing time was failing because
+ of let-in's interpreted as being part of the expansion) *)
+
+Variable b : bool.
+Variable P : bool -> Prop.
+Inductive B : Prop := AC : P b -> B.
+Definition f : B -> True.
+
+Proof.
+intros [].
+destruct b as [|] ; intros _ ; exact Logic.I.
+Defined.
+
+Print f.