Skip to content

Commit

Permalink
Documentation of branch “master” at bf1ada53
Browse files Browse the repository at this point in the history
  • Loading branch information
coqbot committed Jan 21, 2025
1 parent 4fd6f8a commit c5f077c
Show file tree
Hide file tree
Showing 252 changed files with 1,242 additions and 1,195 deletions.
Binary file modified master/refman-stdlib/.doctrees/environment.pickle
Binary file not shown.
Binary file modified master/refman-stdlib/.doctrees/language/coq-library.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/extraction.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/generalized-rewriting.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/implicit-coercions.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/micromega.doctree
Binary file not shown.
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/program.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/rewrite-rules.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/ring.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/sprop.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/type-classes.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/addendum/universe-polymorphism.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/changes.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/environment.pickle
Binary file not shown.
Binary file modified master/refman/.doctrees/language/cic.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/coq-library.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/assumptions.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/basic.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/coinductive.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/conversion.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/inductive.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/modules.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/primitive.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/records.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/sections.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/core/variants.doctree
Binary file not shown.
Binary file not shown.
Binary file modified master/refman/.doctrees/language/extensions/canonical.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/language/extensions/evars.doctree
Binary file not shown.
Binary file not shown.
Binary file modified master/refman/.doctrees/language/extensions/match.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/practical-tools/coq-commands.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/practical-tools/coqide.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/proof-engine/ltac.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/proof-engine/ltac2.doctree
Binary file not shown.
Binary file not shown.
Binary file modified master/refman/.doctrees/proof-engine/tactics.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/proof-engine/vernacular-commands.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/proofs/automatic-tactics/auto.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/proofs/automatic-tactics/logic.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/proofs/writing-proofs/equality.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/proofs/writing-proofs/proof-mode.doctree
Binary file not shown.
Binary file not shown.
Binary file not shown.
Binary file modified master/refman/.doctrees/using/libraries/funind.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/using/libraries/writing.doctree
Binary file not shown.
47 changes: 47 additions & 0 deletions master/refman/_static/coqdoc.css
Original file line number Diff line number Diff line change
Expand Up @@ -70,3 +70,50 @@
.smallcaps {
font-variant: small-caps;
}


:root {
--refman-custom-primary-blue: #260086;
--refman-custom-primary-blue-2: #040b92;
--refman-custom-secondary-orange: #ff540a;
--refman-custom-secondary-orange-2: #ffe9df;
}

.btn-info:hover, a:hover, a.wy-text-info:hover {
color: var(--refman-custom-primary-blue-2) !important
}

.wy-menu-vertical header, .wy-menu-vertical p.caption, .rst-content .wy-alert-neutral.admonition-todo a, .rst-content .wy-alert-neutral.admonition a, .rst-content .wy-alert-neutral.attention a, .rst-content .wy-alert-neutral.caution a, .rst-content .wy-alert-neutral.danger a, .rst-content .wy-alert-neutral.error a, .rst-content .wy-alert-neutral.hint a, .rst-content .wy-alert-neutral.important a, .rst-content .wy-alert-neutral.note a, .rst-content .wy-alert-neutral.seealso a, .rst-content .wy-alert-neutral.tip a, .rst-content .wy-alert-neutral.warning a, .wy-alert.wy-alert-neutral a, a, .wy-text-info, .btn-link, .wy-inline-validate.wy-inline-validate-info .wy-input-context, .wy-nav .wy-menu-vertical header, .rst-versions a, .rst-content a code, .rst-content a tt, html.writer-html4 .rst-content dl:not(.docutils)>dt, html.writer-html5 .rst-content dl[class]:not(.option-list):not(.field-list):not(.footnote):not(.glossary):not(.simple)>dt, html.writer-html4 .rst-content dl:not(.docutils)>dt:before, html.writer-html5 .rst-content dl[class]:not(.option-list):not(.field-list):not(.footnote):not(.glossary):not(.simple)>dt:before {
color: var(--refman-custom-primary-blue) !important
}

