# HG changeset patch # User nipkow # Date 1213363327 -7200 # Node ID e47b069cab351d5d21968f1d8b0f62de42b118d0 # Parent 17b63e145986879e323fcc0c782f3a98ba8ece85 hide -> hide (open) diff -r 17b63e145986 -r e47b069cab35 src/HOL/Fun.thy --- a/src/HOL/Fun.thy Thu Jun 12 23:12:54 2008 +0200 +++ b/src/HOL/Fun.thy Fri Jun 13 15:22:07 2008 +0200 @@ -482,7 +482,7 @@ lemma bij_swap_iff: "bij (swap a b f) = bij f" by (simp add: bij_def) -hide const swap +hide (open) const swap subsection {* Proof tool setup *}