aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3287.v
diff options
context:
space:
mode:
authorGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2017-07-27 14:20:11 +0200
committerGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2017-07-27 15:08:36 +0200
commit036acae205ff0477dbae3a97b44853dc27d03b93 (patch)
tree938a980befb0ec2c30d43473ae511cad01819459 /test-suite/bugs/closed/3287.v
parent87130496c04dc393e32837f1ce95e463938b2202 (diff)
test-suite: more use of the new command Extraction TestCompile
Diffstat (limited to 'test-suite/bugs/closed/3287.v')
-rw-r--r--test-suite/bugs/closed/3287.v9
1 files changed, 3 insertions, 6 deletions
diff --git a/test-suite/bugs/closed/3287.v b/test-suite/bugs/closed/3287.v
index 1b758acd7..4b3e7ff05 100644
--- a/test-suite/bugs/closed/3287.v
+++ b/test-suite/bugs/closed/3287.v
@@ -6,6 +6,7 @@ Definition bar := true.
End Foo.
Recursive Extraction Foo.bar.
+Extraction TestCompile Foo.bar.
Module Foo'.
Definition foo := (I,I).
@@ -13,10 +14,6 @@ Definition bar := true.
End Foo'.
Recursive Extraction Foo'.bar.
+Extraction TestCompile Foo'.bar.
-Module Foo''.
-Definition foo := (I,I).
-Definition bar := true.
-End Foo''.
-
-Extraction Foo.bar.
+Extraction Foo'.bar.