diff options
author | Enrico Tassi <Enrico.Tassi@inria.fr> | 2016-06-06 05:50:07 -0400 |
---|---|---|
committer | Enrico Tassi <Enrico.Tassi@inria.fr> | 2016-06-06 14:04:33 -0400 |
commit | e4d66a03148243f7611f4d7c164e775877184e03 (patch) | |
tree | 0a2581fd31dc3603db6e333de365f230354544a2 /test-suite | |
parent | 0307140281395e8ffa16f2af9f946cc53d540b17 (diff) |
Error box detection run only on error
Advantage: 0 cost if no error occurs
Disadvantage: a box *must* end with the error absorbing command
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/interactive/proof_block.v | 12 |
1 files changed, 11 insertions, 1 deletions
diff --git a/test-suite/interactive/proof_block.v b/test-suite/interactive/proof_block.v index ff920b671..31e349376 100644 --- a/test-suite/interactive/proof_block.v +++ b/test-suite/interactive/proof_block.v @@ -1,3 +1,13 @@ +Goal False /\ True. +Proof. +split. + idtac. + idtac. + exact I. +idtac. +idtac. +exact I. +Qed. Lemma baz : (exists n, n = 3 /\ n = 3) /\ True. Proof. @@ -26,7 +36,7 @@ Qed. Lemma foo1 : False /\ True. Proof. split. - exact I. + { exact I. } { exact I. } Qed. |