# HG changeset patch # User paulson # Date 977310866 -3600 # Node ID 0c8d583326587f066ec0f7d5a4851a15e77c0507 # Parent 7a29b71d635265983c556615500da48738428f44 tidying, removing obsolete lemmas about 0=... and 1=... diff -r 7a29b71d6352 -r 0c8d58332658 src/HOL/Integ/nat_bin.ML --- a/src/HOL/Integ/nat_bin.ML Wed Dec 20 12:13:59 2000 +0100 +++ b/src/HOL/Integ/nat_bin.ML Wed Dec 20 12:14:26 2000 +0100 @@ -309,8 +309,7 @@ AddIffs (map rename_numerals [Suc_not_Zero, Zero_not_Suc, zero_less_Suc, not_less0, less_one, - le0, le_0_eq, - neq0_conv, zero_neq_conv, not_gr0]); + le0, le_0_eq, neq0_conv, not_gr0]); (** Arith **) @@ -323,12 +322,12 @@ (*Non-trivial simplifications*) val other_renamed_arith_simps = map rename_numerals - [diff_is_0_eq, zero_is_diff_eq, zero_less_diff, - mult_is_0, zero_is_mult, zero_less_mult_iff, mult_eq_1_iff]; + [diff_is_0_eq, zero_less_diff, + mult_is_0, zero_less_mult_iff, mult_eq_1_iff]; Addsimps (basic_renamed_arith_simps @ other_renamed_arith_simps); -AddIffs (map rename_numerals [add_is_0, zero_is_add, add_gr_0]); +AddIffs (map rename_numerals [add_is_0, add_gr_0]); Goal "Suc n = n + #1"; by (asm_simp_tac numeral_ss 1); @@ -359,7 +358,6 @@ (*various theorems that aren't in the default simpset*) bind_thm ("add_is_one'", rename_numerals add_is_1); -bind_thm ("one_is_add'", rename_numerals one_is_add); bind_thm ("zero_induct'", rename_numerals zero_induct); bind_thm ("diff_self_eq_0'", rename_numerals diff_self_eq_0); bind_thm ("mult_eq_self_implies_10'", rename_numerals mult_eq_self_implies_10); diff -r 7a29b71d6352 -r 0c8d58332658 src/HOL/Nat.ML --- a/src/HOL/Nat.ML Wed Dec 20 12:13:59 2000 +0100 +++ b/src/HOL/Nat.ML Wed Dec 20 12:14:26 2000 +0100 @@ -43,12 +43,6 @@ qed "neq0_conv"; AddIffs [neq0_conv]; -Goal "!!n::nat. (0 ~= n) = (0 < n)"; -by (case_tac "n" 1); -by Auto_tac; -qed "zero_neq_conv"; -AddIffs [zero_neq_conv]; - (*This theorem is useful with blast_tac: (n=0 ==> False) ==> 0