diff -r b49329185b82 -r dc6769b86fd6 src/HOL/Sledgehammer.thy --- 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 \Tools/Sledgehammer/sledgehammer_commands.ML\ ML_file \Tools/Sledgehammer/sledgehammer_tactics.ML\ +(* +lemma "1 + 1 = 2 \ 0 + (x::nat) = x" + sledgehammer +*) + +(* +declare nat_induct[no_atp] +declare nat_induct_non_zero[no_atp] + +lemma "P 0 \ (\n. P n \ P (Suc n)) \ P n" + sledgehammer [cvc4] (add: nat.induct) +*) + +(* +lemma "1 + 1 = 2 \ 0 + (x::nat) = x" + sledgehammer [verbose, e, dont_preplay, max_facts = 2] (add_0_left one_add_one) +*) + end