src/HOL/Nunchaku/Nunchaku.thy
author blanchet
Wed, 26 Oct 2016 15:21:16 +0200
changeset 64407 5c5b9d945625
parent 64389 6273d4c8325b
child 64469 488d4e627238
permissions -rw-r--r--
proper Nunchaku setup to use CVC4 and Kodkod

(*  Title:      HOL/Nunchaku/Nunchaku.thy
    Author:     Jasmin Blanchette, Inria Nancy, LORIA, MPII
    Copyright   2015, 2016

Nunchaku: Yet another counterexample generator for Isabelle/HOL.

Nunchaku relies on an external program of the same name. The program is still
being actively developed. The sources are available at

    https://github.com/nunchaku-inria

The "$NUNCHAKU" environment variable must be set to the absolute file name of
the "nunchaku" executable. The Isabelle components for CVC4 and Kodkodi are
necessary to use these backends.
*)

theory Nunchaku
imports Main
keywords
  "nunchaku" :: diag and
  "nunchaku_params" :: thy_decl
begin

consts unreachable :: 'a

definition The_unsafe :: "('a \<Rightarrow> bool) \<Rightarrow> 'a" where
  "The_unsafe = The"

definition rmember :: "'a set \<Rightarrow> 'a \<Rightarrow> bool" where
  "rmember A x \<longleftrightarrow> x \<in> A"

ML_file "Tools/nunchaku_util.ML"
ML_file "Tools/nunchaku_collect.ML"
ML_file "Tools/nunchaku_problem.ML"
ML_file "Tools/nunchaku_translate.ML"
ML_file "Tools/nunchaku_model.ML"
ML_file "Tools/nunchaku_reconstruct.ML"
ML_file "Tools/nunchaku_display.ML"
ML_file "Tools/nunchaku_tool.ML"
ML_file "Tools/nunchaku.ML"
ML_file "Tools/nunchaku_commands.ML"

hide_const (open) unreachable The_unsafe rmember

end