src/HOL/Algebra/Algebra.thy
author wenzelm
Sat, 30 Oct 2021 21:07:20 +0200
changeset 74643 fde3a4a4f757
parent 70160 8e9100dcde52
child 77089 b4f892d0625d
permissions -rw-r--r--
provide native executables for arm64-darwin, for more robust startup without Rosetta 2;

(*  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
begin
end