src/Pure/Isar/proof.ML
changeset 41677 fa0da47131d2
parent 41181 9240be8c8c69
child 42042 264f8d0e899f
equal deleted inserted replaced
41676:4639f40b20c9 41677:fa0da47131d2
  1098 local
  1098 local
  1099 
  1099 
  1100 fun future_terminal_proof proof1 proof2 meths int state =
  1100 fun future_terminal_proof proof1 proof2 meths int state =
  1101   if int orelse is_relevant state orelse not (Goal.local_future_enabled ())
  1101   if int orelse is_relevant state orelse not (Goal.local_future_enabled ())
  1102   then proof1 meths state
  1102   then proof1 meths state
  1103   else snd (proof2 (fn state' => Goal.fork (fn () => ((), proof1 meths state'))) state);
  1103   else snd (proof2 (fn state' =>
       
  1104     Goal.fork_name "Proof.future_terminal_proof" (fn () => ((), proof1 meths state'))) state);
  1104 
  1105 
  1105 in
  1106 in
  1106 
  1107 
  1107 fun local_future_terminal_proof x =
  1108 fun local_future_terminal_proof x =
  1108   future_terminal_proof local_terminal_proof local_future_proof x;
  1109   future_terminal_proof local_terminal_proof local_future_proof x;