Skip to content

Commit

Permalink
Reducing CoqIDE start option queries.
Browse files Browse the repository at this point in the history
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15344 85f007b7-540e-0410-9357-904b9bb8a0f7
  • Loading branch information
ppedrot committed May 23, 2012
1 parent a2e1cc5 commit f657fac
Showing 1 changed file with 5 additions and 2 deletions.
7 changes: 5 additions & 2 deletions ide/coqide.ml
Expand Up @@ -1241,8 +1241,11 @@ let create_session file =
let _ =
GtkBase.Widget.add_events proof#as_widget [`ENTER_NOTIFY;`POINTER_MOTION] in
let () =
Coq.grab ct (fun handle ->
List.iter (fun (opts,_,_,_,dflt) -> setopts handle opts dflt) print_items) in
let fold accu (opts, _, _, _, dflt) =
List.fold_left (fun accu opt -> (opt, dflt) :: accu) accu opts
in
let options = List.fold_left fold [] print_items in
Coq.grab ct (fun handle -> Coq.PrintOpt.set handle options) in
let _ =
proof#event#connect#motion_notify ~callback:
(fun e ->
Expand Down

0 comments on commit f657fac

Please sign in to comment.