always expand all paths
authorblanchet
Thu, 26 Jun 2014 19:40:58 +0200
changeset 57386 5980ee29dbf6
parent 57385 0eb0c7b93676
child 57387 2b6fe2a48352
always expand all paths
src/HOL/Tools/Sledgehammer/sledgehammer_mash.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_mash.ML	Thu Jun 26 19:10:34 2014 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_mash.ML	Thu Jun 26 19:40:58 2014 +0200
@@ -129,7 +129,9 @@
 fun add_to_xtab key (next, tab) = (next + 1, Symtab.update_new (key, next) tab)
 fun maybe_add_to_xtab key = perhaps (try (add_to_xtab key))
 
-fun mash_state_dir () = Path.explode "$ISABELLE_HOME_USER/mash" |> tap Isabelle_System.mkdir
+fun mash_state_dir () =
+  Path.expand (Path.explode "$ISABELLE_HOME_USER/mash" |> tap Isabelle_System.mkdir)
+
 fun mash_state_file () = Path.append (mash_state_dir ()) (Path.explode "state")
 
 fun wipe_out_mash_state_dir () =
@@ -744,7 +746,7 @@
 
 fun load_state ctxt overlord (time_state as (memory_time, _)) =
   let val path = mash_state_file () in
-    (case try OS.FileSys.modTime (Path.implode (Path.expand path)) of
+    (case try OS.FileSys.modTime (Path.implode path) of
       NONE => time_state
     | SOME disk_time =>
       if Time.>= (memory_time, disk_time) then
@@ -1292,7 +1294,7 @@
 fun weight_facts_steeply facts =
   facts ~~ map steep_weight_of_fact (0 upto length facts - 1)
 
-val max_proximity_facts = 0 (*###*)
+val max_proximity_facts = 100
 
 fun find_mash_suggestions ctxt max_facts suggs facts chained raw_unknown =
   let
@@ -1722,7 +1724,7 @@
           let val timeout = time_mult learn_timeout_slack timeout in
             Output.urgent_message ("Started MaShing through at least " ^
               string_of_int min_num_facts_to_learn ^ " fact" ^ plural_s min_num_facts_to_learn ^
-              " in the background");
+              " in the background.");
             launch_thread timeout
               (fn () => (true, mash_learn_facts ctxt params prover true 2 false timeout facts))
           end