src/HOL/Library/Finite_Lattice.thy
changeset 51115 7dbd6832a689
parent 50634 009a9fdabbad
child 51489 f738e6dbd844
equal deleted inserted replaced
51114:3e913a575dc6 51115:7dbd6832a689
     1 (* Author: Alessandro Coglio *)
     1 (* Author: Alessandro Coglio *)
     2 
     2 
     3 theory Finite_Lattice
     3 theory Finite_Lattice
     4 imports Product_Lattice
     4 imports Product_Order
     5 begin
     5 begin
     6 
     6 
     7 text {* A non-empty finite lattice is a complete lattice.
     7 text {* A non-empty finite lattice is a complete lattice.
     8 Since types are never empty in Isabelle/HOL,
     8 Since types are never empty in Isabelle/HOL,
     9 a type of classes @{class finite} and @{class lattice}
     9 a type of classes @{class finite} and @{class lattice}