src/HOL/Fun.thy
changeset 36176 3fe7e97ccca8
parent 35584 768f8d92b767
child 37751 89e16802b6cc
--- a/src/HOL/Fun.thy	Fri Apr 16 20:56:40 2010 +0200
+++ b/src/HOL/Fun.thy	Fri Apr 16 21:28:09 2010 +0200
@@ -525,7 +525,7 @@
 lemma bij_swap_iff: "bij (swap a b f) = bij f"
 by (simp add: bij_def)
 
-hide (open) const swap
+hide_const (open) swap
 
 
 subsection {* Inversion of injective functions *}