src/HOLCF/IOA/meta_theory/Sequence.thy
changeset 23778 18f426a137a9
parent 19741 f65265d71426
child 25131 2c8caac48ade
--- a/src/HOLCF/IOA/meta_theory/Sequence.thy	Wed Jul 11 11:54:03 2007 +0200
+++ b/src/HOLCF/IOA/meta_theory/Sequence.thy	Wed Jul 11 11:54:21 2007 +0200
@@ -355,7 +355,7 @@
 
 lemma Seq_Finite_ind:
 "!! P.[| Finite x; P nil; !! a s. [| Finite s; P s|] ==> P (a>>s) |] ==> P x"
-apply (erule (1) sfinite.induct)
+apply (erule (1) Finite.induct)
 apply (tactic {* def_tac 1 *})
 apply (simp add: Consq_def)
 done