changeset 66795 | 420d0080545f |
parent 64272 | f76b6dda2e56 |
child 66817 | 0b12755ccbb2 |
--- a/src/HOL/Nat_Transfer.thy Mon Oct 09 16:14:18 2017 +0100 +++ b/src/HOL/Nat_Transfer.thy Sun Oct 08 22:28:19 2017 +0200 @@ -285,7 +285,7 @@ "(int x) * (int y) = int (x * y)" "tsub (int x) (int y) = int (x - y)" "(int x)^n = int (x^n)" - by (auto simp add: of_nat_mult tsub_def of_nat_power) + by (auto simp add: tsub_def) lemma transfer_int_nat_function_closures: "is_nat x \<Longrightarrow> is_nat y \<Longrightarrow> is_nat (x + y)"