src/HOL/Computational_Algebra/Computational_Algebra.thy
author eberlm <eberlm@in.tum.de>
Sat, 15 Jul 2017 14:32:02 +0100
changeset 66276 acc3b7dd0b21
parent 65417 fc41a5650fb1
child 66805 274b4edca859
permissions -rw-r--r--
More material on powers for HOL-Computational_Algebra/HOL-Number_Theory


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

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

end