src/HOL/Inductive.thy
changeset 11439 9aaab1a160a5
parent 11436 3f74b80d979f
child 11688 56833637db2a
--- a/src/HOL/Inductive.thy	Sun Jul 22 21:30:05 2001 +0200
+++ b/src/HOL/Inductive.thy	Sun Jul 22 21:30:21 2001 +0200
@@ -68,7 +68,7 @@
   hence "(THE x'. f x' = f x) = (THE x'. x' = x)"
     by (simp only: inj_eq)
   also have "... = x" by (rule the_eq_trivial)
-  finally (trans) show ?thesis by (unfold myinv_def)
+  finally show ?thesis by (unfold myinv_def)
 qed
 
 lemma f_myinv_f: "inj f ==> y \<in> range f ==> f (myinv f y) = y"