diff -r 95d7459e5bc0 -r b6589c8ccadd src/HOL/Algebra/README.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Algebra/README.thy Fri Aug 19 23:58:44 2022 +0200 @@ -0,0 +1,74 @@ +theory README imports Main +begin + +section \Algebra --- Classical Algebra, using Explicit Structures and Locales\ + +text \ + This directory contains proofs in classical algebra. It is intended as a + base for any algebraic development in Isabelle. Emphasis is on reusability. + This is achieved by modelling algebraic structures as first-class citizens + of the logic (not axiomatic type classes, say). The library is expected to + grow in future releases of Isabelle. Contributions are welcome. +\ + +subsection \GroupTheory, including Sylow's Theorem\ + +text \ + These proofs are mainly by Florian Kammüller. (Later, Larry Paulson + simplified some of the proofs.) These theories were indeed the original + motivation for locales. + + Here is an outline of the directory's contents: + + \<^item> Theory \<^file>\Group.thy\ defines semigroups, monoids, groups, commutative + monoids, commutative groups, homomorphisms and the subgroup relation. It + also defines the product of two groups (This theory was reimplemented by + Clemens Ballarin). + + \<^item> Theory \<^file>\FiniteProduct.thy\ extends commutative groups by a product + operator for finite sets (provided by Clemens Ballarin). + + \<^item> Theory \<^file>\Coset.thy\ defines the factorization of a group and shows that + the factorization a normal subgroup is a group. + + \<^item> Theory \<^file>\Bij.thy\ defines bijections over sets and operations on them and + shows that they are a group. It shows that automorphisms form a group. + + \<^item> Theory \<^file>\Exponent.thy\ the combinatorial argument underlying Sylow's + first theorem. + + \<^item> Theory \<^file>\Sylow.thy\ contains a proof of the first Sylow theorem. +\ + + +subsection \Rings and Polynomials\ + +text \ + \<^item> Theory \<^file>\Ring.thy\ defines Abelian monoids and groups. The difference to + commutative structures is merely notational: the binary operation is + addition rather than multiplication. Commutative rings are obtained by + inheriting properties from Abelian groups and commutative monoids. Further + structures in the algebraic hierarchy of rings: integral domain. + + \<^item> Theory \<^file>\Module.thy\ introduces the notion of a R-left-module over an + Abelian group, where R is a ring. + + \<^item> Theory \<^file>\UnivPoly.thy\ constructs univariate polynomials over rings and + integral domains. Degree function. Universal Property. +\ + + +subsection \Development of Polynomials using Type Classes\ + +text \ + A development of univariate polynomials for HOL's ring classes is available + at \<^file>\~~/src/HOL/Computational_Algebra/Polynomial.thy\. + + [Jacobson1985] Nathan Jacobson, Basic Algebra I, Freeman, 1985. + + [Ballarin1999] Clemens Ballarin, Computer Algebra and Theorem Proving, + Author's PhD thesis, 1999. Also University of Cambridge, Computer Laboratory + Technical Report number 473. +\ + +end