Skip to content

Commit

Permalink
Documentation of branch “master” at ac0fd362
Browse files Browse the repository at this point in the history
  • Loading branch information
coqbot committed Nov 14, 2024
1 parent b907656 commit 594146f
Show file tree
Hide file tree
Showing 271 changed files with 1,282 additions and 1,284 deletions.
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.
Original file line number Diff line number Diff line change
Expand Up @@ -662,7 +662,6 @@ file is a particular case of a module called a *library file*.
Loads OCaml plugins and their dependencies dynamically. The :n:`@string`
arguments must be valid `findlib <http://projects.camlcity.org/projects/findlib.html>`_
plugin names, for example ``coq-core.plugins.ltac``.
They must also contain a `.` to disambiguate against the removed non-findlib loading method.

Effects (such as adding new commands) from the explicitly requested
plugin are activated, but effects from implicitly loaded
Expand Down
46 changes: 23 additions & 23 deletions master/refman/proof-engine/ltac.html
Original file line number Diff line number Diff line change
Expand Up @@ -4289,40 +4289,40 @@ <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.241s
</span></dt><dd><span>total time: 1.175s

tactic local total calls max
──────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac ------------------------------------- 0.1% 100.0% 1 1.241s
─&lt;Stdlib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 96.8% 26 0.136s
─&lt;Stdlib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 96.8% 26 0.136s
─&lt;Stdlib.Init.Tauto.tauto_intuitionistic&gt; 0.1% 96.7% 26 0.136s
─t_tauto_intuit -------------------------- 0.1% 96.6% 26 0.136s
─&lt;Stdlib.Init.Tauto.simplif&gt; ------------- 62.6% 93.6% 26 0.135s
─&lt;Stdlib.Init.Tauto.is_conj&gt; ------------- 20.0% 20.0% 28756 0.002s
─elim id --------------------------------- 6.3% 6.3% 650 0.016s
─&lt;Stdlib.Init.Tauto.axioms&gt; -------------- 2.0% 3.0% 0 0.002s
─lia ------------------------------------- 0.1% 2.8% 28 0.018s
─tac ------------------------------------- 0.1% 100.0% 1 1.175s
─&lt;Stdlib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 96.8% 26 0.131s
─&lt;Stdlib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 96.7% 26 0.131s
─&lt;Stdlib.Init.Tauto.tauto_intuitionistic&gt; 0.1% 96.7% 26 0.131s
─t_tauto_intuit -------------------------- 0.1% 96.6% 26 0.131s
─&lt;Stdlib.Init.Tauto.simplif&gt; ------------- 63.2% 93.4% 26 0.130s
─&lt;Stdlib.Init.Tauto.is_conj&gt; ------------- 20.3% 20.3% 28756 0.000s
─elim id --------------------------------- 6.3% 6.3% 650 0.009s
─&lt;Stdlib.Init.Tauto.axioms&gt; -------------- 2.1% 3.1% 0 0.002s
─lia ------------------------------------- 0.1% 2.8% 28 0.017s

tactic local total calls max
────────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac --------------------------------------- 0.1% 100.0% 1 1.241s
├─&lt;Stdlib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 96.8% 26 0.136s
│└&lt;Stdlib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 96.8% 26 0.136s
│└&lt;Stdlib.Init.Tauto.tauto_intuitionistic&gt; 0.1% 96.7% 26 0.136s
│└t_tauto_intuit -------------------------- 0.1% 96.6% 26 0.136s
│ ├─&lt;Stdlib.Init.Tauto.simplif&gt; ----------- 62.6% 93.6% 26 0.135s
│ │ ├─&lt;Stdlib.Init.Tauto.is_conj&gt; --------- 20.0% 20.0% 28756 0.002s
│ │ └─elim id ----------------------------- 6.3% 6.3% 650 0.016s
│ └─&lt;Stdlib.Init.Tauto.axioms&gt; ------------ 2.0% 3.0% 0 0.002s
└─lia ------------------------------------- 0.1% 2.8% 28 0.018s
─tac --------------------------------------- 0.1% 100.0% 1 1.175s
├─&lt;Stdlib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 96.8% 26 0.131s
│└&lt;Stdlib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 96.7% 26 0.131s
│└&lt;Stdlib.Init.Tauto.tauto_intuitionistic&gt; 0.1% 96.7% 26 0.131s
│└t_tauto_intuit -------------------------- 0.1% 96.6% 26 0.131s
│ ├─&lt;Stdlib.Init.Tauto.simplif&gt; ----------- 63.2% 93.4% 26 0.130s
│ │ ├─&lt;Stdlib.Init.Tauto.is_conj&gt; --------- 20.3% 20.3% 28756 0.000s
│ │ └─elim id ----------------------------- 6.3% 6.3% 650 0.009s
│ └─&lt;Stdlib.Init.Tauto.axioms&gt; ------------ 2.1% 3.1% 0 0.002s
└─lia ------------------------------------- 0.1% 2.8% 28 0.017s
</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.241s
</span></dt><dd><span>total time: 1.175s

