aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/dp/test2.v
diff options
context:
space:
mode:
Diffstat (limited to 'plugins/dp/test2.v')
-rw-r--r--plugins/dp/test2.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/plugins/dp/test2.v b/plugins/dp/test2.v
index 3e4c0f6dd..0940b1352 100644
--- a/plugins/dp/test2.v
+++ b/plugins/dp/test2.v
@@ -36,7 +36,7 @@ Goal fct O = O.
Admitted.
Fixpoint even (n:nat) : Prop :=
- match n with
+ match n with
O => True
| S O => False
| S (S p) => even p
@@ -64,9 +64,9 @@ BUG avec head prédéfini : manque eta-expansion sur A:Set
Goal forall x, head _ (p _ _ 1 2) = Some x -> fst x = 1.
-Print value.
+Print value.
Print Some.
-
+
zenon.
*)