src/Doc/Implementation/Base.thy
author wenzelm
Tue, 22 Sep 2015 22:38:22 +0200
changeset 61255 15865e0c5598
parent 56420 b266e7a86485
child 61656 cfabbc083977
permissions -rw-r--r--
eliminated separate type Theory.dep: use typeargs uniformly for consts/types; Object_Logic.add_judgment more like Theory.specify_const;

theory Base
imports Main
begin

ML_file "../antiquote_setup.ML"

end