src/HOL/Computational_Algebra/Computational_Algebra.thy
author paulson <lp15@cam.ac.uk>
Fri, 22 Dec 2017 21:00:07 +0000
changeset 67268 bdf25939a550
parent 67165 22a5822f52f7
child 69791 195aeee8b30a
permissions -rw-r--r--
new/improved theories involving convergence; better pretty-printing for bounded quantifiers and sum/product


section \<open>Pieces of computational Algebra\<close>

theory Computational_Algebra
imports
  Euclidean_Algorithm
  Factorial_Ring
  Formal_Power_Series
  Fraction_Field
  Fundamental_Theorem_Algebra
  Group_Closure
  Normalized_Fraction
  Nth_Powers
  Polynomial_FPS
  Polynomial
  Polynomial_Factorial
  Primes
  Squarefree
begin

end