src/HOL/HOL.thy
changeset 67719 bffb7482faaa
parent 67673 c8caefb20564
child 68072 493b818e8e10
equal deleted inserted replaced
67717:5a1b299fe4af 67719:bffb7482faaa
  1402   by auto
  1402   by auto
  1403 
  1403 
  1404 lemma ex_if_distrib: "(\<exists>x. if x = a then P x else Q x) \<longleftrightarrow> P a \<or> (\<exists>x. x\<noteq>a \<and> Q x)"
  1404 lemma ex_if_distrib: "(\<exists>x. if x = a then P x else Q x) \<longleftrightarrow> P a \<or> (\<exists>x. x\<noteq>a \<and> Q x)"
  1405   by auto
  1405   by auto
  1406 
  1406 
       
  1407 lemma if_if_eq_conj: "(if P then if Q then x else y else y) = (if P \<and> Q then x else y)"
       
  1408   by simp
       
  1409 
  1407 text \<open>As a simplification rule, it replaces all function equalities by
  1410 text \<open>As a simplification rule, it replaces all function equalities by
  1408   first-order equalities.\<close>
  1411   first-order equalities.\<close>
  1409 lemma fun_eq_iff: "f = g \<longleftrightarrow> (\<forall>x. f x = g x)"
  1412 lemma fun_eq_iff: "f = g \<longleftrightarrow> (\<forall>x. f x = g x)"
  1410   by auto
  1413   by auto
  1411 
  1414