Skip to content

Commit

Permalink
Merge PR coq#18319: Bump version (8.20+alpha)
Browse files Browse the repository at this point in the history
Reviewed-by: ppedrot
Co-authored-by: ppedrot <[email protected]>
  • Loading branch information
coqbot-app[bot] and ppedrot authored Dec 4, 2023
2 parents 89a5cee + 1d38647 commit ababbf4
Show file tree
Hide file tree
Showing 10 changed files with 30 additions and 9 deletions.
1 change: 1 addition & 0 deletions doc/stdlib/index-list.html.template
Original file line number Diff line number Diff line change
Expand Up @@ -716,6 +716,7 @@ through the <tt>Require Import</tt> command.</p>
theories/Compat/Coq817.v
theories/Compat/Coq818.v
theories/Compat/Coq819.v
theories/Compat/Coq820.v
</dd>

<dt> <b>Array</b>:
Expand Down
1 change: 1 addition & 0 deletions sysinit/coqargs.ml
Original file line number Diff line number Diff line change
Expand Up @@ -227,6 +227,7 @@ let set_option = let open Goptions in function
| opt, OptionAppend v -> set_string_option_append_value_gen ~locality:OptLocal opt v

let get_compat_file = function
| "8.20" -> "Coq.Compat.Coq820"
| "8.19" -> "Coq.Compat.Coq819"
| "8.18" -> "Coq.Compat.Coq818"
| "8.17" -> "Coq.Compat.Coq817"
Expand Down
4 changes: 2 additions & 2 deletions test-suite/success/CompatCurrentFlag.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,3 @@
(* -*- coq-prog-args: ("-compat" "8.19") -*- *)
(* -*- coq-prog-args: ("-compat" "8.20") -*- *)
(** Check that the current compatibility flag actually requires the relevant modules. *)
Import Coq.Compat.Coq819.
Import Coq.Compat.Coq820.
4 changes: 2 additions & 2 deletions test-suite/success/CompatOldFlag.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
(* -*- coq-prog-args: ("-compat" "8.17") -*- *)
(* -*- coq-prog-args: ("-compat" "8.18") -*- *)
(** Check that the current-minus-two compatibility flag actually requires the relevant modules. *)
Import Coq.Compat.Coq820.
Import Coq.Compat.Coq819.
Import Coq.Compat.Coq818.
Import Coq.Compat.Coq817.
6 changes: 6 additions & 0 deletions test-suite/success/CompatOldOldFlag.v
Original file line number Diff line number Diff line change
@@ -0,0 +1,6 @@
(* -*- coq-prog-args: ("-compat" "8.17") -*- *)
(** Check that the current-minus-three compatibility flag actually requires the relevant modules. *)
Import Coq.Compat.Coq820.
Import Coq.Compat.Coq819.
Import Coq.Compat.Coq818.
Import Coq.Compat.Coq817.
4 changes: 2 additions & 2 deletions test-suite/success/CompatPreviousFlag.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
(* -*- coq-prog-args: ("-compat" "8.18") -*- *)
(* -*- coq-prog-args: ("-compat" "8.19") -*- *)
(** Check that the current-minus-one compatibility flag actually requires the relevant modules. *)
Import Coq.Compat.Coq820.
Import Coq.Compat.Coq819.
Import Coq.Compat.Coq818.
2 changes: 1 addition & 1 deletion test-suite/tools/update-compat/run.sh
Original file line number Diff line number Diff line change
Expand Up @@ -6,4 +6,4 @@ SCRIPT_DIR="$( cd "$( dirname "${BASH_SOURCE[0]}" )" >/dev/null && pwd )"
# we assume that the script lives in test-suite/tools/update-compat/,
# and that update-compat.py lives in dev/tools/
cd "${SCRIPT_DIR}/../../.."
dev/tools/update-compat.py --assert-unchanged --release || exit $?
dev/tools/update-compat.py --assert-unchanged --master || exit $?
2 changes: 2 additions & 0 deletions theories/Compat/Coq819.v
Original file line number Diff line number Diff line change
Expand Up @@ -9,3 +9,5 @@
(************************************************************************)

(** Compatibility file for making Coq act similar to Coq v8.19 *)

Require Export Coq.Compat.Coq820.
11 changes: 11 additions & 0 deletions theories/Compat/Coq820.v
Original file line number Diff line number Diff line change
@@ -0,0 +1,11 @@
(************************************************************************)
(* * The Coq Proof Assistant / The Coq Development Team *)
(* v * Copyright INRIA, CNRS and contributors *)
(* <O___,, * (see version control and CREDITS file for authors & dates) *)
(* \VV/ **************************************************************)
(* // * This file is distributed under the terms of the *)
(* * GNU Lesser General Public License Version 2.1 *)
(* * (see LICENSE file for the text of the license) *)
(************************************************************************)

(** Compatibility file for making Coq act similar to Coq v8.20 *)
4 changes: 2 additions & 2 deletions tools/configure/configure.ml
Original file line number Diff line number Diff line change
Expand Up @@ -22,8 +22,8 @@ open CmdArgs.Prefs

let (/) = Filename.concat

let coq_version = "8.19+alpha"
let vo_magic = 81899
let coq_version = "8.20+alpha"
let vo_magic = 81999
let is_a_released_version = false

(** Default OCaml binaries *)
Expand Down

0 comments on commit ababbf4

Please sign in to comment.