src/Pure/Isar/proof.ML
changeset 79113 5109e4b2a292
parent 78705 fde0b195cb7d
equal deleted inserted replaced
79112:fd9de06c0ecf 79113:5109e4b2a292
  1337 
  1337 
  1338 local
  1338 local
  1339 
  1339 
  1340 fun future_terminal_proof proof1 proof2 done state =
  1340 fun future_terminal_proof proof1 proof2 done state =
  1341   if Future.proofs_enabled 3 andalso
  1341   if Future.proofs_enabled 3 andalso
  1342     not (Proofterm.proofs_enabled ()) andalso
  1342     not (Proofterm.any_proofs_enabled ()) andalso
  1343     not (is_relevant state)
  1343     not (is_relevant state)
  1344   then
  1344   then
  1345     state |> future_proof (fn state' =>
  1345     state |> future_proof (fn state' =>
  1346       let val pos = Position.thread_data () in
  1346       let val pos = Position.thread_data () in
  1347         Execution.fork {name = "Proof.future_terminal_proof", pos = pos, pri = ~1}
  1347         Execution.fork {name = "Proof.future_terminal_proof", pos = pos, pri = ~1}