src/HOL/Statespace/distinct_tree_prover.ML
changeset 51717 9e7d1c139569
parent 51701 1e29891759c4
child 55972 51b342baecda
--- a/src/HOL/Statespace/distinct_tree_prover.ML	Tue Apr 16 17:54:14 2013 +0200
+++ b/src/HOL/Statespace/distinct_tree_prover.ML	Thu Apr 18 17:07:01 2013 +0200
@@ -356,16 +356,15 @@
     | _ => no_tac))
 
 fun distinctFieldSolver names =
-  mk_solver "distinctFieldSolver" (distinctTree_tac names o Simplifier.the_context);
+  mk_solver "distinctFieldSolver" (distinctTree_tac names);
 
 fun distinct_simproc names =
   Simplifier.simproc_global @{theory HOL} "DistinctTreeProver.distinct_simproc" ["x = y"]
-    (fn thy => fn ss => fn (Const (@{const_name HOL.eq}, _) $ x $ y) =>
-      (case try Simplifier.the_context ss of
-        SOME ctxt =>
+    (fn ctxt =>
+      (fn Const (@{const_name HOL.eq}, _) $ x $ y =>
           Option.map (fn neq => @{thm neq_to_eq_False} OF [neq])
             (get_fst_success (neq_x_y ctxt x y) names)
-      | NONE => NONE));
+        | _ => NONE));
 
 end;