Skip to content

Commit

Permalink
Start a GoodDefaults file collecting recommended option settings.
Browse files Browse the repository at this point in the history
  • Loading branch information
Zimmi48 committed May 30, 2024
1 parent c67f36d commit 3218c65
Show file tree
Hide file tree
Showing 2 changed files with 16 additions and 1 deletion.
3 changes: 2 additions & 1 deletion doc/stdlib/index-list.html.template
Original file line number Diff line number Diff line change
Expand Up @@ -696,13 +696,14 @@ through the <tt>Require Import</tt> command.</p>
</dd>

<dt> <b>Compat</b>:
Compatibility wrappers for previous versions of Coq
Compatibility wrappers for previous versions of Coq and recommended options at the time of a given Coq release
</dt>
<dd>
theories/Compat/AdmitAxiom.v
theories/Compat/Coq818.v
theories/Compat/Coq819.v
theories/Compat/Coq820.v
theories/Compat/GoodDefaults_8_20.v
user-contrib/Ltac2/Compat/Coq818.v
user-contrib/Ltac2/Compat/Coq819.v
</dd>
Expand Down
14 changes: 14 additions & 0 deletions theories/Compat/GoodDefaults_8_20.v
Original file line number Diff line number Diff line change
@@ -0,0 +1,14 @@
(************************************************************************)
(* * 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) *)
(************************************************************************)

(** File exporting recommended option settings at the time of releasing Coq v8.20 *)


#[ export ] Set Default Goal Selector "!".

0 comments on commit 3218c65

Please sign in to comment.