diff options
author | Enrico Tassi <Enrico.Tassi@inria.fr> | 2016-05-23 16:57:31 +0200 |
---|---|---|
committer | Enrico Tassi <Enrico.Tassi@inria.fr> | 2016-06-06 14:04:33 -0400 |
commit | 821937aee71bf9439158e27e06f7b4f74289b209 (patch) | |
tree | 7e06be2dbbfd3c7168a6056b4a198bad44bab1f3 /test-suite | |
parent | 8baf120d5cf5045d188f7d926162643a6e7ebcd0 (diff) |
STM: proof block detection made optional + simple test
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/interactive/proof_block.v | 56 |
1 files changed, 56 insertions, 0 deletions
diff --git a/test-suite/interactive/proof_block.v b/test-suite/interactive/proof_block.v new file mode 100644 index 000000000..ff920b671 --- /dev/null +++ b/test-suite/interactive/proof_block.v @@ -0,0 +1,56 @@ + +Lemma baz : (exists n, n = 3 /\ n = 3) /\ True. +Proof. +split. { eexists. split. par: trivial. } +trivial. +Qed. + +Lemma baz1 : (True /\ False) /\ True. +Proof. +split. { split. par: trivial. } +trivial. +Qed. + +Lemma foo : (exists n, n = 3 /\ n = 3) /\ True. +Proof. +split. + { idtac. + unshelve eexists. + { apply 3. } + { split. + { idtac. trivialx. } + { reflexivity. } } } + trivial. +Qed. + +Lemma foo1 : False /\ True. +Proof. +split. + exact I. + { exact I. } +Qed. + +Definition banana := true + 4. + +Check banana. + +Lemma bar : (exists n, n = 3 /\ n = 3) /\ True. +Proof. +split. + - idtac. + unshelve eexists. + + apply 3. + + split. + * idtacx. trivial. + * reflexivity. + - trivial. +Qed. + +Lemma baz2 : ((1=0 /\ False) /\ True) /\ False. +Proof. +split. split. split. + - solve [ auto ]. + - solve [ trivial ]. + - solve [ trivial ]. + - exact 6. +Qed.
\ No newline at end of file |