aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/coqwc/BZ5756.v
diff options
context:
space:
mode:
authorGravatar Paul Steckler <steck@stecksoft.com>2017-10-03 16:33:14 -0400
committerGravatar Paul Steckler <steck@stecksoft.com>2017-10-03 16:33:14 -0400
commita85dc414e57265444b0d8623bcafe15f49179ee4 (patch)
tree3a95a8edb43f1ed8637fc240114f819b458633d6 /test-suite/coqwc/BZ5756.v
parentb9740771e8113cb9e607793887be7a12587d0326 (diff)
add coqwc tests
Diffstat (limited to 'test-suite/coqwc/BZ5756.v')
-rw-r--r--test-suite/coqwc/BZ5756.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/test-suite/coqwc/BZ5756.v b/test-suite/coqwc/BZ5756.v
new file mode 100644
index 000000000..ccb12076a
--- /dev/null
+++ b/test-suite/coqwc/BZ5756.v
@@ -0,0 +1,3 @@
+Definition myNextValue := 0. (* OK *)
+Definition x := myNextValue. (* not OK *)
+Definition y := 0.