Skip to content

Commit

Permalink
Documentation of branch “master” at f76afe01
Browse files Browse the repository at this point in the history
  • Loading branch information
coqbot committed Jan 14, 2025
1 parent 96168bf commit 904a0d9
Show file tree
Hide file tree
Showing 249 changed files with 1,194 additions and 1,194 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.
50 changes: 25 additions & 25 deletions master/refman/proof-engine/ltac.html
Original file line number Diff line number Diff line change
Expand Up @@ -4286,42 +4286,42 @@ <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.219s
</span></dt><dd><span>total time: 1.687s

tactic local total calls max
───────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac -------------------------------------- 0.1% 100.0% 1 2.219s
─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 93.7% 26 0.139s
─&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 93.6% 26 0.139s
─&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.0% 93.6% 26 0.139s
─t_tauto_intuit --------------------------- 0.1% 93.5% 26 0.139s
─&lt;Corelib.Init.Tauto.simplif&gt; ------------- 60.6% 90.0% 26 0.136s
─&lt;Corelib.Init.Tauto.is_conj&gt; ------------- 20.9% 20.9% 28756 0.017s
─lia -------------------------------------- 0.1% 6.1% 28 0.095s
Zify.zify -------------------------------- 4.5% 5.0% 54 0.095s
elim id ---------------------------------- 4.6% 4.6% 650 0.001s
─&lt;Corelib.Init.Tauto.axioms&gt; -------------- 2.5% 3.4% 0 0.006s
─tac -------------------------------------- 0.1% 100.0% 1 1.687s
─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 94.4% 26 0.102s
─&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 94.4% 26 0.102s
─&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.0% 94.3% 26 0.102s
─t_tauto_intuit --------------------------- 0.1% 94.3% 26 0.102s
─&lt;Corelib.Init.Tauto.simplif&gt; ------------- 60.4% 90.9% 26 0.099s
─&lt;Corelib.Init.Tauto.is_conj&gt; ------------- 22.1% 22.1% 28756 0.016s
─lia -------------------------------------- 0.1% 5.3% 28 0.062s
elim id ---------------------------------- 4.6% 4.6% 650 0.000s
Zify.zify -------------------------------- 3.9% 4.4% 54 0.061s
─&lt;Corelib.Init.Tauto.axioms&gt; -------------- 2.3% 3.3% 0 0.004s

tactic local total calls max
─────────────────────────────────────────────┴──────┴──────┴───────┴─────────┘
─tac ---------------------------------------- 0.1% 100.0% 1 2.219s
├─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 93.7% 26 0.139s
│└&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 93.6% 26 0.139s
│└&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.0% 93.6% 26 0.139s
│└t_tauto_intuit --------------------------- 0.1% 93.5% 26 0.139s
│ ├─&lt;Corelib.Init.Tauto.simplif&gt; ----------- 60.6% 90.0% 26 0.136s
│ │ ├─&lt;Corelib.Init.Tauto.is_conj&gt; --------- 20.9% 20.9% 28756 0.017s
│ │ └─elim id ------------------------------ 4.6% 4.6% 650 0.001s
│ └─&lt;Corelib.Init.Tauto.axioms&gt; ------------ 2.5% 3.4% 0 0.006s
└─lia -------------------------------------- 0.1% 6.1% 28 0.095s
└Zify.zify -------------------------------- 4.5% 5.0% 54 0.095s
─tac ---------------------------------------- 0.1% 100.0% 1 1.687s
├─&lt;Corelib.Init.Tauto.with_uniform_flags&gt; -- 0.0% 94.4% 26 0.102s
│└&lt;Corelib.Init.Tauto.tauto_gen&gt; ----------- 0.0% 94.4% 26 0.102s
│└&lt;Corelib.Init.Tauto.tauto_intuitionistic&gt; 0.0% 94.3% 26 0.102s
│└t_tauto_intuit --------------------------- 0.1% 94.3% 26 0.102s
│ ├─&lt;Corelib.Init.Tauto.simplif&gt; ----------- 60.4% 90.9% 26 0.099s
│ │ ├─&lt;Corelib.Init.Tauto.is_conj&gt; --------- 22.1% 22.1% 28756 0.016s
│ │ └─elim id ------------------------------ 4.6% 4.6% 650 0.000s
│ └─&lt;Corelib.Init.Tauto.axioms&gt; ------------ 2.3% 3.3% 0 0.004s
└─lia -------------------------------------- 0.1% 5.3% 28 0.062s
└Zify.zify -------------------------------- 3.9% 4.4% 54 0.061s
</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.219s
</span></dt><dd><span>total time: 1.687s

tactic local total calls max
───────┴──────┴──────┴───────┴─────────┘
─lia -- 0.1% 6.1% 28 0.095s
─lia -- 0.1% 5.3% 28 0.062s

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 @@ -2640,15 +2640,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.12 secs (0.083u,0.037s) (successful)
</span></dt><dd><span>Finished transaction in 0.103 secs (0.067u,0.035s) (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.728 secs (0.727u,0.001s) (successful)
</span></dt><dd><span>Finished transaction in 0.576 secs (0.575u,0.001s) (successful)
1 goal

H : id (fact 8)</span><span> =</span><span> fact 8
Expand Down Expand Up @@ -2676,7 +2676,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. secs (0.u,0.s) (successful)
</span></dt><dd><span>Finished transaction in 0.001 secs (0.u,0.001s) (successful)
1 goal

H : id (fact 100)</span><span> =</span><span> fact 100
Expand Down Expand Up @@ -2722,7 +2722,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.001 secs (0.001u,0.s) (successful)
</span></dt><dd><span>Finished transaction in 0. secs (0.u,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/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 904a0d9

Please sign in to comment.