src/HOL/HOL.thy
changeset 32740 9dd0a2f83429
parent 32734 06c13b2e562e
child 33022 c95102496490
equal deleted inserted replaced
32739:31e75ad9ae17 32740:9dd0a2f83429
  1968 
  1968 
  1969 ML {*
  1969 ML {*
  1970 structure Eval_Method =
  1970 structure Eval_Method =
  1971 struct
  1971 struct
  1972 
  1972 
  1973 val eval_ref : (unit -> bool) option ref = ref NONE;
  1973 val eval_ref : (unit -> bool) option Unsynchronized.ref = Unsynchronized.ref NONE;
  1974 
  1974 
  1975 end;
  1975 end;
  1976 *}
  1976 *}
  1977 
  1977 
  1978 oracle eval_oracle = {* fn ct =>
  1978 oracle eval_oracle = {* fn ct =>