src/HOL/Old_Number_Theory/Factorization.thy
changeset 41413 64cd30d6b0b8
parent 38159 e9b4835a54ee
child 44890 22f665a2e91c
--- a/src/HOL/Old_Number_Theory/Factorization.thy	Wed Dec 29 13:51:17 2010 +0100
+++ b/src/HOL/Old_Number_Theory/Factorization.thy	Wed Dec 29 17:34:41 2010 +0100
@@ -6,7 +6,7 @@
 header {* Fundamental Theorem of Arithmetic (unique factorization into primes) *}
 
 theory Factorization
-imports Primes Permutation
+imports Primes "~~/src/HOL/Library/Permutation"
 begin