equal
deleted
inserted
replaced
106 @{index_ML eta_contract: "bool Unsynchronized.ref"} & default @{ML true} \\ |
106 @{index_ML eta_contract: "bool Unsynchronized.ref"} & default @{ML true} \\ |
107 @{index_ML goals_limit: "int Unsynchronized.ref"} & default @{ML 10} \\ |
107 @{index_ML goals_limit: "int Unsynchronized.ref"} & default @{ML 10} \\ |
108 @{index_ML Proof.show_main_goal: "bool Unsynchronized.ref"} & default @{ML false} \\ |
108 @{index_ML Proof.show_main_goal: "bool Unsynchronized.ref"} & default @{ML false} \\ |
109 @{index_ML show_hyps: "bool Unsynchronized.ref"} & default @{ML false} \\ |
109 @{index_ML show_hyps: "bool Unsynchronized.ref"} & default @{ML false} \\ |
110 @{index_ML show_tags: "bool Unsynchronized.ref"} & default @{ML false} \\ |
110 @{index_ML show_tags: "bool Unsynchronized.ref"} & default @{ML false} \\ |
111 @{index_ML show_question_marks: "bool Unsynchronized.ref"} & default @{ML true} \\ |
111 @{index_ML show_question_marks: "bool Config.T"} & default @{ML true} \\ |
112 \end{mldecls} |
112 \end{mldecls} |
113 |
113 |
114 These global ML variables control the detail of information that is |
114 These global ML variables control the detail of information that is |
115 displayed for types, terms, theorems, goals etc. |
115 displayed for types, terms, theorems, goals etc. |
116 |
116 |