src/HOL/NSA/NSA.thy
changeset 28952 15a4b2cf8c34
parent 28562 4e74209f113e
child 30080 4cf42465b3da
equal deleted inserted replaced
28948:1860f016886d 28952:15a4b2cf8c34
     6 *)
     6 *)
     7 
     7 
     8 header{*Infinite Numbers, Infinitesimals, Infinitely Close Relation*}
     8 header{*Infinite Numbers, Infinitesimals, Infinitely Close Relation*}
     9 
     9 
    10 theory NSA
    10 theory NSA
    11 imports HyperDef "../Real/RComplete"
    11 imports HyperDef RComplete
    12 begin
    12 begin
    13 
    13 
    14 definition
    14 definition
    15   hnorm :: "'a::norm star \<Rightarrow> real star" where
    15   hnorm :: "'a::norm star \<Rightarrow> real star" where
    16   [transfer_unfold]: "hnorm = *f* norm"
    16   [transfer_unfold]: "hnorm = *f* norm"