Skip to content

Commit

Permalink
Documentation of branch “master” at 69301cf4
Browse files Browse the repository at this point in the history
  • Loading branch information
coqbot committed Jan 27, 2025
1 parent b18e291 commit c378cc7
Show file tree
Hide file tree
Showing 249 changed files with 1,188 additions and 1,186 deletions.
2 changes: 1 addition & 1 deletion master/api/rocq-runtime/Mod_subst/index.html

Large diffs are not rendered by default.

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.
50 changes: 26 additions & 24 deletions master/refman/proof-engine/ltac.html
Original file line number Diff line number Diff line change
Expand Up @@ -3377,7 +3377,7 @@ <h3>Timing a tactic that evaluates to a term: time_constr<a class="headerlink" h
  </span><span class="coqdoc-tactic">pose</span><span> </span><span class="coqdoc-var">v</span><span>.</span><span>
</span></dt><dd><span>Tactic evaluation (depth 1) ran for 0. secs (0.u,0.s)
Tactic evaluation (depth 1) ran for 0. secs (0.u,0.s)
Tactic evaluation ran for 0. secs (0.u,0.s)
Tactic evaluation ran for 0.002 secs (0.u,0.001s)
1 goal

n := 100 : nat
Expand Down Expand Up @@ -4292,38 +4292,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: 2.069s
</span></dt><dd><span>total time: 1.599s

tactic local total calls max
───────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac -------------------------------------- 0.1% 100.0% 1 2.069s
─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 98.0% 26 0.174s
─&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 97.9% 26 0.174s
─&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.0% 97.9% 26 0.174s
─t_tauto_intuit --------------------------- 0.1% 97.8% 26 0.174s
─&lt;Corelib.Init.Tauto.simplif&gt; ------------- 67.1% 94.5% 26 0.171s
─&lt;Corelib.Init.Tauto.is_conj&gt; ------------- 19.0% 19.0% 28756 0.000s
─elim id ---------------------------------- 4.5% 4.5% 650 0.001s
─&lt;Corelib.Init.Tauto.axioms&gt; -------------- 2.3% 3.2% 0 0.003s
─tac -------------------------------------- 0.1% 100.0% 1 1.599s
─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 97.7% 26 0.124s
─&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 97.6% 26 0.124s
─&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.1% 97.6% 26 0.124s
─t_tauto_intuit --------------------------- 0.1% 97.5% 26 0.124s
─&lt;Corelib.Init.Tauto.simplif&gt; ------------- 58.9% 89.6% 26 0.122s
─&lt;Corelib.Init.Tauto.is_conj&gt; ------------- 23.7% 23.7% 28756 0.067s
─&lt;Corelib.Init.Tauto.axioms&gt; -------------- 6.8% 7.8% 0 0.073s
─elim id ---------------------------------- 3.7% 3.7% 650 0.001s
─lia -------------------------------------- 0.1% 2.1% 28 0.014s

tactic local total calls max
───────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac -------------------------------------- 0.1% 100.0% 1 2.069s
└&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 98.0% 26 0.174s
└&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 97.9% 26 0.174s
└&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.0% 97.9% 26 0.174s
└t_tauto_intuit --------------------------- 0.1% 97.8% 26 0.174s
├─&lt;Corelib.Init.Tauto.simplif&gt; ----------- 67.1% 94.5% 26 0.171s
│ ├─&lt;Corelib.Init.Tauto.is_conj&gt; --------- 19.0% 19.0% 28756 0.000s
│ └─elim id ------------------------------ 4.5% 4.5% 650 0.001s
└─&lt;Corelib.Init.Tauto.axioms&gt; ------------ 2.3% 3.2% 0 0.003s
tactic local total calls max
─────────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac ---------------------------------------- 0.1% 100.0% 1 1.599s
├─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 97.7% 26 0.124s
│└&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 97.6% 26 0.124s
│└&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.1% 97.6% 26 0.124s
│└t_tauto_intuit --------------------------- 0.1% 97.5% 26 0.124s
│ ├─&lt;Corelib.Init.Tauto.simplif&gt; ----------- 58.9% 89.6% 26 0.122s
│ │ ├─&lt;Corelib.Init.Tauto.is_conj&gt; --------- 23.7% 23.7% 28756 0.067s
│ │ └─elim id ------------------------------ 3.7% 3.7% 650 0.001s
│ └─&lt;Corelib.Init.Tauto.axioms&gt; ------------ 6.8% 7.8% 0 0.073s
└─lia -------------------------------------- 0.1% 2.1% 28 0.014s
</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: 2.069s
</span></dt><dd><span>total time: 1.599s

