summaryrefslogtreecommitdiff
path: root/test-suite/modules/Tescik.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/modules/Tescik.v')
-rw-r--r--test-suite/modules/Tescik.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/test-suite/modules/Tescik.v b/test-suite/modules/Tescik.v
index 8dadace7..1d1b1e0a 100644
--- a/test-suite/modules/Tescik.v
+++ b/test-suite/modules/Tescik.v
@@ -7,20 +7,20 @@ End ELEM.
Module Nat.
Definition A := nat.
Definition x := 0.
-End Nat.
+End Nat.
Module List (X: ELEM).
Inductive list : Set :=
| nil : list
| cons : X.A -> list -> list.
-
+
Definition head (l : list) := match l with
| nil => X.x
| cons x _ => x
end.
Definition singl (x : X.A) := cons x nil.
-
+
Lemma head_singl : forall x : X.A, head (singl x) = x.
auto.
Qed.