{HOL,ZF}/indrule/ind_tac: now calls DEPTH_SOLVE_1 instead of REPEAT, to
solve the goal fully before proceeding
{HOL,ZF}/indrule/mutual_ind_tac: ensures that calls to "prem" cannot loop;
calls DEPTH_SOLVE_1 instead of REPEAT to solve the goal fully
{HOL,ZF}/intr_elim/intro_tacsf: now calls DEPTH_SOLVE_1 instead of REPEAT to
solve the goal fully
(* Title: HOL/Finite.thy
ID: $Id$
Author: Lawrence C Paulson, Cambridge University Computer Laboratory
Copyright 1994 University of Cambridge
Finite powerset operator
*)
Finite = Lfp +
consts Fin :: "'a set => 'a set set"
inductive "Fin(A)"
intrs
emptyI "{} : Fin(A)"
insertI "[| a: A; b: Fin(A) |] ==> insert(a,b) : Fin(A)"
end