Skip to content

Commit

Permalink
coqide: Add preference for unjustified conclusions’ background color
Browse files Browse the repository at this point in the history
  • Loading branch information
Frigory33 committed Aug 10, 2024
1 parent ac6aabe commit 0b8ee14
Show file tree
Hide file tree
Showing 4 changed files with 7 additions and 3 deletions.
6 changes: 4 additions & 2 deletions ide/coqide/preferences.ml
Original file line number Diff line number Diff line change
Expand Up @@ -498,8 +498,6 @@ let create_tag name default =
List.iter iter [Tags.Script.table; Tags.Proof.table; Tags.Message.table];
tags := Util.String.Map.add name pref !tags

(* note these appear to only set the defaults; they don't override
the user selection from the Edit/Preferences/Tags dialog *)
let () =
let iter (name, tag) = create_tag name tag in
List.iter iter [
Expand Down Expand Up @@ -537,8 +535,12 @@ let processing_color =
let incompletely_processed_color =
new preference ~name:["incompletely_processed_color"] ~init:"light sky blue" ~repr:Repr.(string)

let unjustified_conclusion_color =
new preference ~name:["unjustified_conclusion_color"] ~init:"gold" ~repr:Repr.(string)

let _ = attach_bg processing_color Tags.Script.to_process
let _ = attach_bg incompletely_processed_color Tags.Script.incomplete
let _ = attach_bg unjustified_conclusion_color Tags.Script.unjustified

let breakpoint_color =
new preference ~name:["breakpoint_color"] ~init:"#db5860" ~repr:Repr.(string)
Expand Down
1 change: 1 addition & 0 deletions ide/coqide/preferences.mli
Original file line number Diff line number Diff line change
Expand Up @@ -100,6 +100,7 @@ val document_tabs_pos : string preference
val processing_color : string preference
val processed_color : string preference
val incompletely_processed_color : string preference
val unjustified_conclusion_color : string preference
val breakpoint_color : string preference
val db_stopping_point_color : string preference
val error_color : string preference
Expand Down
1 change: 1 addition & 0 deletions ide/coqide/preferences_ui.ml
Original file line number Diff line number Diff line change
Expand Up @@ -542,6 +542,7 @@ let configure ?(apply = fun () -> ()) parent =
"Processed text", [processed_color];
"Text being processed", [processing_color];
"Incompletely processed Qed", [incompletely_processed_color];
"Unjustified conclusions", [unjustified_conclusion_color];
"Breakpoints", [breakpoint_color];
"Debugger stopping point", [db_stopping_point_color];
"Errors", [error_color; error_fg_color];
Expand Down
2 changes: 1 addition & 1 deletion ide/coqide/tags.ml
Original file line number Diff line number Diff line change
Expand Up @@ -26,7 +26,7 @@ struct
let processed = make_tag table ~name:"processed" []
let debugging = make_tag table ~name:"debugging" []
let incomplete = make_tag table ~name:"incomplete" [`EDITABLE false]
let unjustified = make_tag table ~name:"unjustified" [`BACKGROUND "gold"]
let unjustified = make_tag table ~name:"unjustified" []
let tooltip = make_tag table ~name:"tooltip" [] (* debug:`BACKGROUND "blue" *)
let ephemere =
[warning; error; error_bg; to_process; processed; debugging;
Expand Down

0 comments on commit 0b8ee14

Please sign in to comment.