removed an unfortunate sledgehammer command
authorpaulson <lp15@cam.ac.uk>
Sun, 01 Jan 2023 12:24:00 +0000
changeset 76838 04c7ec38874e
parent 76837 d908a7d3ed1b
child 76857 3bd08d0432d7
child 76874 d6b02d54dbf8
removed an unfortunate sledgehammer command
src/HOL/Analysis/Function_Topology.thy
--- a/src/HOL/Analysis/Function_Topology.thy	Sun Jan 01 01:43:02 2023 +0000
+++ b/src/HOL/Analysis/Function_Topology.thy	Sun Jan 01 12:24:00 2023 +0000
@@ -335,11 +335,8 @@
   "openin (product_topology X I) S \<longleftrightarrow>
     (\<forall>x \<in> S. \<exists>U. finite {i \<in> I. U i \<noteq> topspace(X i)} \<and>
                  (\<forall>i \<in> I. openin (X i) (U i)) \<and> x \<in> Pi\<^sub>E I U \<and> Pi\<^sub>E I U \<subseteq> S)"
-sledgehammer [isar_proofs, provers = "cvc4 z3 spass e vampire verit", timeout = 77]
   unfolding openin_product_topology arbitrary_union_of_alt product_topology_base_alt topspace_product_topology
-  apply safe
-  apply (drule bspec; blast)+
-  done
+  by (smt (verit, best))
 
 lemma closure_of_product_topology:
   "(product_topology X I) closure_of (PiE I S) = PiE I (\<lambda>i. (X i) closure_of (S i))"