added inv_def for compatibility as a lemma
authornipkow
Tue, 20 Oct 2009 13:20:42 +0200
changeset 33014 85d7a096e63f
parent 33013 5c29cc66a029
child 33015 575bd6548df9
added inv_def for compatibility as a lemma
src/HOL/Hilbert_Choice.thy
--- a/src/HOL/Hilbert_Choice.thy	Tue Oct 20 11:36:19 2009 +0200
+++ b/src/HOL/Hilbert_Choice.thy	Tue Oct 20 13:20:42 2009 +0200
@@ -91,6 +91,9 @@
 
 subsection {*Function Inverse*}
 
+lemma inv_def: "inv f = (%y. SOME x. f x = y)"
+by(simp add: inv_onto_def)
+
 lemma inv_onto_into: "x : f ` A ==> inv_onto A f x : A"
 apply (simp add: inv_onto_def)
 apply (fast intro: someI2)