aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/trac/trac-200.thy
blob: fabd04f61e59f4f96f9d06ef8af296d80dd6af43 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
(* See trac #200 *)
theory Trac200 imports Main begin

(* Test simulating sledgehammer asynchronous output *)

ML {* Thread.fork (fn () =>
  (OS.Process.sleep (Time.fromSeconds 3); priority "urgent message"), []) *}

(* Want to preserve correct term output *)

term "x"

end