src/HOL/HOL.thy
changeset 34873 c6449a41b214
parent 34305 25ff5e139a1d
child 34886 873c31d9f10d
equal deleted inserted replaced
34872:6ca970cfa873 34873:c6449a41b214
  1814 code_datatype "prop" Trueprop
  1814 code_datatype "prop" Trueprop
  1815 
  1815 
  1816 text {* Code equations *}
  1816 text {* Code equations *}
  1817 
  1817 
  1818 lemma [code]:
  1818 lemma [code]:
  1819   shows "(False \<Longrightarrow> P) \<equiv> Trueprop True" 
  1819   shows "(True \<Longrightarrow> PROP Q) \<equiv> PROP Q" 
  1820     and "(True \<Longrightarrow> PROP Q) \<equiv> PROP Q" 
  1820     and "(PROP Q \<Longrightarrow> True) \<equiv> Trueprop True"
  1821     and "(P \<Longrightarrow> False) \<equiv> Trueprop (\<not> P)"
  1821     and "(P \<Longrightarrow> R) \<equiv> Trueprop (P \<longrightarrow> R)" by (auto intro!: equal_intr_rule)
  1822     and "(PROP Q \<Longrightarrow> True) \<equiv> Trueprop True" by (auto intro!: equal_intr_rule)
       
  1823 
  1822 
  1824 lemma [code]:
  1823 lemma [code]:
  1825   shows "False \<and> P \<longleftrightarrow> False"
  1824   shows "False \<and> P \<longleftrightarrow> False"
  1826     and "True \<and> P \<longleftrightarrow> P"
  1825     and "True \<and> P \<longleftrightarrow> P"
  1827     and "P \<and> False \<longleftrightarrow> False"
  1826     and "P \<and> False \<longleftrightarrow> False"