aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/trac/trac-200.thy
blob: 96a0c177c6b8cbc105db7e3a08426f617d0386c7 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
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