src/HOL/ZF/Games.thy
changeset 19769 c40ce2de2020
parent 19203 778507520684
child 22282 71b4aefad227
--- a/src/HOL/ZF/Games.thy	Sun Jun 04 10:52:47 2006 +0200
+++ b/src/HOL/ZF/Games.thy	Mon Jun 05 14:22:58 2006 +0200
@@ -323,7 +323,7 @@
   have option_of: "option_of = inv_image is_option_of Rep_game"
     apply (rule set_ext)
     apply (case_tac "x")
-    by (simp add: inv_image_def option_to_is_option_of) 
+    by (simp add: option_to_is_option_of) 
   show ?thesis
     apply (simp add: option_of)
     apply (auto intro: wf_inv_image wf_is_option_of)