ex/{bin.ML,comb.ML,prop.ML}: replaced NewSext by Syntax.simple_sext
domrange/image_subset,vimage_subset: deleted needless premise!
misc: This slightly simplifies two proofs in Schroeder-Bernstein Theorem
ind-syntax/rule_concl: recoded to avoid exceptions
intr-elim: now checks conclusions of introduction rules
func/fun_disjoint_Un: now uses ex_ex1I
list-fn/hd,tl,drop: new
simpdata/bquant_simps: new
list/list_case_type: restored!
bool.thy: changed 1 from a "def" to a translation
Removed occurreces of one_def in bool.ML, nat.ML, univ.ML, ex/integ.ML
nat/succ_less_induct: new induction principle
arith/add_mono: new results about monotonicity
simpdata/mem_simps: removed the ones for succ and cons; added succI1,
consI2 to ZF_ss
upair/succ_iff: new, for use with simp_tac (cons_iff already existed)
ordinal/Ord_0_in_succ: renamed from Ord_0_mem_succ
nat/nat_0_in_succ: new
ex/prop-log/hyps_thms_if: split up the fast_tac call for more speed
#! /bin/sh
# simp FILE1 ... FILEn
#
# leaves previous versions as XXX~~
#
for f in $*
do
echo $f. \ Backup file is $f~~
mv $f $f~~; sed -e '
s/\<ASM_SIMP_TAC\>/asm_simp_tac/g
s/\<SIMP_TAC\>/simp_tac/g
s/\<addrews\>/addsimps/g
s/addsplits \(\[[^]]*\]\)/setloop (split_tac \1)/g
s/addsplits/setloop split_tac/g
s/\<setauto\>/setsolver/g
' $f~~ > $f
done
echo Finished.