From 6faef9c38104c09ce1a6e7db2589a746484ecfb4 Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Wed, 7 Mar 2018 11:17:49 -0500 Subject: Add empty compat file for Coq 8.8 This closes #6598 --- doc/stdlib/index-list.html.template | 1 + theories/Compat/Coq87.v | 1 + theories/Compat/Coq88.v | 11 +++++++++++ 3 files changed, 13 insertions(+) create mode 100644 theories/Compat/Coq88.v diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template index a2739e457..8c09b23a5 100644 --- a/doc/stdlib/index-list.html.template +++ b/doc/stdlib/index-list.html.template @@ -598,5 +598,6 @@ through the Require Import command.

theories/Compat/AdmitAxiom.v theories/Compat/Coq86.v theories/Compat/Coq87.v + theories/Compat/Coq88.v diff --git a/theories/Compat/Coq87.v b/theories/Compat/Coq87.v index 89556ee75..dc1397aff 100644 --- a/theories/Compat/Coq87.v +++ b/theories/Compat/Coq87.v @@ -9,6 +9,7 @@ (************************************************************************) (** Compatibility file for making Coq act similar to Coq v8.7 *) +Require Export Coq.Compat.Coq88. (* In 8.7, omega wasn't taking advantage of local abbreviations, see bug 148 and PR#768. For adjusting this flag, we're forced to diff --git a/theories/Compat/Coq88.v b/theories/Compat/Coq88.v new file mode 100644 index 000000000..4142af05d --- /dev/null +++ b/theories/Compat/Coq88.v @@ -0,0 +1,11 @@ +(************************************************************************) +(* * The Coq Proof Assistant / The Coq Development Team *) +(* v * INRIA, CNRS and contributors - Copyright 1999-2018 *) +(*