src/HOL/Predicate.thy
changeset 34007 aea892559fc5
parent 33988 901001414358
child 34065 6f8f9835e219
equal deleted inserted replaced
33996:e4fb0daadcff 34007:aea892559fc5
   724      | Insert x P \<Rightarrow> Insert x (P \<squnion> Seq g)
   724      | Insert x P \<Rightarrow> Insert x (P \<squnion> Seq g)
   725      | Join P xq \<Rightarrow> adjunct (Seq g) (Join P xq))"
   725      | Join P xq \<Rightarrow> adjunct (Seq g) (Join P xq))"
   726 proof (cases "f ()")
   726 proof (cases "f ()")
   727   case Empty
   727   case Empty
   728   thus ?thesis
   728   thus ?thesis
   729     unfolding Seq_def by (simp add: sup_commute [of "\<bottom>"]  sup_bot)
   729     unfolding Seq_def by (simp add: sup_commute [of "\<bottom>"])
   730 next
   730 next
   731   case Insert
   731   case Insert
   732   thus ?thesis
   732   thus ?thesis
   733     unfolding Seq_def by (simp add: sup_assoc)
   733     unfolding Seq_def by (simp add: sup_assoc)
   734 next
   734 next