Skip to content

Commit

Permalink
Documentation of branch “master” at c011e08a
Browse files Browse the repository at this point in the history
  • Loading branch information
coqbot committed Jan 16, 2024
1 parent f418961 commit 6023cd2
Show file tree
Hide file tree
Showing 255 changed files with 1,442 additions and 1,289 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/program.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/universe-polymorphism.doctree
Binary file not shown.
Binary file modified master/refman/.doctrees/environment.pickle
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/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 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/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.
40 changes: 20 additions & 20 deletions master/refman/proof-engine/ltac.html
Original file line number Diff line number Diff line change
Expand Up @@ -4241,37 +4241,37 @@ <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.871s
</span></dt><dd><span>total time: 2.728s

tactic local total calls max
────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac ----------------------------------- 2.0% 100.0% 1 2.871s
─&lt;Coq.Init.Tauto.with_uniform_flags&gt; --- 0.0% 96.3% 26 0.263s
─&lt;Coq.Init.Tauto.tauto_gen&gt; ------------ 0.0% 96.2% 26 0.263s
─&lt;Coq.Init.Tauto.tauto_intuitionistic&gt; - 0.0% 96.2% 26 0.263s
─t_tauto_intuit ------------------------ 0.1% 96.1% 26 0.263s
─&lt;Coq.Init.Tauto.simplif&gt; -------------- 61.0% 93.0% 26 0.259s
─&lt;Coq.Init.Tauto.is_conj&gt; -------------- 17.9% 17.9% 28756 0.024s
─intro --------------------------------- 6.9% 6.9% 1300 0.151s
─tac ----------------------------------- 0.1% 100.0% 1 2.728s
─&lt;Coq.Init.Tauto.with_uniform_flags&gt; --- 0.0% 96.8% 26 0.226s
─&lt;Coq.Init.Tauto.tauto_gen&gt; ------------ 0.0% 96.8% 26 0.226s
─&lt;Coq.Init.Tauto.tauto_intuitionistic&gt; - 0.0% 96.8% 26 0.226s
─t_tauto_intuit ------------------------ 0.0% 96.7% 26 0.225s
─&lt;Coq.Init.Tauto.simplif&gt; -------------- 60.8% 93.9% 26 0.223s
─&lt;Coq.Init.Tauto.is_conj&gt; -------------- 19.2% 19.2% 28756 0.024s
─intro --------------------------------- 6.8% 6.8% 1300 0.140s
─elim id ------------------------------- 5.5% 5.5% 650 0.001s
─&lt;Coq.Init.Tauto.axioms&gt; --------------- 2.2% 3.1% 0 0.004s
─&lt;Coq.Init.Tauto.axioms&gt; --------------- 2.0% 2.8% 0 0.005s

tactic local total calls max
────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac ----------------------------------- 2.0% 100.0% 1 2.871s
└&lt;Coq.Init.Tauto.with_uniform_flags&gt; --- 0.0% 96.3% 26 0.263s
└&lt;Coq.Init.Tauto.tauto_gen&gt; ------------ 0.0% 96.2% 26 0.263s
└&lt;Coq.Init.Tauto.tauto_intuitionistic&gt; - 0.0% 96.2% 26 0.263s
└t_tauto_intuit ------------------------ 0.1% 96.1% 26 0.263s
├─&lt;Coq.Init.Tauto.simplif&gt; ------------ 61.0% 93.0% 26 0.259s
│ ├─&lt;Coq.Init.Tauto.is_conj&gt; ---------- 17.9% 17.9% 28756 0.024s
│ ├─intro ----------------------------- 6.9% 6.9% 1300 0.151s
─tac ----------------------------------- 0.1% 100.0% 1 2.728s
└&lt;Coq.Init.Tauto.with_uniform_flags&gt; --- 0.0% 96.8% 26 0.226s
└&lt;Coq.Init.Tauto.tauto_gen&gt; ------------ 0.0% 96.8% 26 0.226s
└&lt;Coq.Init.Tauto.tauto_intuitionistic&gt; - 0.0% 96.8% 26 0.226s
└t_tauto_intuit ------------------------ 0.0% 96.7% 26 0.225s
├─&lt;Coq.Init.Tauto.simplif&gt; ------------ 60.8% 93.9% 26 0.223s
│ ├─&lt;Coq.Init.Tauto.is_conj&gt; ---------- 19.2% 19.2% 28756 0.024s
│ ├─intro ----------------------------- 6.8% 6.8% 1300 0.140s
│ └─elim id --------------------------- 5.5% 5.5% 650 0.001s
└─&lt;Coq.Init.Tauto.axioms&gt; ------------- 2.2% 3.1% 0 0.004s
└─&lt;Coq.Init.Tauto.axioms&gt; ------------- 2.0% 2.8% 0 0.005s