.rst-content .note .admonition-title,.rst-content .note .wy-alert-title,.rst-content .seealso .admonition-title,.rst-content .seealso .wy-alert-title,.rst-content .wy-alert-info.admonition-todo .admonition-title,.rst-content .wy-alert-info.admonition-todo .wy-alert-title,.rst-content .wy-alert-info.admonition .admonition-title,.rst-content .wy-alert-info.admonition .wy-alert-title,.rst-content .wy-alert-info.attention .admonition-title,.rst-content .wy-alert-info.attention .wy-alert-title,.rst-content .wy-alert-info.caution .admonition-title,.rst-content .wy-alert-info.caution .wy-alert-title,.rst-content .wy-alert-info.danger .admonition-title,.rst-content .wy-alert-info.danger .wy-alert-title,.rst-content .wy-alert-info.error .admonition-title,.rst-content .wy-alert-info.error .wy-alert-title,.rst-content .wy-alert-info.hint .admonition-title,.rst-content .wy-alert-info.hint .wy-alert-title,.rst-content .wy-alert-info.important .admonition-title,.rst-content .wy-alert-info.important .wy-alert-title,.rst-content .wy-alert-info.tip .admonition-title,.rst-content .wy-alert-info.tip .wy-alert-title,.rst-content .wy-alert-info.warning .admonition-title,.rst-content .wy-alert-info.warning .wy-alert-title,.rst-content .wy-alert.wy-alert-info .admonition-title,.wy-alert.wy-alert-info .rst-content .admonition-title,.wy-alert.wy-alert-info .wy-alert-title {
background: var(--refman-custom-primary-blue) !important
}

html.writer-html4 .rst-content dl:not(.docutils)>dt,html.writer-html5 .rst-content dl[class]:not(.option-list):not(.field-list):not(.footnote):not(.glossary):not(.simple)>dt {
background: var(--refman-custom-secondary-orange-2) !important;
color: var(--refman-custom-primary-blue) !important;
border-top: 3px solid var(--refman-custom-secondary-orange) !important;
}

.wy-tray-container li.wy-tray-item-info, .btn-info, .wy-menu-vertical a:active, .wy-side-nav-search, .wy-dropdown-menu>dd>a:hover, .wy-dropdown.wy-dropdown-bubble .wy-dropdown-menu a:hover, .wy-side-nav-search img, .wy-nav .wy-menu-vertical a:hover, .wy-nav-top, .wy-nav-top img {
background-color: var(--refman-custom-secondary-orange) !important
}

.wy-side-nav-search input[type=text] {
border-color: var(--refman-custom-primary-blue-2) !important
}

.rst-versions, .wy-nav-side {
background: #dedede !important;
}

.wy-side-nav-search>div.version {
color: #dedede !important;
}

.wy-menu-vertical a:hover {
background-color: #494949 !important;
color: #dedede !important;
}
54 changes: 27 additions & 27 deletions master/refman/proof-engine/ltac.html
Original file line number Diff line number Diff line change
Expand Up @@ -4287,44 +4287,44 @@ <h3>Profiling <code class="docutils literal notranslate"><span class="pre">L</sp
</span></dt><dd><span>No more goals.
</span></dd>
<dt><span></span><span class="coqdoc-keyword">Show</span><span> </span><span class="coqdoc-keyword">Ltac</span><span> </span><span class="coqdoc-var">Profile</span><span>.</span><span>
</span></dt><dd><span>total time: 1.271s
</span></dt><dd><span>total time: 2.175s

