src/HOL/Nitpick_Examples/Record_Nits.thy
changeset 35284 9edc2bd6d2bd
parent 35078 6fd1052fe463
child 38185 b51677438b3a
equal deleted inserted replaced
35283:7ae51d5ea05d 35284:9edc2bd6d2bd
     9 
     9 
    10 theory Record_Nits
    10 theory Record_Nits
    11 imports Main
    11 imports Main
    12 begin
    12 begin
    13 
    13 
    14 nitpick_params [sat_solver = MiniSat_JNI, max_threads = 1, timeout = 60 s]
    14 nitpick_params [max_potential = 0, sat_solver = MiniSat_JNI, max_threads = 1,
       
    15                 timeout = 60 s]
    15 
    16 
    16 record point2d =
    17 record point2d =
    17   xc :: int
    18   xc :: int
    18   yc :: int
    19   yc :: int
    19 
    20