lh-l4v/lib/Defs.thy

19 lines
352 B
Plaintext
Raw Normal View History

(*
2020-03-09 06:18:30 +00:00
* Copyright 2020, Data61, CSIRO (ABN 41 687 119 230)
*
2020-03-09 06:18:30 +00:00
* SPDX-License-Identifier: BSD-2-Clause
*)
2017-07-12 05:13:51 +00:00
(* Resurrect old "defs" command which was removed in Isabelle 2016.
* Should be replaced with overloading..definition..end blocks. *)
theory Defs
imports Main
keywords "defs" :: thy_decl and "consts'" :: thy_decl
begin
ML_file "defs.ML"
end