tactic local total calls max
───────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac -------------------------------------- 0.1% 100.0% 1 1.271s
─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 90.8% 26 0.132s
─&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 90.8% 26 0.132s
─&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.1% 90.7% 26 0.132s
─t_tauto_intuit --------------------------- 0.1% 90.6% 26 0.132s
─&lt;Corelib.Init.Tauto.simplif&gt; ------------- 61.2% 87.4% 26 0.130s
─&lt;Corelib.Init.Tauto.is_conj&gt; ------------- 19.6% 19.6% 28756 0.003s
─lia -------------------------------------- 0.1% 8.8% 28 0.078s
─Zify.zify -------------------------------- 0.3% 7.0% 54 0.077s
─zify_op ---------------------------------- 6.3% 6.3% 54 0.077s
─elim id ---------------------------------- 3.3% 3.3% 650 0.001s
─&lt;Corelib.Init.Tauto.axioms&gt; -------------- 2.3% 3.2% 0 0.004s
─tac -------------------------------------- 0.1% 100.0% 1 2.175s
─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 94.0% 26 0.122s
─&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 93.9% 26 0.122s
─&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.0% 93.9% 26 0.122s
─t_tauto_intuit --------------------------- 0.1% 93.8% 26 0.122s
─&lt;Corelib.Init.Tauto.simplif&gt; ------------- 62.0% 90.3% 26 0.118s
─&lt;Corelib.Init.Tauto.is_conj&gt; ------------- 20.5% 20.5% 28756 0.003s
─lia -------------------------------------- 0.1% 5.7% 28 0.091s
─Zify.zify -------------------------------- 0.3% 4.8% 54 0.090s
─zify_op ---------------------------------- 4.3% 4.3% 54 0.090s
─elim id ---------------------------------- 4.1% 4.1% 650 0.000s
─&lt;Corelib.Init.Tauto.axioms&gt; -------------- 2.5% 3.5% 0 0.005s

tactic local total calls max
─────────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac ---------------------------------------- 0.1% 100.0% 1 1.271s
├─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 90.8% 26 0.132s
│└&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 90.8% 26 0.132s
│└&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.1% 90.7% 26 0.132s
│└t_tauto_intuit --------------------------- 0.1% 90.6% 26 0.132s
│ ├─&lt;Corelib.Init.Tauto.simplif&gt; ----------- 61.2% 87.4% 26 0.130s
│ │ ├─&lt;Corelib.Init.Tauto.is_conj&gt; --------- 19.6% 19.6% 28756 0.003s
│ │ └─elim id ------------------------------ 3.3% 3.3% 650 0.001s
│ └─&lt;Corelib.Init.Tauto.axioms&gt; ------------ 2.3% 3.2% 0 0.004s
└─lia -------------------------------------- 0.1% 8.8% 28 0.078s
└Zify.zify -------------------------------- 0.3% 7.0% 54 0.077s
└zify_op ---------------------------------- 6.3% 6.3% 54 0.077s
─tac ---------------------------------------- 0.1% 100.0% 1 2.175s
├─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 94.0% 26 0.122s
│└&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 93.9% 26 0.122s
│└&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.0% 93.9% 26 0.122s
│└t_tauto_intuit --------------------------- 0.1% 93.8% 26 0.122s
│ ├─&lt;Corelib.Init.Tauto.simplif&gt; ----------- 62.0% 90.3% 26 0.118s
│ │ ├─&lt;Corelib.Init.Tauto.is_conj&gt; --------- 20.5% 20.5% 28756 0.003s
│ │ └─elim id ------------------------------ 4.1% 4.1% 650 0.000s
│ └─&lt;Corelib.Init.Tauto.axioms&gt; ------------ 2.5% 3.5% 0 0.005s
└─lia -------------------------------------- 0.1% 5.7% 28 0.091s
└Zify.zify -------------------------------- 0.3% 4.8% 54 0.090s
└zify_op ---------------------------------- 4.3% 4.3% 54 0.090s
</span></dd>
<dt><span></span><span class="coqdoc-keyword">Show</span><span> </span><span class="coqdoc-keyword">Ltac</span><span> </span><span class="coqdoc-var">Profile</span><span> &quot;lia&quot;.</span><span>
</span></dt><dd><span>total time: 1.271s
</span></dt><dd><span>total time: 2.175s

tactic local total calls max
───────┴──────┴──────┴───────┴─────────┘
─lia -- 0.1% 8.8% 28 0.078s
─lia -- 0.1% 5.7% 28 0.091s

