src/Doc/Tutorial/Types/Numbers.thy
changeset 69597 ff784d5a5bfb
parent 68636 f33ffa0a27a1
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
    15 
    15 
    16 fun h :: "nat \<Rightarrow> nat" where
    16 fun h :: "nat \<Rightarrow> nat" where
    17 "h i = (if i = 3 then 2 else i)"
    17 "h i = (if i = 3 then 2 else i)"
    18 
    18 
    19 text\<open>
    19 text\<open>
    20 @{term"h 3 = 2"}
    20 \<^term>\<open>h 3 = 2\<close>
    21 @{term"h i  = i"}
    21 \<^term>\<open>h i  = i\<close>
    22 \<close>
    22 \<close>
    23 
    23 
    24 text\<open>
    24 text\<open>
    25 @{thm[display] numeral_One[no_vars]}
    25 @{thm[display] numeral_One[no_vars]}
    26 \rulename{numeral_One}
    26 \rulename{numeral_One}