src/Doc/JEdit/Base.thy
author wenzelm
Wed, 19 Apr 2017 16:24:59 +0200
changeset 65511 ea42dfd95ec8
parent 61656 cfabbc083977
child 69605 a96320074298
permissions -rw-r--r--
optionally explore all sessions -- potentially slow, e.g. for AFP;

(*:maxLineLen=78:*)

theory Base
imports Main
begin

ML_file "../antiquote_setup.ML"

end