src/HOL/Probability/ex/Dining_Cryptographers.thy
changeset 57492 74bf65a1910a
parent 56994 8d5e5ec1cac3
child 60585 48fdff264eb2
--- a/src/HOL/Probability/ex/Dining_Cryptographers.thy	Wed Jul 02 17:34:45 2014 +0200
+++ b/src/HOL/Probability/ex/Dining_Cryptographers.thy	Wed Jun 11 14:24:23 2014 +1000
@@ -239,7 +239,7 @@
   ultimately
   have "{dc \<in> dc_crypto. payer dc = Some i \<and> inversion dc = xs} =
     {(Some i, zs), (Some i, map Not zs)}"
-    using `i < n`
+    using `i < n` [[ hypsubst_thin = true ]]
   proof (safe, simp_all add:dc_crypto payer_def)
     fix b assume [simp]: "length b = n"
       and *: "inversion (Some i, b) = xs" and "b \<noteq> zs"