aboutsummaryrefslogtreecommitdiffstats
path: root/common/Events.v
diff options
context:
space:
mode:
authorPierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2022-12-22 16:20:15 +0100
committerGitHub <noreply@github.com>2022-12-22 16:20:15 +0100
commitfc79b13a30f124e9ac2d658773c395e0a74e2d1e (patch)
treef81eb0494f192d3abe40c7ce50a4bf77c9596766 /common/Events.v
parent8d21a7fa245637b684ddb4c12f4bfa6295569fb6 (diff)
downloadcompcert-fc79b13a30f124e9ac2d658773c395e0a74e2d1e.tar.gz
compcert-fc79b13a30f124e9ac2d658773c395e0a74e2d1e.zip
Use `exfalso` instead of `elimtype False` (#470)
Adapt w.r.t. coq/coq#16904.
Diffstat (limited to 'common/Events.v')
-rw-r--r--common/Events.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/common/Events.v b/common/Events.v
index 2e076523..1b70ecd6 100644
--- a/common/Events.v
+++ b/common/Events.v
@@ -199,7 +199,7 @@ Program Definition split_traceinf' (t: trace) (T: traceinf') (NE: t <> E0): even
| e :: t' => (e, Econsinf' t' T _)
end.
Next Obligation.
- elimtype False. elim NE. auto.
+ exfalso. elim NE. auto.
Qed.
Next Obligation.
red; intro; subst; intuition eauto.