We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
1 parent 3dd7511 commit e678d71Copy full SHA for e678d71
Make.compat
@@ -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
@@ -680,14 +680,9 @@ through the <tt>Require Import</tt> command.</p>
680
theories/Wellfounded/Well_Ordering.v
681
</dd>
682
683
- <dt> <b>Setoids</b>:
684
- </dt>
685
- <dd>
686
- theories/Setoids/Setoid.v
687
- </dd>
688
-
689
<dt> <b>Compat</b>:
690
Compatibility wrappers for previous versions of Coq
+ in namespace Stdlib.Compat.
691
</dt>
692
<dd>
693
theories/Compat/AdmitAxiom.v
0 commit comments