src/HOL/Complex/ex/Sqrt_Script.thy
changeset 21404 eb85850d3eb7
parent 19736 d8d0f8f51d69
child 27651 16a26996c30e
equal deleted inserted replaced
21403:dd58f13a8eb4 21404:eb85850d3eb7
    51 
    51 
    52 
    52 
    53 subsection {* The set of rational numbers *}
    53 subsection {* The set of rational numbers *}
    54 
    54 
    55 definition
    55 definition
    56   rationals :: "real set"    ("\<rat>")
    56   rationals :: "real set"    ("\<rat>") where
    57   "\<rat> = {x. \<exists>m n. n \<noteq> 0 \<and> \<bar>x\<bar> = real (m::nat) / real (n::nat)}"
    57   "\<rat> = {x. \<exists>m n. n \<noteq> 0 \<and> \<bar>x\<bar> = real (m::nat) / real (n::nat)}"
    58 
    58 
    59 
    59 
    60 subsection {* Main theorem *}
    60 subsection {* Main theorem *}
    61 
    61