src/HOL/Nitpick_Examples/Record_Nits.thy
changeset 34083 652719832159
parent 33197 de6285ebcc05
child 35076 cc19e2aef17e
equal deleted inserted replaced
34082:61b7aa37f4b7 34083:652719832159
     8 header {* Examples Featuring Nitpick Applied to Records *}
     8 header {* Examples Featuring Nitpick Applied to Records *}
     9 
     9 
    10 theory Record_Nits
    10 theory Record_Nits
    11 imports Main
    11 imports Main
    12 begin
    12 begin
       
    13 
       
    14 nitpick_params [sat_solver = MiniSatJNI, max_threads = 1, timeout = 60 s]
    13 
    15 
    14 record point2d =
    16 record point2d =
    15   xc :: int
    17   xc :: int
    16   yc :: int
    18   yc :: int
    17 
    19