| changeset 69785 | 9e326f6f8a24 |
| parent 66276 | acc3b7dd0b21 |
| child 69790 | 154cf64e403e |
--- a/src/HOL/Number_Theory/Number_Theory.thy Sat Feb 02 15:52:14 2019 +0100 +++ b/src/HOL/Number_Theory/Number_Theory.thy Mon Feb 04 12:16:03 2019 +0100 @@ -2,7 +2,14 @@ section \<open>Comprehensive number theory\<close> theory Number_Theory -imports Fib Residues Eratosthenes Quadratic_Reciprocity Pocklington Prime_Powers +imports + Fib + Residues + Eratosthenes + Quadratic_Reciprocity + Pocklington + Prime_Powers + Residue_Primitive_Roots begin end