aboutsummaryrefslogtreecommitdiff
path: root/ci/test1.v
diff options
context:
space:
mode:
authorCyril Anaclet2020-05-04 11:24:20 +0200
committerCyril Anaclet2020-05-04 11:24:20 +0200
commit866a9da96a53c387050e7d8f7df9a0a3e35b435f (patch)
treefafeba08cc9f0569576b786c1d422044ea533296 /ci/test1.v
parent31108dc120285765142b2bb4f44f34febbe79188 (diff)
test: Add tests and some fix
Diffstat (limited to 'ci/test1.v')
-rw-r--r--ci/test1.v14
1 files changed, 12 insertions, 2 deletions
diff --git a/ci/test1.v b/ci/test1.v
index fc1fc943..3812adbd 100644
--- a/ci/test1.v
+++ b/ci/test1.v
@@ -1,7 +1,7 @@
Definition trois := 3. (*test-definition*)
Print trois.
Eval compute in 10 * trois * trois.
-
+
Lemma easy_proof : forall A : Prop, A -> A.
@@ -9,4 +9,14 @@ Proof using .
intros A.
intros proof_of_A. (*test-insert*)
exact proof_of_A.
-Qed. (*test-lemma*)
+Qed. (*test-lemma*)
+
+Lemma false_proof : forall A B : bool, A = B.
+Proof.
+ intros A B.
+ destruct A.
+ destruct B.
+ reflexivity. (*error*)
+ reflexivity.
+Qed. (*test-lemma2*)
+