src/HOL/Nitpick_Examples/Typedef_Nits.thy
changeset 54633 86e0b402994c
parent 51706 0a4b4735d8bd
child 54680 93f6d33a754e
equal deleted inserted replaced
54632:7a14f831d02d 54633:86e0b402994c
     9 
     9 
    10 theory Typedef_Nits
    10 theory Typedef_Nits
    11 imports Complex_Main
    11 imports Complex_Main
    12 begin
    12 begin
    13 
    13 
    14 nitpick_params [verbose, card = 1\<emdash>4, sat_solver = MiniSat_JNI, max_threads = 1,
    14 nitpick_params [verbose, card = 1\<emdash>4, sat_solver = Riss3g, max_threads = 1,
    15                 timeout = 240]
    15                 timeout = 240]
    16 
    16 
    17 definition "three = {0\<Colon>nat, 1, 2}"
    17 definition "three = {0\<Colon>nat, 1, 2}"
    18 typedef three = three
    18 typedef three = three
    19 unfolding three_def by blast
    19 unfolding three_def by blast