diff -r c4f2cac288d2 -r 4005298550a6 src/HOL/Hilbert_Choice.thy --- a/src/HOL/Hilbert_Choice.thy Tue Apr 09 21:05:48 2019 +0100 +++ b/src/HOL/Hilbert_Choice.thy Wed Apr 10 13:34:55 2019 +0100 @@ -43,6 +43,11 @@ subsection \Hilbert's Epsilon-operator\ +lemma Eps_cong: + assumes "\x. P x = Q x" + shows "Eps P = Eps Q" + using ext[of P Q, OF assms] by simp + text \ Easier to apply than \someI\ if the witness comes from an existential formula.