</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.871s
</span></dt><dd><span>total time: 2.728s

tactic local total calls max
────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
Expand Down
8 changes: 4 additions & 4 deletions master/refman/proofs/writing-proofs/equality.html
Original file line number Diff line number Diff line change
Expand Up @@ -2554,15 +2554,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.191 secs (0.157u,0.033s) (successful)
</span></dt><dd><span>Finished transaction in 0.122 secs (0.103u,0.017s) (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 1.363 secs (1.361u,0.002s) (successful)
</span></dt><dd><span>Finished transaction in 1.076 secs (1.075u,0.001s) (successful)
1 goal

H : id (fact 8)</span><span> =</span><span> fact 8
Expand Down Expand Up @@ -2590,7 +2590,7 @@ <h3>Computing in a term: eval and Eval<a class="headerlink" href="#computing-in-
Timeout!
</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">reflexivity</span><span>.</span><span>
</span></dt><dd><span>Finished transaction in 0.001 secs (0.001u,0.s) (successful)
</span></dt><dd><span>Finished transaction in 0.003 secs (0.003u,0.s) (successful)
1 goal

H : id (fact 100)</span><span> =</span><span> fact 100
Expand Down Expand Up @@ -2636,7 +2636,7 @@ <h3>Computing in a term: eval and Eval<a class="headerlink" href="#computing-in-
</span></dt><dd><span>No more goals.
</span></dd>
<dt><span></span><span class="coqdoc-keyword">Time</span><span> </span><span class="coqdoc-keyword">Defined</span><span>.</span><span>
</span></dt><dd><span>Finished transaction in 0. secs (0.u,0.s) (successful)
</span></dt><dd><span>Finished transaction in 0.001 secs (0.001u,0.s) (successful)
</span></dd>
</dl>
</div>
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/Coq.Arith.Arith_base.html
Original file line number Diff line number Diff line change
Expand Up @@ -58,7 +58,7 @@ <h1 class="libtitle">Library Coq.Arith.Arith_base</h1>
</div>

<div class="doc">
<a id="lab631"></a><h1 class="section"><span class="inlinecode"><span class="id" title="var">arith</span></span> hint database</h1>
<a id="lab17"></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 Coq.Arith.Arith_base</h1>
</div>

<div class="doc">
<a id="lab632"></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="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>

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

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

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

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

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

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

<div class="doc">
<a id="lab617"></a><h2 class="section">Basic specifications : pred add sub mul</h2>
<a id="lab3"></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 Coq.Arith.PeanoNat</h1>
</div>

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

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

<div class="doc">
<a id="lab619"></a><h2 class="section">Decidability of equality over <span class="inlinecode"><span class="id" title="var">nat</span></span>.</h2>
<a id="lab5"></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 Coq.Arith.PeanoNat</h1>
</div>

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

<div class="doc">
<a id="lab628"></a><h2 class="section">Properties of <span class="inlinecode"><span class="id" title="var">iter</span></span></h2>
<a id="lab14"></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 @@ -529,7 +529,7 @@ <h1 class="libtitle">Library Coq.Arith.PeanoNat</h1>
</div>

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

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

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

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

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

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

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

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

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

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

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

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

<div class="doc">
<a id="lab427"></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="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>

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

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

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

<div class="doc">
<a id="lab429"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">negb</span></span></h1>
<a id="lab40"></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 Coq.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab430"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">orb</span></span></h1>
<a id="lab41"></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 Coq.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab431"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">andb</span></span></h1>
<a id="lab42"></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 Coq.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab432"></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="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>

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

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

<div class="doc">
<a id="lab433"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">implb</span></span></h1>
<a id="lab44"></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 Coq.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab434"></a><h1 class="section">Properties of <span class="inlinecode"><span class="id" title="var">xorb</span></span></h1>
<a id="lab45"></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 Coq.Bool.Bool</h1>
</div>

<div class="doc">
<a id="lab435"></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="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>

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

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

<div class="doc">
<a id="lab436"></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="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>

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

<div class="doc">
<a id="lab437"></a><h1 class="section">Reflect: a specialized inductive type for</h1>
<a id="lab48"></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 6023cd2

Please sign in to comment.