Skip to content

Commit

Permalink
release 1.30.0
Browse files Browse the repository at this point in the history
  • Loading branch information
SKolodynski committed May 26, 2024
1 parent 6f7ff74 commit ea33786
Show file tree
Hide file tree
Showing 114 changed files with 11,727 additions and 9,770 deletions.
2 changes: 1 addition & 1 deletion Dockerfile
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
## Dockerfile for IsarMathLib

FROM slawekkol/isarmathlib:isabelle-zf-2023
FROM slawekkol/isarmathlib:isabelle-zf-2024

COPY IsarMathLib /home/isabelle/IsarMathLib

Expand Down
12 changes: 7 additions & 5 deletions IsarMathLib/IntModule_ZF.thy
Original file line number Diff line number Diff line change
Expand Up @@ -1054,8 +1054,8 @@ proof(rule nat_induct[of z2 "\<lambda>t. Fold(P,\<one>,(z1#*t)\<times>{g}) = Fol
}
qed

text\<open>Multiplying 2 int_of natural numbers, is the same as multiplying the natural
numbers and then applying int_of\<close>
text\<open>Multiplying 2 int\_of natural numbers, is the same as multiplying the natural
numbers and then applying int\_of\<close>

lemma int_of_mult:
assumes "nr:nat" "ns:nat"
Expand Down Expand Up @@ -1257,17 +1257,19 @@ sublocale abelian_group_int_action < int_action:module0 ints IntegerAddition Int
using groupAssum apply simp using isAbelian apply simp using group_action_int
unfolding IsLeftModule_def apply simp done

text\<open>
(*
lemma (in abelian_group_int) one_one:
shows "\<one> = TheNeutralElement(ints,IntegerMultiplication)"
cannot be interpreted. First the unit integer.
\<close>
\<close>*)

abbreviation (in abelian_group_int_action) zone ("\<one>\<^sub>\<int>") where
"\<one>\<^sub>\<int> \<equiv> ione"

text\<open>Then, the unit in the abelian group\<close>

abbreviation (in abelian_group_int_action) gone ("\<one>\<^sub>G") where
"\<one>\<^sub>G \<equiv> neut"
"\<one>\<^sub>G \<equiv> neut"

end
4 changes: 2 additions & 2 deletions IsarMathLib/document/root.tex
Original file line number Diff line number Diff line change
Expand Up @@ -66,8 +66,8 @@
\maketitle

\begin{abstract}
This is the proof document of the IsarMathLib project version 1.29.0.
IsarMathLib is a library of formalized mathematics for Isabelle2023 (ZF logic).
This is the proof document of the IsarMathLib project version 1.30.0.
IsarMathLib is a library of formalized mathematics for Isabelle2024 (ZF logic).

\end{abstract}

Expand Down
2 changes: 1 addition & 1 deletion README.md
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ IsarMathLib is a library of formalized mathematics for Isabelle/ZF.
[Isabelle](https://www.cl.cam.ac.uk/research/hvg/Isabelle/index.html) is a theorem proving environment developed at Cambridge University and TU Munich.
Isabelle needs to be installed on the machine before you can generate IsarMathLib proof documents or verify the proofs. The Isabelle site provides the installation instructions. IsarMathLib is always tested only with the version of Isabelle that is current at the time of IsarMathLib release.

IsarMathLib needs Isabelle/ZF logic that is not shipped precompiled in the Isabelle distribution bundle. To build the ZF heap go to the directory where you have unpacked Isabelle and type "./bin/isabelle build -b ZF". Alternatively, one can change the default logic in the etc/settings file from HOL to ZF and then start Isabelle environment with the main `Isabelle2023` executable script. This should start with building the ZF heap image.
IsarMathLib needs Isabelle/ZF logic that is not shipped precompiled in the Isabelle distribution bundle. To build the ZF heap go to the directory where you have unpacked Isabelle and type "./bin/isabelle build -b ZF". Alternatively, one can change the default logic in the etc/settings file from HOL to ZF and then start Isabelle environment with the main `Isabelle2024` executable script. This should start with building the ZF heap image.

Before processing the IsarMathLib project theories, make sure you have LaTeX installed (including extras, for example in Ubuntu run "apt-get install texlive-latex-extras").

Expand Down
136 changes: 68 additions & 68 deletions docs/IsarMathLib/AbelianGroup_ZF.html

Large diffs are not rendered by default.

160 changes: 80 additions & 80 deletions docs/IsarMathLib/Cardinal_ZF.html

Large diffs are not rendered by default.

118 changes: 59 additions & 59 deletions docs/IsarMathLib/CommutativeSemigroup_ZF.html

Large diffs are not rendered by default.

286 changes: 143 additions & 143 deletions docs/IsarMathLib/Complex_ZF.html

Large diffs are not rendered by default.

46 changes: 23 additions & 23 deletions docs/IsarMathLib/DirectProduct_ZF.html

Large diffs are not rendered by default.

104 changes: 52 additions & 52 deletions docs/IsarMathLib/Enumeration_ZF.html

Large diffs are not rendered by default.

254 changes: 127 additions & 127 deletions docs/IsarMathLib/EquivClass1.html

Large diffs are not rendered by default.

114 changes: 57 additions & 57 deletions docs/IsarMathLib/Field_ZF.html

Large diffs are not rendered by default.

118 changes: 59 additions & 59 deletions docs/IsarMathLib/FinOrd_ZF.html

Large diffs are not rendered by default.

188 changes: 94 additions & 94 deletions docs/IsarMathLib/Finite1.html

Large diffs are not rendered by default.

258 changes: 129 additions & 129 deletions docs/IsarMathLib/FiniteSeq_ZF.html

Large diffs are not rendered by default.

364 changes: 182 additions & 182 deletions docs/IsarMathLib/Finite_State_Machines_ZF.html

Large diffs are not rendered by default.

178 changes: 89 additions & 89 deletions docs/IsarMathLib/Finite_ZF.html

Large diffs are not rendered by default.

48 changes: 24 additions & 24 deletions docs/IsarMathLib/Finite_ZF_1.html

Large diffs are not rendered by default.

80 changes: 40 additions & 40 deletions docs/IsarMathLib/Fol1.html

Large diffs are not rendered by default.

166 changes: 83 additions & 83 deletions docs/IsarMathLib/Fold_ZF.html

Large diffs are not rendered by default.

144 changes: 72 additions & 72 deletions docs/IsarMathLib/Generalization_ZF.html

Large diffs are not rendered by default.

310 changes: 155 additions & 155 deletions docs/IsarMathLib/Group_ZF.html

Large diffs are not rendered by default.

168 changes: 84 additions & 84 deletions docs/IsarMathLib/Group_ZF_1.html

Large diffs are not rendered by default.

136 changes: 68 additions & 68 deletions docs/IsarMathLib/Group_ZF_1b.html

Large diffs are not rendered by default.

218 changes: 109 additions & 109 deletions docs/IsarMathLib/Group_ZF_2.html

Large diffs are not rendered by default.

404 changes: 202 additions & 202 deletions docs/IsarMathLib/Group_ZF_3.html

Large diffs are not rendered by default.

84 changes: 42 additions & 42 deletions docs/IsarMathLib/Group_ZF_4.html

Large diffs are not rendered by default.

132 changes: 66 additions & 66 deletions docs/IsarMathLib/Group_ZF_5.html

Large diffs are not rendered by default.

364 changes: 182 additions & 182 deletions docs/IsarMathLib/InductiveSeq_ZF.html

Large diffs are not rendered by default.

36 changes: 18 additions & 18 deletions docs/IsarMathLib/IntDiv_ZF_IML.html

Large diffs are not rendered by default.

1,292 changes: 1,292 additions & 0 deletions docs/IsarMathLib/IntModule_ZF.html

Large diffs are not rendered by default.

526 changes: 263 additions & 263 deletions docs/IsarMathLib/Int_ZF_1.html

Large diffs are not rendered by default.

378 changes: 189 additions & 189 deletions docs/IsarMathLib/Int_ZF_2.html

Large diffs are not rendered by default.

258 changes: 129 additions & 129 deletions docs/IsarMathLib/Int_ZF_3.html

Large diffs are not rendered by default.

446 changes: 223 additions & 223 deletions docs/IsarMathLib/Int_ZF_IML.html

Large diffs are not rendered by default.

558 changes: 279 additions & 279 deletions docs/IsarMathLib/Introduction.html

Large diffs are not rendered by default.

84 changes: 42 additions & 42 deletions docs/IsarMathLib/Lattice_ZF.html

Large diffs are not rendered by default.

50 changes: 25 additions & 25 deletions docs/IsarMathLib/Loop_ZF.html

Large diffs are not rendered by default.

76 changes: 38 additions & 38 deletions docs/IsarMathLib/MMI_Complex_ZF.html

Large diffs are not rendered by default.

272 changes: 136 additions & 136 deletions docs/IsarMathLib/MMI_Complex_ZF_1.html

Large diffs are not rendered by default.

336 changes: 168 additions & 168 deletions docs/IsarMathLib/MMI_Complex_ZF_2.html

Large diffs are not rendered by default.

20 changes: 10 additions & 10 deletions docs/IsarMathLib/MMI_examples.html
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@
<h1>Theory MMI_examples</h1>
</div>

<pre class="source"><span class="comment1"><span>(</span><span>*</span><span>
<pre class="source"><span class="comment1"><span>(*
This file is a part of MMIsar - a translation of Metamath's set.mm to Isabelle 2005 (ZF logic).

Copyright (C) 2006 Slawomir Kolodynski
Expand All @@ -37,22 +37,22 @@ <h1>Theory MMI_examples</h1>
STRICT LIABILITY, OR TORT (INCLUDING NEGLIGENCE OR OTHERWISE) ARISING IN ANY WAY OUT OF THE
USE OF THIS SOFTWARE, EVEN IF ADVISED OF THE POSSIBILITY OF SUCH DAMAGE.

</span><span>*</span><span>)</span></span><span>
*)</span></span><span>

</span><span class="keyword1"><span class="command"><span>section</span></span></span><span> </span><span class="quoted"><span class="plain_text"><span></span><span>Metamath examples</span><span></span></span></span><span>
</span><span class="keyword1"><span class="command"><span>section</span></span></span><span> </span><span class="quoted"><span class="plain_text"><span>‹Metamath examples›</span></span></span><span>

</span><span class="keyword1"><span class="command"><span>theory</span></span></span><span> </span><a href="MMI_examples.html"><span>MMI_examples</span></a><span> </span><span class="keyword2"><span class="keyword"><span>imports</span></span></span><span> </span><a href="MMI_Complex_ZF.html"><span>MMI_Complex_ZF</span></a><span>

</span><span class="keyword2"><span class="keyword"><span>begin</span></span></span><span>

</span><span class="keyword1"><span class="command"><span>text</span></span></span><span class="quoted"><span class="plain_text"><span></span><span>This theory contains 10 theorems translated from
</span><span> Metamath (with proofs). It is included
</span><span> in the proof document as an illustration of how a translated
</span><span> Metamath proof looks like. The "known\_theorems.txt"
</span><span> file included in the IsarMathLib distribution provides
</span><span> a list of all translated facts.</span><span></span></span></span><span>
</span><span class="keyword1"><span class="command"><span>text</span></span></span><span class="quoted"><span class="plain_text"><span>‹This theory contains 10 theorems translated from
Metamath (with proofs). It is included
in the proof document as an illustration of how a translated
Metamath proof looks like. The "known\_theorems.txt"
file included in the IsarMathLib distribution provides
a list of all translated facts.›</span></span></span><span>

</span><span class="comment1"><span>(</span><span>*</span><span>*****201-210***************************</span><span>*</span><span>)</span></span><span>
</span><span class="comment1"><span>(******201-210****************************)</span></span><span>

</span><span class="keyword1"><span class="command"><span>lemma</span></span></span><span> </span><span class="main"><span>(</span></span><span class="keyword2"><span class="keyword"><span>in</span></span></span><span> </span><a class="entity_ref" href="MMI_prelude.html#MMI_prelude.MMIsar0|locale"><span>MMIsar0</span></a><span class="main"><span>)</span></span><span> </span><span class="entity_def" id="MMI_examples.MMIsar0.MMI_dividt|fact"><span class="entity_def" id="MMI_examples.MMIsar0.MMI_dividt|thm"><span>MMI_dividt</span></span></span><span class="main"><span>:</span></span><span>
</span><span class="keyword2"><span class="keyword"><span>shows</span></span></span><span> </span><span class="quoted"><span class="quoted"><span>"</span><span class="main"><span>(</span></span><span> </span><span class="free"><span>A</span></span><span> </span><span class="main"><a class="entity_ref" href="../../FOL/ZF/ZF_Base.html#ZF_Base.mem|const"><span></span></a></span><span> </span><span class="main"><span class="free"><span></span></span></span><span> </span><span class="main"><a class="entity_ref" href="../../FOL/ZF/IFOL.html#IFOL.conj|const"><span></span></a></span><span> </span><span class="free"><span>A</span></span><span> </span><span class="main"><a class="entity_ref" href="../../FOL/ZF/IFOL.html#IFOL.not_equal|const"><span></span></a></span><span> </span><span class="main"><span class="free"><span>𝟬</span></span></span><span> </span><span class="main"><span>)</span></span><span> </span><span class="main"><a class="entity_ref" href="../../FOL/ZF/IFOL.html#IFOL.imp|const"><span></span></a></span><span> </span><span class="main"><span>(</span></span><span> </span><span class="free"><span>A</span></span><span> </span><span class="main"><span class="free"><span>\&lt;cdiv&gt;</span></span></span><span> </span><span class="free"><span>A</span></span><span> </span><span class="main"><span>)</span></span><span> </span><span class="main"><a class="entity_ref" href="../../FOL/ZF/IFOL.html#IFOL.eq|const"><span>=</span></a></span><span> </span><span class="main"><span class="free"><span>𝟭</span></span></span><span>"</span></span></span><span>
Expand Down
Loading

0 comments on commit ea33786

Please sign in to comment.