From 85b1c4091e13dec13fe03f28e81b256c60f9f7ef Mon Sep 17 00:00:00 2001 From: Pierre-Marie Pédrot Date: Mon, 10 Jan 2022 14:54:18 +0100 Subject: Adapt w.r.t. coq/coq#15442 (#425) coq/coq#15442 changes the way `Program` names things, to make it uniform w.r.t. the standard naming schema. This commit removes dependencies on the names chosen by `Program`. Should be backwards compatible. Co-authored-by: Xavier Leroy --- common/Events.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'common/Events.v') diff --git a/common/Events.v b/common/Events.v index c4a6e7f9..0ada1207 100644 --- a/common/Events.v +++ b/common/Events.v @@ -198,7 +198,7 @@ Next Obligation. elimtype False. elim NE. auto. Qed. Next Obligation. - red; intro. elim (H e). rewrite H0. auto. + red; intro; subst; intuition eauto. Qed. CoFixpoint traceinf_of_traceinf' (T': traceinf') : traceinf := -- cgit