From a85dc414e57265444b0d8623bcafe15f49179ee4 Mon Sep 17 00:00:00 2001 From: Paul Steckler Date: Tue, 3 Oct 2017 16:33:14 -0400 Subject: add coqwc tests --- test-suite/coqwc/BZ5637.out | 2 ++ test-suite/coqwc/BZ5637.v | 5 +++++ test-suite/coqwc/BZ5756.out | 2 ++ test-suite/coqwc/BZ5756.v | 3 +++ test-suite/coqwc/false.out | 2 ++ test-suite/coqwc/false.v | 8 ++++++++ test-suite/coqwc/next-obligation.out | 2 ++ test-suite/coqwc/next-obligation.v | 10 ++++++++++ test-suite/coqwc/theorem.out | 2 ++ test-suite/coqwc/theorem.v | 10 ++++++++++ 10 files changed, 46 insertions(+) create mode 100644 test-suite/coqwc/BZ5637.out create mode 100644 test-suite/coqwc/BZ5637.v create mode 100644 test-suite/coqwc/BZ5756.out create mode 100644 test-suite/coqwc/BZ5756.v create mode 100644 test-suite/coqwc/false.out create mode 100644 test-suite/coqwc/false.v create mode 100644 test-suite/coqwc/next-obligation.out create mode 100644 test-suite/coqwc/next-obligation.v create mode 100644 test-suite/coqwc/theorem.out create mode 100644 test-suite/coqwc/theorem.v (limited to 'test-suite/coqwc') diff --git a/test-suite/coqwc/BZ5637.out b/test-suite/coqwc/BZ5637.out new file mode 100644 index 000000000..f0b5e4f7e --- /dev/null +++ b/test-suite/coqwc/BZ5637.out @@ -0,0 +1,2 @@ + spec proof comments + 5 0 0 coqwc/BZ5637.v diff --git a/test-suite/coqwc/BZ5637.v b/test-suite/coqwc/BZ5637.v new file mode 100644 index 000000000..6428b10ff --- /dev/null +++ b/test-suite/coqwc/BZ5637.v @@ -0,0 +1,5 @@ +Local Obligation Tactic := idtac. +Definition a := 1. +Definition b := 1. +Definition c := 1. +Definition d := 1. diff --git a/test-suite/coqwc/BZ5756.out b/test-suite/coqwc/BZ5756.out new file mode 100644 index 000000000..039d1e500 --- /dev/null +++ b/test-suite/coqwc/BZ5756.out @@ -0,0 +1,2 @@ + spec proof comments + 3 0 2 coqwc/BZ5756.v 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. diff --git a/test-suite/coqwc/false.out b/test-suite/coqwc/false.out new file mode 100644 index 000000000..14c5713f6 --- /dev/null +++ b/test-suite/coqwc/false.out @@ -0,0 +1,2 @@ + spec proof comments + 3 3 1 coqwc/false.v diff --git a/test-suite/coqwc/false.v b/test-suite/coqwc/false.v new file mode 100644 index 000000000..640f9ea7f --- /dev/null +++ b/test-suite/coqwc/false.v @@ -0,0 +1,8 @@ +Axiom x : nat. + +Definition foo (x : nat) := x + 1. + +Lemma bar : False. + idtac. + idtac. (* truth is overrated *) +Admitted. diff --git a/test-suite/coqwc/next-obligation.out b/test-suite/coqwc/next-obligation.out new file mode 100644 index 000000000..7a0fd777c --- /dev/null +++ b/test-suite/coqwc/next-obligation.out @@ -0,0 +1,2 @@ + spec proof comments + 1 7 0 coqwc/next-obligation.v diff --git a/test-suite/coqwc/next-obligation.v b/test-suite/coqwc/next-obligation.v new file mode 100644 index 000000000..786df9891 --- /dev/null +++ b/test-suite/coqwc/next-obligation.v @@ -0,0 +1,10 @@ +(* make sure all proof lines are counted *) + +Goal True. + Next Obligation. + idtac. + Next Obligation. + idtac. + Next Obligation. + idtac. +Qed. diff --git a/test-suite/coqwc/theorem.out b/test-suite/coqwc/theorem.out new file mode 100644 index 000000000..d01507bf7 --- /dev/null +++ b/test-suite/coqwc/theorem.out @@ -0,0 +1,2 @@ + spec proof comments + 1 9 2 coqwc/theorem.v diff --git a/test-suite/coqwc/theorem.v b/test-suite/coqwc/theorem.v new file mode 100644 index 000000000..901c9074f --- /dev/null +++ b/test-suite/coqwc/theorem.v @@ -0,0 +1,10 @@ +Theorem foo : True. +Proof. + idtac. (* comment *) + idtac. + idtac. + idtac. (* comment *) + idtac. + idtac. + auto. +Qed. -- cgit v1.2.3