src/HOL/Predicate.thy
changeset 32582 a382876d3290
parent 32578 22117a76f943
child 32601 47d0c967c64e
equal deleted inserted replaced
32581:44ac2e398411 32582:a382876d3290
   872   top ("\<top>") and
   872   top ("\<top>") and
   873   bot ("\<bottom>") and
   873   bot ("\<bottom>") and
   874   bind (infixl "\<guillemotright>=" 70)
   874   bind (infixl "\<guillemotright>=" 70)
   875 
   875 
   876 hide (open) type pred seq
   876 hide (open) type pred seq
   877 hide (open) const Pred eval single bind if_pred not_pred
   877 hide (open) const Pred eval single bind is_empty singleton if_pred not_pred
   878   Empty Insert Join Seq member pred_of_seq "apply" adjunct eq map
   878   Empty Insert Join Seq member pred_of_seq "apply" adjunct null the_only eq map
   879 
   879 
   880 end
   880 end