| changeset 44277 | bcb696533579 |
| parent 44121 | 44adaa6db327 |
| child 44921 | 58eef4843641 |
--- a/src/HOL/HOL.thy Thu Aug 18 13:10:24 2011 +0200 +++ b/src/HOL/HOL.thy Thu Aug 18 13:25:17 2011 +0200 @@ -1394,6 +1394,11 @@ "f (if c then x else y) = (if c then f x else f y)" by simp +text{*As a simplification rule, it replaces all function equalities by + first-order equalities.*} +lemma fun_eq_iff: "f = g \<longleftrightarrow> (\<forall>x. f x = g x)" + by auto + subsubsection {* Generic cases and induction *}