aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/subtac/test/Mutind.v
diff options
context:
space:
mode:
Diffstat (limited to 'plugins/subtac/test/Mutind.v')
-rw-r--r--plugins/subtac/test/Mutind.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/plugins/subtac/test/Mutind.v b/plugins/subtac/test/Mutind.v
index ac49ca96a..01e2d75f3 100644
--- a/plugins/subtac/test/Mutind.v
+++ b/plugins/subtac/test/Mutind.v
@@ -1,11 +1,11 @@
Require Import List.
-Program Fixpoint f a : { x : nat | x > 0 } :=
+Program Fixpoint f a : { x : nat | x > 0 } :=
match a with
| 0 => 1
| S a' => g a a'
end
-with g a b : { x : nat | x > 0 } :=
+with g a b : { x : nat | x > 0 } :=
match b with
| 0 => 1
| S b' => f b'