src/HOL/Integ/NatBin.ML
changeset 7127 48e235179ffb
parent 7086 f9aa63a5a8b6
child 7519 8e4a21d1ba4f
--- a/src/HOL/Integ/NatBin.ML	Wed Jul 28 22:01:58 1999 +0200
+++ b/src/HOL/Integ/NatBin.ML	Thu Jul 29 12:44:57 1999 +0200
@@ -146,7 +146,7 @@
 Goal "(#0::int) <= z ==> nat z div nat z' = nat (z div z')";
 by (case_tac "#0 <= z'" 1);
 by (auto_tac (claset(), 
-	      simpset() addsimps [div_nonneg_neg, DIVISION_BY_ZERO_DIV]));
+	      simpset() addsimps [div_nonneg_neg_le0, DIVISION_BY_ZERO_DIV]));
 by (zdiv_undefined_case_tac "z' = #0" 1);
  by (simp_tac (simpset() addsimps [numeral_0_eq_0, DIVISION_BY_ZERO_DIV]) 1);
 by (auto_tac (claset() addSEs [nonneg_eq_int], simpset()));