diff options
| author | Hendrik Tews | 2021-03-19 20:54:47 +0100 |
|---|---|---|
| committer | Hendrik Tews | 2021-04-16 22:53:05 +0200 |
| commit | 3802db410447bbc27e50dc5461b055c4e12a7e9a (patch) | |
| tree | f77e8e60ef2d85101e16e27889afbcd15a0db3d8 /ci/simple-tests/omit_test.v | |
| parent | f7943ba646c258a0a4a5b397b8a920d5d13ecf31 (diff) | |
add test for omit proofs feature
Diffstat (limited to 'ci/simple-tests/omit_test.v')
| -rw-r--r-- | ci/simple-tests/omit_test.v | 25 |
1 files changed, 25 insertions, 0 deletions
diff --git a/ci/simple-tests/omit_test.v b/ci/simple-tests/omit_test.v new file mode 100644 index 00000000..b8d177cc --- /dev/null +++ b/ci/simple-tests/omit_test.v @@ -0,0 +1,25 @@ + +Definition classical_logic : Prop := forall(P : Prop), ~~P -> P. + +(* automatic test marker 1 *) + +Lemma classic_excluded_middle : + (forall(P : Prop), P \/ ~ P) -> classical_logic. +Proof. + intros H P H0. + (* automatic test marker 2 *) + specialize (H P). +Abort. + +Lemma classic_excluded_middle : + (forall(P : Prop), P \/ ~ P) -> classical_logic. +Proof using. + intros H P H0. + specialize (H P). + (* automatic test marker 3 *) + destruct H. + trivial. + contradiction. +Qed. + +(* automatic test marker 4 *) |
