src/Doc/System/Base.thy
author wenzelm
Thu, 24 Apr 2014 13:10:42 +0200
changeset 56694 c4e77643aad6
parent 56059 2390391584c2
child 61656 cfabbc083977
permissions -rw-r--r--
proper signaling after each state update (NB: ML version does this uniformly via timed_access);

theory Base
imports Pure
begin

ML_file "../antiquote_setup.ML"

end