tactic local total calls max
───────┴──────┴──────┴───────┴─────────┘
Expand Down
6 changes: 3 additions & 3 deletions master/refman/proofs/writing-proofs/equality.html
Original file line number Diff line number Diff line change
Expand Up @@ -2641,15 +2641,15 @@ <h3>Computing in a term: eval and Eval<a class="headerlink" href="#computing-in-
True
</span></dd>
<dt><span></span><span class="coqdoc-keyword">Time</span><span> </span><span class="coqdoc-tactic">assert</span><span> (</span><span class="coqdoc-var">id</span><span> (</span><span class="coqdoc-var">fact</span><span> 8) = </span><span class="coqdoc-var">fact</span><span> 8) </span><span class="coqdoc-tactic">by</span><span> </span><span class="coqdoc-tactic">reflexivity</span><span>.</span><span>
</span></dt><dd><span>Finished transaction in 0.151 secs (0.065u,0.085s) (successful)
</span></dt><dd><span>Finished transaction in 0.123 secs (0.082u,0.041s) (successful)
1 goal

H : id (fact 8)</span><span> =</span><span> fact 8
============================
True
</span></dd>
<dt><span></span><span class="coqdoc-keyword">Time</span><span> </span><span class="coqdoc-tactic">assert</span><span> (</span><span class="coqdoc-var">id</span><span> (</span><span class="coqdoc-var">fact</span><span> 9) = </span><span class="coqdoc-var">fact</span><span> 9) </span><span class="coqdoc-tactic">by</span><span> </span><span class="coqdoc-tactic">reflexivity</span><span>.</span><span>
</span></dt><dd><span>Finished transaction in 0.706 secs (0.702u,0.003s) (successful)
</span></dt><dd><span>Finished transaction in 0.591 secs (0.583u,0.008s) (successful)
1 goal

H : id (fact 8)</span><span> =</span><span> fact 8
Expand Down Expand Up @@ -2712,7 +2712,7 @@ <h3>Computing in a term: eval and Eval<a class="headerlink" href="#computing-in-
True
</span></dd>
<dt><span></span><span class="coqdoc-keyword">Time</span><span> </span><span class="coqdoc-tactic">assert</span><span> (</span><span class="coqdoc-var">id</span><span> (</span><span class="coqdoc-var">fact</span><span> 100) = </span><span class="coqdoc-var">fact</span><span> 100) </span><span class="coqdoc-tactic">by</span><span> </span><span class="coqdoc-var">with_strategy</span><span> -1 [</span><span class="coqdoc-var">id</span><span>] </span><span class="coqdoc-tactic">abstract</span><span> </span><span class="coqdoc-tactic">reflexivity</span><span>.</span><span>
</span></dt><dd><span>Finished transaction in 0.002 secs (0.002u,0.s) (successful)
</span></dt><dd><span>Finished transaction in 0.001 secs (0.001u,0.s) (successful)
1 goal

H : id (fact 100)</span><span> =</span><span> fact 100
Expand Down
2 changes: 1 addition & 1 deletion master/refman/searchindex.js

Large diffs are not rendered by default.

4 changes: 2 additions & 2 deletions master/stdlib/Stdlib.Arith.Arith_base.html
Original file line number Diff line number Diff line change
Expand Up @@ -57,7 +57,7 @@ <h1 class="libtitle">Library Stdlib.Arith.Arith_base</h1>
</div>

<div class="doc">
<a id="lab17"></a><h1 class="section"><span class="inlinecode"><span class="id" title="var">arith</span></span> hint database</h1>
<a id="lab1"></a><h1 class="section"><span class="inlinecode"><span class="id" title="var">arith</span></span> hint database</h1>

</div>
<div class="code">
Expand All @@ -79,7 +79,7 @@ <h1 class="libtitle">Library Stdlib.Arith.Arith_base</h1>
</div>

<div class="doc">
<a id="lab18"></a><h2 class="section"><span class="inlinecode"><span class="id" title="var">lt</span></span> and <span class="inlinecode"><span class="id" title="var">le</span></span></h2>
<a id="lab2"></a><h2 class="section"><span class="inlinecode"><span class="id" title="var">lt</span></span> and <span class="inlinecode"><span class="id" title="var">le</span></span></h2>

</div>
<div class="code">
Expand Down
2 changes: 1 addition & 1 deletion master/stdlib/Stdlib.Arith.EqNat.html
Original file line number Diff line number Diff line change
Expand Up @@ -55,7 +55,7 @@ <h1 class="libtitle">Library Stdlib.Arith.EqNat</h1>
Equality on natural numbers
<div class="paragraph"> </div>

