| author | paulson <lp15@cam.ac.uk> | 
| Tue, 01 Mar 2022 15:05:27 +0000 | |
| changeset 75168 | ff60b4acd6dd | 
| parent 70817 | dd675800469d | 
| permissions | -rw-r--r-- | 
| 65417 | 1 | |
| 2 | section \<open>Pieces of computational Algebra\<close> | |
| 3 | ||
| 4 | theory Computational_Algebra | |
| 5 | imports | |
| 6 | Euclidean_Algorithm | |
| 7 | Factorial_Ring | |
| 69791 
195aeee8b30a
Formal Laurent series and overhaul of Formal power series (due to Jeremy Sylvestre)
 Manuel Eberl <eberlm@in.tum.de> parents: 
67165diff
changeset | 8 | Formal_Laurent_Series | 
| 65417 | 9 | Fraction_Field | 
| 10 | Fundamental_Theorem_Algebra | |
| 67165 | 11 | Group_Closure | 
| 65417 | 12 | Normalized_Fraction | 
| 66276 
acc3b7dd0b21
More material on powers for HOL-Computational_Algebra/HOL-Number_Theory
 eberlm <eberlm@in.tum.de> parents: 
65417diff
changeset | 13 | Nth_Powers | 
| 65417 | 14 | Polynomial_FPS | 
| 15 | Polynomial | |
| 66805 
274b4edca859
Polynomial_Factorial does not depend on Field_as_Ring as such
 haftmann parents: 
66276diff
changeset | 16 | Polynomial_Factorial | 
| 65417 | 17 | Primes | 
| 66276 
acc3b7dd0b21
More material on powers for HOL-Computational_Algebra/HOL-Number_Theory
 eberlm <eberlm@in.tum.de> parents: 
65417diff
changeset | 18 | Squarefree | 
| 65417 | 19 | begin | 
| 20 | ||
| 21 | end |