aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2015-12-14 20:29:45 +0100
committerGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2015-12-14 20:29:45 +0100
commitc3aa4c065fac0e37d67ca001aec47b1c2138e648 (patch)
tree51f3ef627076a179aeb48c22d7d0deed4e28acc8
parent6ab322a9b0725aaa9fa6f457db061f2635598fe9 (diff)
extraction_impl.v: fix a typo
-rw-r--r--test-suite/success/extraction_impl.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/success/extraction_impl.v b/test-suite/success/extraction_impl.v
index a72715f29..dfdeff82f 100644
--- a/test-suite/success/extraction_impl.v
+++ b/test-suite/success/extraction_impl.v
@@ -64,7 +64,7 @@ Fixpoint enat_nat' n (e:enat n) : nat :=
end.
Extraction Implicit enat_nat' [n].
-Recursive Extraction enat_nat.
+Recursive Extraction enat_nat'.
(** Bug #4228 *)