Skip to content

Instantly share code, notes, and snippets.

@Kuniwak
Created July 15, 2022 01:01
Show Gist options
  • Star 0 You must be signed in to star a gist
  • Fork 0 You must be signed in to fork a gist
  • Save Kuniwak/3034c2d5762cb93f0b92ec5fedb45df4 to your computer and use it in GitHub Desktop.
Save Kuniwak/3034c2d5762cb93f0b92ec5fedb45df4 to your computer and use it in GitHub Desktop.
theory "Well_Not_Dense_Order" imports Main begin
context wellorder
begin
definition bot :: 'a
where "bot ≡ LEAST x. True"
sublocale order_bot bot less_eq less
proof standard
fix a
show "bot ≤ a"
unfolding bot_def by (simp add: local.Least_le)
qed
lemma no_dense:
fixes a :: 'a
assumes "a ≠ bot"
and "⋀a b. ⟦⋀x. ⟦a ≤ x; x ≤ b⟧ ⟹ thesis; a ≠ b⟧ ⟹ thesis"
shows "thesis"
using assms le_bot by metis
end
end
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment