src/HOL/Library/Float.thy
changeset 59487 adaa430fc0f7
parent 58989 99831590def5
child 59554 4044f53326c9
equal deleted inserted replaced
59486:2025a17bb20f 59487:adaa430fc0f7
    25 end
    25 end
    26 
    26 
    27 lemma type_definition_float': "type_definition real float_of float"
    27 lemma type_definition_float': "type_definition real float_of float"
    28   using type_definition_float unfolding real_of_float_def .
    28   using type_definition_float unfolding real_of_float_def .
    29 
    29 
    30 setup_lifting (no_code) type_definition_float'
    30 setup_lifting type_definition_float'
    31 
    31 
    32 lemmas float_of_inject[simp]
    32 lemmas float_of_inject[simp]
    33 
    33 
    34 declare [[coercion "real :: float \<Rightarrow> real"]]
    34 declare [[coercion "real :: float \<Rightarrow> real"]]
    35 
    35