removed test failing on some platform
authordesharna
Tue, 10 Oct 2023 11:20:57 +0200
changeset 78745 f9c559d33ff3
parent 78744 a11c461a1a3a
child 78746 a748a244a028
removed test failing on some platform
src/HOL/Metis_Examples/Sledgehammer_Isar_Proofs.thy
--- a/src/HOL/Metis_Examples/Sledgehammer_Isar_Proofs.thy	Mon Oct 09 21:41:26 2023 +0200
+++ b/src/HOL/Metis_Examples/Sledgehammer_Isar_Proofs.thy	Tue Oct 10 11:20:57 2023 +0200
@@ -13,26 +13,4 @@
 
 sledgehammer_params [verit, isar_proof, minimize = false, slices = 1, compress = 1]
 
-lemma
-  fixes a b c :: int
-  shows "a + b = c \<Longrightarrow> c - b = a"
-  sledgehammer [expect = some_preplayed] ()
-proof -
-  assume a1: "a + b = c"
-  have "c - b \<le> a \<or> c \<noteq> a + b"
-    by force
-  then have f2: "c - b \<le> a"
-    using a1 by force
-  have "a \<le> c - b \<or> c \<noteq> a + b"
-    by force
-  then have "a \<le> c - b"
-    using a1 by force
-  then have f3: "c - b \<le> a \<and> a \<le> c - b"
-    using f2 by fastforce
-  have "c - b = a \<or> \<not> c - b \<le> a \<or> \<not> a \<le> c - b"
-    by auto
-  then show ?thesis
-    using f3 by meson
-qed
-
 end