src/HOL/Hilbert_Choice.thy
changeset 74123 7c5842b06114
parent 73623 5020054b3a16
child 75607 3c544d64c218
--- a/src/HOL/Hilbert_Choice.thy	Thu Aug 05 07:12:49 2021 +0000
+++ b/src/HOL/Hilbert_Choice.thy	Thu Aug 05 07:12:49 2021 +0000
@@ -1170,18 +1170,6 @@
 
 end
 
-context complete_boolean_algebra
-begin
-
-lemma dual_complete_boolean_algebra:
-  "class.complete_boolean_algebra Sup Inf sup (\<ge>) (>) inf \<top> \<bottom> (\<lambda>x y. x \<squnion> - y) uminus"
-  by (rule class.complete_boolean_algebra.intro,
-      rule dual_complete_distrib_lattice,
-      rule dual_boolean_algebra)
-end
-
-
-
 instantiation set :: (type) complete_distrib_lattice
 begin
 instance proof (standard, clarsimp)