src/HOL/SMT.thy
changeset 50317 4d1590544b91
parent 48892 0b2407f406e8
child 55007 0c07990363a3
--- a/src/HOL/SMT.thy	Mon Dec 03 15:23:36 2012 +0100
+++ b/src/HOL/SMT.thy	Mon Dec 03 16:07:28 2012 +0100
@@ -256,6 +256,8 @@
 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.
+Certificate files should be used at most once in a certain theory context,
+to avoid race conditions with other concurrent accesses.
 *}
 
 declare [[ smt_certificates = "" ]]