changeset 4613 | 67a726003cf8 |
parent 4104 | 84433b1ab826 |
child 4640 | ac6cf9f18653 |
--- a/src/HOL/Nat.thy Mon Feb 09 14:40:59 1998 +0100 +++ b/src/HOL/Nat.thy Mon Feb 09 18:09:35 1998 +0100 @@ -16,8 +16,8 @@ ("nat", {case_const = Bound 0, case_rewrites = [], constructors = [], induct_tac = nat_ind_tac, exhaustion = natE, - exhaust_tac = fn v => ALLNEWSUBGOALS (res_inst_tac [("n",v)] natE) - (rotate_tac ~1), + exhaust_tac = fn v => (res_inst_tac [("n",v)] natE) + THEN_ALL_NEW (rotate_tac ~1), nchotomy = ProtoPure.flexpair_def, case_cong = ProtoPure.flexpair_def}) |}