src/HOL/Sledgehammer.thy
changeset 75029 dc6769b86fd6
parent 73684 a63d76ba0a03
child 75030 919fb49ba201
--- a/src/HOL/Sledgehammer.thy	Mon Jan 31 16:09:23 2022 +0100
+++ b/src/HOL/Sledgehammer.thy	Mon Jan 31 16:09:23 2022 +0100
@@ -35,4 +35,22 @@
 ML_file \<open>Tools/Sledgehammer/sledgehammer_commands.ML\<close>
 ML_file \<open>Tools/Sledgehammer/sledgehammer_tactics.ML\<close>
 
+(*
+lemma "1 + 1 = 2 \<and> 0 + (x::nat) = x"
+  sledgehammer
+*)
+
+(*
+declare nat_induct[no_atp]
+declare nat_induct_non_zero[no_atp]
+
+lemma "P 0 \<Longrightarrow> (\<And>n. P n \<Longrightarrow> P (Suc n)) \<Longrightarrow> P n"
+  sledgehammer [cvc4] (add: nat.induct)
+*)
+
+(*
+lemma "1 + 1 = 2 \<and> 0 + (x::nat) = x"
+  sledgehammer [verbose, e, dont_preplay, max_facts = 2] (add_0_left one_add_one)
+*)
+
 end