src/HOL/ex/Hex_Bin_Examples.thy
changeset 69597 ff784d5a5bfb
parent 61343 5b5656a63bd6
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
    23 
    23 
    24 text "Unary minus works as for decimal numerals"
    24 text "Unary minus works as for decimal numerals"
    25 lemma "- 0x0A = - 10" by (rule refl)
    25 lemma "- 0x0A = - 10" by (rule refl)
    26 
    26 
    27 text \<open>
    27 text \<open>
    28   Hex and bin numerals are printed as decimal: @{term "0b10"}
    28   Hex and bin numerals are printed as decimal: \<^term>\<open>0b10\<close>
    29 \<close>
    29 \<close>
    30 term "0b10"
    30 term "0b10"
    31 term "0x0A"
    31 term "0x0A"
    32 
    32 
    33 text \<open>
    33 text \<open>