src/HOL/Nitpick_Examples/Manual_Nits.thy
changeset 49812 e3945ddcb9aa
parent 48812 9509fc5485b2
child 49834 b27bbb021df1
equal deleted inserted replaced
49811:3fc6b3289c31 49812:e3945ddcb9aa
    92 nitpick [show_datatypes, expect = genuine]
    92 nitpick [show_datatypes, expect = genuine]
    93 oops
    93 oops
    94 
    94 
    95 subsection {* 2.7. Typedefs, Records, Rationals, and Reals *}
    95 subsection {* 2.7. Typedefs, Records, Rationals, and Reals *}
    96 
    96 
    97 typedef three = "{0\<Colon>nat, 1, 2}"
    97 definition "three = {0\<Colon>nat, 1, 2}"
    98 by blast
    98 typedef (open) three = three
       
    99   unfolding three_def by blast
    99 
   100 
   100 definition A :: three where "A \<equiv> Abs_three 0"
   101 definition A :: three where "A \<equiv> Abs_three 0"
   101 definition B :: three where "B \<equiv> Abs_three 1"
   102 definition B :: three where "B \<equiv> Abs_three 1"
   102 definition C :: three where "C \<equiv> Abs_three 2"
   103 definition C :: three where "C \<equiv> Abs_three 2"
   103 
   104