<a id="lab1"></a><h1 class="section">Propositional equality</h1>
<a id="lab18"></a><h1 class="section">Propositional equality</h1>

</div>
<div class="code">
Expand Down
30 changes: 15 additions & 15 deletions master/stdlib/Stdlib.Arith.PeanoNat.html
Original file line number Diff line number Diff line change
Expand Up @@ -148,7 +148,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab2"></a><h2 class="section">Remaining constants not defined in Stdlib.Init.Nat</h2>
<a id="lab3"></a><h2 class="section">Remaining constants not defined in Stdlib.Init.Nat</h2>

<div class="paragraph"> </div>

Expand All @@ -166,7 +166,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab3"></a><h2 class="section">Basic specifications : pred add sub mul</h2>
<a id="lab4"></a><h2 class="section">Basic specifications : pred add sub mul</h2>

</div>
<div class="code">
Expand Down Expand Up @@ -208,7 +208,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab4"></a><h2 class="section">Boolean comparisons</h2>
<a id="lab5"></a><h2 class="section">Boolean comparisons</h2>

</div>
<div class="code">
Expand Down Expand Up @@ -240,7 +240,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab5"></a><h2 class="section">Decidability of equality over <span class="inlinecode"><span class="id" title="var">nat</span></span>.</h2>
<a id="lab6"></a><h2 class="section">Decidability of equality over <span class="inlinecode"><span class="id" title="var">nat</span></span>.</h2>

</div>
<div class="code">
Expand All @@ -252,7 +252,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab6"></a><h2 class="section">Ternary comparison</h2>
<a id="lab7"></a><h2 class="section">Ternary comparison</h2>

<div class="paragraph"> </div>

Expand Down Expand Up @@ -281,7 +281,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab7"></a><h2 class="section">Minimum, maximum</h2>
<a id="lab8"></a><h2 class="section">Minimum, maximum</h2>

</div>
<div class="code">
Expand Down Expand Up @@ -331,7 +331,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab8"></a><h2 class="section">Power</h2>
<a id="lab9"></a><h2 class="section">Power</h2>

</div>
<div class="code">
Expand All @@ -349,7 +349,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab9"></a><h2 class="section">Square</h2>
<a id="lab10"></a><h2 class="section">Square</h2>

</div>
<div class="code">
Expand All @@ -361,7 +361,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab10"></a><h2 class="section">Parity</h2>
<a id="lab11"></a><h2 class="section">Parity</h2>

</div>
<div class="code">
Expand Down Expand Up @@ -405,7 +405,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab11"></a><h2 class="section">Division</h2>
<a id="lab12"></a><h2 class="section">Division</h2>

</div>
<div class="code">
Expand Down Expand Up @@ -434,7 +434,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab12"></a><h2 class="section">Square root</h2>
<a id="lab13"></a><h2 class="section">Square root</h2>

</div>
<div class="code">
Expand All @@ -458,7 +458,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab13"></a><h2 class="section">Logarithm</h2>
<a id="lab14"></a><h2 class="section">Logarithm</h2>

</div>
<div class="code">
Expand All @@ -480,7 +480,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab14"></a><h2 class="section">Properties of <span class="inlinecode"><span class="id" title="var">iter</span></span></h2>
<a id="lab15"></a><h2 class="section">Properties of <span class="inlinecode"><span class="id" title="var">iter</span></span></h2>

</div>
<div class="code">
Expand Down Expand Up @@ -532,7 +532,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab15"></a><h2 class="section">Gcd</h2>
<a id="lab16"></a><h2 class="section">Gcd</h2>

</div>
<div class="code">
Expand Down Expand Up @@ -560,7 +560,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab16"></a><h2 class="section">Bitwise operations</h2>
<a id="lab17"></a><h2 class="section">Bitwise operations</h2>

</div>
<div class="code">
Expand Down
Loading

0 comments on commit c5f077c

Please sign in to comment.