src/HOL/Algebra/Algebra.thy
author Fabian Huch <huch@in.tum.de>
Wed, 24 Jan 2024 18:41:21 +0100
changeset 79527 f1f08ca40d96
parent 77406 c2013f617a70
child 80084 173548e4d5d0
permissions -rw-r--r--
make build process state protected to avoid copying in subclasses (e.g. for database connections);

(*  Title:      HOL/Algebra/Algebra.thy *)

theory Algebra
  imports Sylow Chinese_Remainder Zassenhaus Galois_Connection Generated_Fields Free_Abelian_Groups
     Divisibility Embedded_Algebras IntRing Sym_Groups Exact_Sequence Polynomials Algebraic_Closure
     Left_Coset SimpleGroups SndIsomorphismGrp
begin
end