src/HOL/Rings.thy
changeset 55187 6d0d93316daf
parent 54703 499f92dc6e45
child 55912 e12a0ab9917c
--- a/src/HOL/Rings.thy	Thu Jan 30 17:34:42 2014 +0100
+++ b/src/HOL/Rings.thy	Thu Jan 30 16:09:03 2014 +0100
@@ -99,6 +99,14 @@
   "of_bool p = of_bool q \<longleftrightarrow> p = q"
   by (simp add: of_bool_def)
 
+lemma split_of_bool [split]:
+  "P (of_bool p) \<longleftrightarrow> (p \<longrightarrow> P 1) \<and> (\<not> p \<longrightarrow> P 0)"
+  by (cases p) simp_all
+
+lemma split_of_bool_asm:
+  "P (of_bool p) \<longleftrightarrow> \<not> (p \<and> \<not> P 1 \<or> \<not> p \<and> \<not> P 0)"
+  by (cases p) simp_all
+  
 end  
 
 class semiring_1 = zero_neq_one + semiring_0 + monoid_mult