src/HOL/Nonstandard_Analysis/Examples/NSPrimes.thy
changeset 66453 cc19f7ca2ed6
parent 65417 fc41a5650fb1
child 70749 5d06b7bb9d22
equal deleted inserted replaced
66452:450cefec7c11 66453:cc19f7ca2ed6
     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/Computational_Algebra/Primes" "../Hyperreal"
    10   imports "HOL-Computational_Algebra.Primes" "HOL-Nonstandard_Analysis.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