--- a/src/HOL/Library/Finite_Lattice.thy Mon Apr 10 23:21:47 2023 +0200
+++ b/src/HOL/Library/Finite_Lattice.thy Tue Apr 11 11:59:02 2023 +0000
@@ -2,10 +2,14 @@
Author: Alessandro Coglio
*)
+section \<open>Finite Lattices\<close>
+
theory Finite_Lattice
imports Product_Order
begin
+subsection \<open>Finite Complete Lattices\<close>
+
text \<open>A non-empty finite lattice is a complete lattice.
Since types are never empty in Isabelle/HOL,
a type of classes \<^class>\<open>finite\<close> and \<^class>\<open>lattice\<close>