diff -r f06e5a5a4b46 -r a9599d3d7610 src/HOL/Library/Old_SMT.thy --- a/src/HOL/Library/Old_SMT.thy Thu Nov 05 10:35:37 2015 +0100 +++ b/src/HOL/Library/Old_SMT.thy Thu Nov 05 10:39:49 2015 +0100 @@ -51,7 +51,7 @@ definition weight :: "int \ bool \ bool" where "weight _ P = P" text \ -Weights must be non-negative. The value @{text 0} is equivalent to providing +Weights must be non-negative. The value \0\ is equivalent to providing no weight at all. Weights should only be used at quantifiers and only inside triggers (if the @@ -150,7 +150,7 @@ text \ The current configuration can be printed by the command -@{text old_smt_status}, which shows the values of most options. +\old_smt_status\, which shows the values of most options. \ @@ -158,14 +158,14 @@ subsection \General configuration options\ text \ -The option @{text old_smt_solver} can be used to change the target SMT -solver. The possible values can be obtained from the @{text old_smt_status} +The option \old_smt_solver\ can be used to change the target SMT +solver. The possible values can be obtained from the \old_smt_status\ command. Due to licensing restrictions, Yices and Z3 are not installed/enabled by default. Z3 is free for non-commercial applications and can be enabled -by setting the @{text OLD_Z3_NON_COMMERCIAL} environment variable to -@{text yes}. +by setting the \OLD_Z3_NON_COMMERCIAL\ environment variable to +\yes\. \ declare [[ old_smt_solver = z3 ]] @@ -242,7 +242,7 @@ subsection \Certificates\ text \ -By setting the option @{text old_smt_certificates} to the name of a file, +By setting the option \old_smt_certificates\ to the name of a file, all following applications of an SMT solver a cached in that file. Any further application of the same SMT solver (using the very same configuration) re-uses the cached certificate instead of invoking the @@ -250,7 +250,7 @@ The filename should be given as an explicit path. It is good practice to use the name of the current theory (with ending -@{text ".certs"} instead of @{text ".thy"}) as the certificates file. +\.certs\ instead of \.thy\) as the certificates file. Certificate files should be used at most once in a certain theory context, to avoid race conditions with other concurrent accesses. \ @@ -258,11 +258,11 @@ declare [[ old_smt_certificates = "" ]] text \ -The option @{text old_smt_read_only_certificates} controls whether only +The option \old_smt_read_only_certificates\ controls whether only stored certificates are should be used or invocation of an SMT solver -is allowed. When set to @{text true}, no SMT solver will ever be +is allowed. When set to \true\, no SMT solver will ever be invoked and only the existing certificates found in the configured -cache are used; when set to @{text false} and there is no cached +cache are used; when set to \false\ and there is no cached certificate for some proposition, then the configured SMT solver is invoked. \ @@ -275,7 +275,7 @@ text \ The SMT method, when applied, traces important information. To -make it entirely silent, set the following option to @{text false}. +make it entirely silent, set the following option to \false\. \ declare [[ old_smt_verbose = true ]] @@ -283,7 +283,7 @@ text \ For tracing the generated problem file given to the SMT solver as well as the returned result of the solver, the option -@{text old_smt_trace} should be set to @{text true}. +\old_smt_trace\ should be set to \true\. \ declare [[ old_smt_trace = false ]] @@ -292,7 +292,7 @@ From the set of assumptions given to the SMT solver, those assumptions used in the proof are traced when the following option is set to @{term true}. This only works for Z3 when it runs in non-oracle mode -(see options @{text old_smt_solver} and @{text old_smt_oracle} above). +(see options \old_smt_solver\ and \old_smt_oracle\ above). \ declare [[ old_smt_trace_used_facts = false ]] @@ -304,9 +304,9 @@ text \ Several prof rules of Z3 are not very well documented. There are two lemma groups which can turn failing Z3 proof reconstruction attempts -into succeeding ones: the facts in @{text z3_rule} are tried prior to +into succeeding ones: the facts in \z3_rule\ are tried prior to any implemented reconstruction procedure for all uncertain Z3 proof -rules; the facts in @{text z3_simp} are only fed to invocations of +rules; the facts in \z3_simp\ are only fed to invocations of the simplifier when reconstructing theory-specific proof steps. \