tactic local total calls max
───────┴──────┴──────┴───────┴─────────┘

─lia -- 0.1% 2.1% 28 0.014s

tactic local total calls max
───────┴──────┴──────┴───────┴─────────┘
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 @@ -2646,15 +2646,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.206 secs (0.101u,0.105s) (successful)
</span></dt><dd><span>Finished transaction in 0.132 secs (0.054u,0.078s) (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.824 secs (0.824u,0.s) (successful)
</span></dt><dd><span>Finished transaction in 0.664 secs (0.658u,0.006s) (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 @@ -276,7 +276,7 @@ <h1 class="libtitle">Library Stdlib.Arith.Arith_base</h1>
</div>

<div class="doc">
<a id="lab1"></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 @@ -298,7 +298,7 @@ <h1 class="libtitle">Library Stdlib.Arith.Arith_base</h1>
</div>

<div class="doc">
<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>
<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 @@ -274,7 +274,7 @@ <h1 class="libtitle">Library Stdlib.Arith.EqNat</h1>
Equality on natural numbers
<div class="paragraph"> </div>

<a id="lab18"></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 @@ -367,7 +367,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab3"></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 @@ -385,7 +385,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab4"></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 @@ -427,7 +427,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab5"></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 @@ -459,7 +459,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab6"></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 @@ -471,7 +471,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab7"></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 @@ -500,7 +500,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

<div class="doc">
<a id="lab8"></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 @@ -550,7 +550,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

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

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

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

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

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

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

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

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

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

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

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

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

<div class="doc">
<a id="lab15"></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 @@ -751,7 +751,7 @@ <h1 class="libtitle">Library Stdlib.Arith.PeanoNat</h1>
</div>

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

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

<div class="doc">
<a id="lab17"></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 @@ -308,7 +308,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab690"></a><h1 class="section">Decidability</h1>
<a id="lab261"></a><h1 class="section">Decidability</h1>

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

<div class="doc">
<a id="lab691"></a><h1 class="section">Discrimination</h1>
<a id="lab262"></a><h1 class="section">Discrimination</h1>

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

<div class="doc">
<a id="lab692"></a><h1 class="section">Order on booleans</h1>
<a id="lab263"></a><h1 class="section">Order on booleans</h1>

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

<div class="doc">
<a id="lab693"></a><h1 class="section">Equality</h1>
<a id="lab264"></a><h1 class="section">Equality</h1>

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

<div class="doc">
<a id="lab694"></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="lab265"></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 @@ -460,7 +460,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab695"></a><h1 class="section">De Morgan laws</h1>
<a id="lab266"></a><h1 class="section">De Morgan laws</h1>

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

<div class="doc">
<a id="lab696"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">negb</span></span></h1>
<a id="lab267"></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 @@ -517,7 +517,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab697"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">orb</span></span></h1>
<a id="lab268"></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 @@ -645,7 +645,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab698"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">andb</span></span></h1>
<a id="lab269"></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 @@ -762,7 +762,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab699"></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="lab270"></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 @@ -812,7 +812,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab700"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">implb</span></span></h1>
<a id="lab271"></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 @@ -866,7 +866,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab701"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">xorb</span></span></h1>
<a id="lab272"></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 @@ -1028,7 +1028,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab702"></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="lab273"></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 @@ -1142,7 +1142,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab703"></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="lab274"></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 @@ -1170,7 +1170,7 @@ <h1 class="libtitle">Library Stdlib.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab704"></a><h1 class="section">Reflect: a specialized inductive type for</h1>
<a id="lab275"></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 c378cc7

Please sign in to comment.