src/HOL/Finite_Set.thy
changeset 22451 989182f660e0
parent 22425 c252770ae2d0
child 22473 753123c89d72
equal deleted inserted replaced
22450:51ee032f9591 22451:989182f660e0
  1977   empty_fold1SetE [rule del]  insert_fold1SetE [rule del]
  1977   empty_fold1SetE [rule del]  insert_fold1SetE [rule del]
  1978   -- {* No more proofs involve these relations. *}
  1978   -- {* No more proofs involve these relations. *}
  1979 
  1979 
  1980 subsubsection{* Semi-Lattices *}
  1980 subsubsection{* Semi-Lattices *}
  1981 
  1981 
       
  1982 (*FIXME integrate with Orderings.thy/OrderedGroup.thy*)
  1982 locale ACIfSL = ACIf +
  1983 locale ACIfSL = ACIf +
  1983   fixes below :: "'a \<Rightarrow> 'a \<Rightarrow> bool" (infixl "\<sqsubseteq>" 50)
  1984   fixes below :: "'a \<Rightarrow> 'a \<Rightarrow> bool" (infixl "\<sqsubseteq>" 50)
  1984   and strict_below :: "'a \<Rightarrow> 'a \<Rightarrow> bool" (infixl "\<sqsubset>" 50)
  1985   and strict_below :: "'a \<Rightarrow> 'a \<Rightarrow> bool" (infixl "\<sqsubset>" 50)
  1985   assumes below_def: "(x \<sqsubseteq> y) = (x\<cdot>y = x)"
  1986   assumes below_def: "(x \<sqsubseteq> y) = (x\<cdot>y = x)"
  1986   defines strict_below_def:  "(x \<sqsubset> y) \<equiv> (x \<sqsubseteq> y \<and> x \<noteq> y)"
  1987   defines strict_below_def:  "(x \<sqsubset> y) \<equiv> (x \<sqsubseteq> y \<and> x \<noteq> y)"
  2165 
  2166 
  2166 
  2167 
  2167 
  2168 
  2168 subsubsection{* Lattices *}
  2169 subsubsection{* Lattices *}
  2169 
  2170 
       
  2171 (*FIXME integrate with FixedPoint.thy*)
  2170 locale Lattice = lattice +
  2172 locale Lattice = lattice +
  2171   fixes Inf :: "'a set \<Rightarrow> 'a" ("\<Sqinter>_" [900] 900)
  2173   fixes Inf :: "'a set \<Rightarrow> 'a" ("\<Sqinter>_" [900] 900)
  2172   and Sup :: "'a set \<Rightarrow> 'a" ("\<Squnion>_" [900] 900)
  2174   and Sup :: "'a set \<Rightarrow> 'a" ("\<Squnion>_" [900] 900)
  2173   defines "Inf == fold1 inf"  and "Sup == fold1 sup"
  2175   defines "Inf == fold1 inf"  and "Sup == fold1 sup"
  2174 
  2176