Skip to content

Commit e678d71

Browse files
committed
Add Makefile for compat
1 parent 3dd7511 commit e678d71

File tree

2 files changed

+8
-6
lines changed

2 files changed

+8
-6
lines changed

Make.compat

+7
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,7 @@
1+
theories/Compat/AdmitAxiom.v
2+
theories/Compat/Coq818.v
3+
theories/Compat/Coq819.v
4+
theories/Compat/Coq820.v
5+
theories/Compat/Coq821.v
6+
7+
-Q theories/Compat Stdlib.Compat

doc/stdlib/index-list.html.template

+1-6
Original file line numberDiff line numberDiff line change
@@ -680,14 +680,9 @@ through the <tt>Require Import</tt> command.</p>
680680
theories/Wellfounded/Well_Ordering.v
681681
</dd>
682682

683-
<dt> <b>Setoids</b>:
684-
</dt>
685-
<dd>
686-
theories/Setoids/Setoid.v
687-
</dd>
688-
689683
<dt> <b>Compat</b>:
690684
Compatibility wrappers for previous versions of Coq
685+
in namespace Stdlib.Compat.
691686
</dt>
692687
<dd>
693688
theories/Compat/AdmitAxiom.v

0 commit comments

Comments
 (0)