Skip to content

Commit

Permalink
Add links to refman in test files
Browse files Browse the repository at this point in the history
The goal is to ease maintenance if one of the test files fails following
a change in some command behaviour regarding locality.
  • Loading branch information
Villetaneuse committed Aug 5, 2024
1 parent 7d93822 commit e287e41
Show file tree
Hide file tree
Showing 5 changed files with 88 additions and 5 deletions.
18 changes: 17 additions & 1 deletion test-suite/success/locality_attributes_modules.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,23 @@
(** This file tests how locality attributes affect usual vernacular commands.
PLEASE, when this file fails to compute following a voluntary change in
Coq's behaviour, modify accordingly the tables in [sections.rst] and
[modules.rst] in [doc/sphinx/language/core] *)
[modules.rst] in [doc/sphinx/language/core].
Also look at the corresponding discussions about locality attributes in the
refman (directory doc/sphinx)
- For Definition, Lemma, ..., look at language/core/definitions.rst
- For Axiom, Conjecture, ..., look at language/core/assumptions.rst
- For abbreviations, look at user-extensions/syntax-extensions.rst
- For Notations, look at user-extensions/syntax-extensions.rst
- For Tactic Notations, look at user-extensions/syntax-extensions.rst
- For Ltac, look at proof-engine/ltac.rst
- For Canonical Structures, look at language/extensions/canonical.rst
- For Hints, look at proofs/automatic-tactics/auto.rst
- For Coercions, look at addendum/implicit-coercions.rst
- For Ltac2, look at proof-engine/ltac2.rst
- For Ltac2 Notations, look at proof-engine/ltac2.rst
- For Set, look at language/core/basic.rst
*)

(** This structure is used to test availability or not of a
[Canonical Structure]. *)
Expand Down
18 changes: 17 additions & 1 deletion test-suite/success/locality_attributes_modules_ltac2.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,23 @@
(** This file tests how locality attributes affect usual vernacular commands.
PLEASE, when this file fails to compute following a voluntary change in
Coq's behaviour, modify accordingly the tables in [sections.rst] and
[modules.rst] in [doc/sphinx/language/core] *)
[modules.rst] in [doc/sphinx/language/core]
Also look at the corresponding discussions about locality attributes in the
refman (directory doc/sphinx)
- For Definition, Lemma, ..., look at language/core/definitions.rst
- For Axiom, Conjecture, ..., look at language/core/assumptions.rst
- For abbreviations, look at user-extensions/syntax-extensions.rst
- For Notations, look at user-extensions/syntax-extensions.rst
- For Tactic Notations, look at user-extensions/syntax-extensions.rst
- For Ltac, look at proof-engine/ltac.rst
- For Canonical Structures, look at language/extensions/canonical.rst
- For Hints, look at proofs/automatic-tactics/auto.rst
- For Coercions, look at addendum/implicit-coercions.rst
- For Ltac2, look at proof-engine/ltac2.rst
- For Ltac2 Notations, look at proof-engine/ltac2.rst
- For Set, look at language/core/basic.rst
*)

From Ltac2 Require Import Ltac2.

Expand Down
19 changes: 18 additions & 1 deletion test-suite/success/locality_attributes_sections.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,24 @@
(** This file tests how locality attributes affect usual vernacular commands.
PLEASE, when this file fails to compute following a voluntary change in
Coq's behaviour, modify accordingly the tables in [sections.rst] and
[modules.rst] in [doc/sphinx/language/core] *)
[modules.rst] in [doc/sphinx/language/core].
Also look at the corresponding discussions about locality attributes in the
refman (directory doc/sphinx)
- For Definition, Lemma, ..., look at language/core/definitions.rst
- For Axiom, Conjecture, ..., look at language/core/assumptions.rst
- For abbreviations, look at user-extensions/syntax-extensions.rst
- For Notations, look at user-extensions/syntax-extensions.rst
- For Tactic Notations, look at user-extensions/syntax-extensions.rst
- For Ltac, look at proof-engine/ltac.rst
- For Canonical Structures, look at language/extensions/canonical.rst
- For Hints, look at proofs/automatic-tactics/auto.rst
- For Coercions, look at addendum/implicit-coercions.rst
- For Ltac2, look at proof-engine/ltac2.rst
- For Ltac2 Notations, look at proof-engine/ltac2.rst
- For Set, look at language/core/basic.rst
*)


(** This structure is used to test availability or not of a
[Canonical Structure]. *)
Expand Down
19 changes: 18 additions & 1 deletion test-suite/success/locality_attributes_sections_in_modules.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,24 @@
(** This file tests how locality attributes affect usual vernacular commands.
PLEASE, when this file fails to compute following a voluntary change in
Coq's behaviour, modify accordingly the tables in [sections.rst] and
[modules.rst] in [doc/sphinx/language/core] *)
[modules.rst] in [doc/sphinx/language/core].
Also look at the corresponding discussions about locality attributes in the
refman (directory doc/sphinx)
- For Definition, Lemma, ..., look at language/core/definitions.rst
- For Axiom, Conjecture, ..., look at language/core/assumptions.rst
- For abbreviations, look at user-extensions/syntax-extensions.rst
- For Notations, look at user-extensions/syntax-extensions.rst
- For Tactic Notations, look at user-extensions/syntax-extensions.rst
- For Ltac, look at proof-engine/ltac.rst
- For Canonical Structures, look at language/extensions/canonical.rst
- For Hints, look at proofs/automatic-tactics/auto.rst
- For Coercions, look at addendum/implicit-coercions.rst
- For Ltac2, look at proof-engine/ltac2.rst
- For Ltac2 Notations, look at proof-engine/ltac2.rst
- For Set, look at language/core/basic.rst
*)


(** This structure is used to test availability or not of a
[Canonical Structure]. *)
Expand Down
19 changes: 18 additions & 1 deletion test-suite/success/locality_attributes_sections_ltac2.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,24 @@
(** This file tests how locality attributes affect usual vernacular commands.
PLEASE, when this file fails to compute following a voluntary change in
Coq's behaviour, modify accordingly the tables in [sections.rst] and
[modules.rst] in [doc/sphinx/language/core] *)
[modules.rst] in [doc/sphinx/language/core].
Also look at the corresponding discussions about locality attributes in the
refman (directory doc/sphinx)
- For Definition, Lemma, ..., look at language/core/definitions.rst
- For Axiom, Conjecture, ..., look at language/core/assumptions.rst
- For abbreviations, look at user-extensions/syntax-extensions.rst
- For Notations, look at user-extensions/syntax-extensions.rst
- For Tactic Notations, look at user-extensions/syntax-extensions.rst
- For Ltac, look at proof-engine/ltac.rst
- For Canonical Structures, look at language/extensions/canonical.rst
- For Hints, look at proofs/automatic-tactics/auto.rst
- For Coercions, look at addendum/implicit-coercions.rst
- For Ltac2, look at proof-engine/ltac2.rst
- For Ltac2 Notations, look at proof-engine/ltac2.rst
- For Set, look at language/core/basic.rst
*)


From Ltac2 Require Import Ltac2.

Expand Down

0 comments on commit e287e41

Please sign in to comment.