tactic local total calls max
───────┴──────┴──────┴───────┴─────────┘
─lia -- 0.1% 2.8% 28 0.018s
─lia -- 0.1% 2.8% 28 0.017s

tactic local total calls max
───────┴──────┴──────┴───────┴─────────┘
Expand Down
3 changes: 1 addition & 2 deletions master/refman/proof-engine/vernacular-commands.html
Original file line number Diff line number Diff line change
Expand Up @@ -2124,8 +2124,7 @@ <h2>Query commands<a class="headerlink" href="#query-commands" title="Permalink
<em class="property"><span class="sigannot"><span class="pre">Command</span></span></em> <span class="sig-name descname"><span class="notation"><span><span><span class="pre">Declare</span></span></span> <span><span><span class="pre">ML</span></span></span> <span><span><span class="pre">Module</span></span></span> <span class="repeat-wrapper"><span class="repeat"><a class="reference internal" href="../language/core/basic.html#grammar-token-string"><span class="hole"><span class="pre">string</span></span></a></span><span class="notation-sup"><span class="pre">+</span></span></span></span></span><a class="headerlink" href="#coq:cmd.Declare-ML-Module" title="Permalink to this definition"></a></dt>
<dd><p>Loads OCaml plugins and their dependencies dynamically. The <code class="docutils literal notranslate"><span class="notation"><a class="reference internal" href="../language/core/basic.html#grammar-token-string"><span class="hole"><span class="pre">string</span></span></a></span></code>
arguments must be valid <a class="reference external" href="http://projects.camlcity.org/projects/findlib.html">findlib</a>
plugin names, for example <code class="docutils literal notranslate"><span class="pre">coq-core.plugins.ltac</span></code>.
They must also contain a <code class="docutils literal notranslate"><span class="pre">.</span></code> to disambiguate against the removed non-findlib loading method.</p>
plugin names, for example <code class="docutils literal notranslate"><span class="pre">coq-core.plugins.ltac</span></code>.</p>
<p>Effects (such as adding new commands) from the explicitly requested
plugin are activated, but effects from implicitly loaded
dependencies are not activated.</p>
Expand Down
4 changes: 2 additions & 2 deletions master/refman/proofs/writing-proofs/equality.html
Original file line number Diff line number Diff line change
Expand Up @@ -2636,15 +2636,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.138 secs (0.115u,0.023s) (successful)
</span></dt><dd><span>Finished transaction in 0.113 secs (0.097u,0.015s) (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.604 secs (0.602u,0.001s) (successful)
</span></dt><dd><span>Finished transaction in 0.543 secs (0.543u,0.s) (successful)
1 goal

H : id (fact 8)</span><span> =</span><span> fact 8
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 @@ -58,7 +58,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="lab238"></a><h1 class="section"><span class="inlinecode"><span class="id" title="var">arith</span></span> hint database</h1>

</div>
<div class="code">
Expand All @@ -80,7 +80,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="lab239"></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 @@ -56,7 +56,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="lab237"></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 @@ -149,7 +149,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="lab222"></a><h2 class="section">Remaining constants not defined in Stdlib.Init.Nat</h2>

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

Expand All @@ -167,7 +167,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="lab223"></a><h2 class="section">Basic specifications : pred add sub mul</h2>

</div>
<div class="code">
Expand Down Expand Up @@ -209,7 +209,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="lab224"></a><h2 class="section">Boolean comparisons</h2>

</div>
<div class="code">
Expand Down Expand Up @@ -241,7 +241,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="lab225"></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 @@ -253,7 +253,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="lab226"></a><h2 class="section">Ternary comparison</h2>

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

Expand Down Expand Up @@ -282,7 +282,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="lab227"></a><h2 class="section">Minimum, maximum</h2>

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

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

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

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

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

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

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

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

</div>
<div class="code">
Expand Down Expand Up @@ -435,7 +435,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="lab232"></a><h2 class="section">Square root</h2>

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

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

</div>
<div class="code">
Expand All @@ -481,7 +481,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="lab234"></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 @@ -533,7 +533,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

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

</div>
<div class="code">
Expand Down Expand Up @@ -561,7 +561,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="lab236"></a><h2 class="section">Bitwise operations</h2>

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

<div class="doc">
<a id="lab34"></a><h1 class="section">Decidability</h1>
<a id="lab263"></a><h1 class="section">Decidability</h1>

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

<div class="doc">
<a id="lab35"></a><h1 class="section">Discrimination</h1>
<a id="lab264"></a><h1 class="section">Discrimination</h1>

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

<div class="doc">
<a id="lab36"></a><h1 class="section">Order on booleans</h1>
<a id="lab265"></a><h1 class="section">Order on booleans</h1>

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

<div class="doc">
<a id="lab37"></a><h1 class="section">Equality</h1>
<a id="lab266"></a><h1 class="section">Equality</h1>

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

<div class="doc">
<a id="lab38"></a><h1 class="section">A synonym of <span class="inlinecode"><span class="id" title="keyword">if</span></span> on <span class="inlinecode"><span class="id" title="var">bool</span></span></h1>
<a id="lab267"></a><h1 class="section">A synonym of <span class="inlinecode"><span class="id" title="keyword">if</span></span> on <span class="inlinecode"><span class="id" title="var">bool</span></span></h1>

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

<div class="doc">
<a id="lab39"></a><h1 class="section">De Morgan laws</h1>
<a id="lab268"></a><h1 class="section">De Morgan laws</h1>

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

<div class="doc">
<a id="lab40"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">negb</span></span></h1>
<a id="lab269"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">negb</span></span></h1>

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

<div class="doc">
<a id="lab41"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">orb</span></span></h1>
<a id="lab270"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">orb</span></span></h1>

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

<div class="doc">
<a id="lab42"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">andb</span></span></h1>
<a id="lab271"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">andb</span></span></h1>

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

<div class="doc">
<a id="lab43"></a><h1 class="section">Properties mixing <span class="inlinecode"><span class="id" title="var">andb</span></span> and <span class="inlinecode"><span class="id" title="var">orb</span></span></h1>
<a id="lab272"></a><h1 class="section">Properties mixing <span class="inlinecode"><span class="id" title="var">andb</span></span> and <span class="inlinecode"><span class="id" title="var">orb</span></span></h1>

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

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

<div class="doc">
<a id="lab44"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">implb</span></span></h1>
<a id="lab273"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">implb</span></span></h1>

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

<div class="doc">
<a id="lab45"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">xorb</span></span></h1>
<a id="lab274"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">xorb</span></span></h1>

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

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

<div class="doc">
<a id="lab46"></a><h1 class="section">Reflection of <span class="inlinecode"><span class="id" title="var">bool</span></span> into <span class="inlinecode"><span class="id" title="keyword">Prop</span></span></h1>
<a id="lab275"></a><h1 class="section">Reflection of <span class="inlinecode"><span class="id" title="var">bool</span></span> into <span class="inlinecode"><span class="id" title="keyword">Prop</span></span></h1>

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

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

<div class="doc">
<a id="lab47"></a><h1 class="section">Alternative versions of <span class="inlinecode"><span class="id" title="var">andb</span></span> and <span class="inlinecode"><span class="id" title="var">orb</span></span></h1>
<a id="lab276"></a><h1 class="section">Alternative versions of <span class="inlinecode"><span class="id" title="var">andb</span></span> and <span class="inlinecode"><span class="id" title="var">orb</span></span></h1>

with lazy behavior (for vm_compute)
</div>
Expand Down Expand Up @@ -952,7 +952,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab48"></a><h1 class="section">Reflect: a specialized inductive type for</h1>
<a id="lab277"></a><h1 class="section">Reflect: a specialized inductive type for</h1>

relating propositions and booleans,
as popularized by the Ssreflect library.
Expand Down
Loading

0 comments on commit 594146f

Please sign in to comment.