src/HOL/Nonstandard_Analysis/Examples/NSPrimes.thy
changeset 65417 fc41a5650fb1
parent 64601 37ce6ceacbb7
child 66453 cc19f7ca2ed6
equal deleted inserted replaced
65416:f707dbcf11e3 65417:fc41a5650fb1
     5 *)
     5 *)
     6 
     6 
     7 section \<open>The Nonstandard Primes as an Extension of the Prime Numbers\<close>
     7 section \<open>The Nonstandard Primes as an Extension of the Prime Numbers\<close>
     8 
     8 
     9 theory NSPrimes
     9 theory NSPrimes
    10   imports "~~/src/HOL/Number_Theory/Primes" "../Hyperreal"
    10   imports "~~/src/HOL/Computational_Algebra/Primes" "../Hyperreal"
    11 begin
    11 begin
    12 
    12 
    13 text \<open>These can be used to derive an alternative proof of the infinitude of
    13 text \<open>These can be used to derive an alternative proof of the infinitude of
    14 primes by considering a property of nonstandard sets.\<close>
    14 primes by considering a property of nonstandard sets.\<close>
    15 
    15