# HG changeset patch # User nipkow # Date 1494758792 -7200 # Node ID 416aa3b00cbea0f179bc6ffec03b60f4c5865e75 # Parent bdd17b18e10356f7078ff1b1946d06995597bf85 added lemma diff -r bdd17b18e103 -r 416aa3b00cbe src/HOL/Hilbert_Choice.thy --- a/src/HOL/Hilbert_Choice.thy Fri May 12 20:03:50 2017 +0200 +++ b/src/HOL/Hilbert_Choice.thy Sun May 14 12:46:32 2017 +0200 @@ -30,11 +30,14 @@ in Syntax.const @{syntax_const "_Eps"} $ x $ t end)] \ \ \to avoid eta-contraction of body\ -definition inv_into :: "'a set \ ('a \ 'b) \ ('b \ 'a)" - where "inv_into A f \ \x. SOME y. y \ A \ f y = x" +definition inv_into :: "'a set \ ('a \ 'b) \ ('b \ 'a)" where +"inv_into A f = (\x. SOME y. y \ A \ f y = x)" -abbreviation inv :: "('a \ 'b) \ ('b \ 'a)" - where "inv \ inv_into UNIV" +lemma inv_into_def2: "inv_into A f x = (SOME y. y \ A \ f y = x)" +by(simp add: inv_into_def) + +abbreviation inv :: "('a \ 'b) \ ('b \ 'a)" where +"inv \ inv_into UNIV" subsection \Hilbert's Epsilon-operator\