Theory Errorable
chapter ‹Preliminaries›
section ‹Errorable›
theory Errorable
imports Main
begin
notation bot (‹⊥›)
typedef 'a errorable (‹_⇩⊥› [21] 21) = "UNIV :: 'a option set" ..
definition errorable :: "'a ⇒ 'a errorable" (‹_⇩⊥› [1000] 1000) where
"errorable x = Abs_errorable (Some x)"
instantiation errorable :: (type) bot
begin
definition "⊥ ≡ Abs_errorable None"
instance ..
end
free_constructors case_errorable for
errorable
| "⊥ :: 'a errorable"
unfolding errorable_def bot_errorable_def
apply (metis Abs_errorable_cases not_None_eq)
apply (metis Abs_errorable_inverse UNIV_I option.inject)
by (simp add: Abs_errorable_inject)
copy_bnf 'a errorable
end