src/HOL/Complex/ex/NSPrimes.thy
changeset 19736 d8d0f8f51d69
parent 17429 e8d6ed3aacfe
child 20733 4ccef1ac4c9b
--- a/src/HOL/Complex/ex/NSPrimes.thy	Sat May 27 17:42:00 2006 +0200
+++ b/src/HOL/Complex/ex/NSPrimes.thy	Sat May 27 17:42:02 2006 +0200
@@ -13,22 +13,15 @@
 text{*These can be used to derive an alternative proof of the infinitude of
 primes by considering a property of nonstandard sets.*}
 
-
-constdefs
+definition
   hdvd  :: "[hypnat, hypnat] => bool"       (infixl "hdvd" 50)
-   "(M::hypnat) hdvd N == ( *p2* (op dvd)) M N"
-
-declare hdvd_def [transfer_unfold]
+  [transfer_unfold]: "(M::hypnat) hdvd N = ( *p2* (op dvd)) M N"
 
-constdefs
   starprime :: "hypnat set"
-  "starprime == ( *s* {p. prime p})"
+  [transfer_unfold]: "starprime = ( *s* {p. prime p})"
 
-declare starprime_def [transfer_unfold]
-
-constdefs
   choicefun :: "'a set => 'a"
-  "choicefun E == (@x. \<exists>X \<in> Pow(E) -{{}}. x : X)"
+  "choicefun E = (@x. \<exists>X \<in> Pow(E) -{{}}. x : X)"
 
 consts injf_max :: "nat => ('a::{order} set) => 'a"
 primrec