lh-l4v/lib/Crunch.thy

27 lines
518 B
Plaintext
Raw Normal View History

2014-07-14 19:32:44 +00:00
(*
* Copyright 2014, NICTA
*
* This software may be distributed and modified according to the terms of
* the BSD 2-Clause license. Note that NO WARRANTY is provided.
* See "LICENSE_BSD2.txt" for details.
*
* @TAG(NICTA_BSD)
*)
theory Crunch
imports
"Monad_WP/wp/WPSimp"
Lib
"ml-helpers/MLUtils"
keywords "crunch" "crunch_ignore" "crunches" :: thy_decl
2014-07-14 19:32:44 +00:00
begin
named_theorems "crunch_def"
named_theorems "crunch_rules"
named_theorems "crunch_param_rules"
2014-07-14 19:32:44 +00:00
ML_file "crunch-cmd.ML"
ML_file "Crunch.ML"
end