(* Title: HOL/Nitpick_Examples/Hotel_Nits.thy Author: Jasmin Blanchette, TU Muenchen Copyright 2010-2011 Nitpick example based on Tobias Nipkow's hotel key card formalization. *) section ‹Nitpick Example Based on Tobias Nipkow's Hotel Key Card Formalization› theory Hotel_Nits imports Main begin nitpick_params [verbose, max_potential = 0, sat_solver = MiniSat, max_threads = 1, timeout = 240] typedecl guest typedecl key typedecl room type_synonym keycard = "key × key"