Skip to content

Instantly share code, notes, and snippets.

@astahfrom
Created November 17, 2017 18:59
Show Gist options
  • Save astahfrom/d4b87d0bbac6d94742ecdfd8605369f7 to your computer and use it in GitHub Desktop.
Save astahfrom/d4b87d0bbac6d94742ecdfd8605369f7 to your computer and use it in GitHub Desktop.
Isabelle exception
theory THM0_741 imports Main begin
datatype 'a s = S 'a
datatype 'a t = T ‹'a s›
primrec f :: ‹'a s ⇒ 'a set› where
‹f (S x) = {x}›
primrec g :: ‹'a t ⇒ 'a set› where
‹g (T x) = f x›
lemma trigger: ‹f t ⊆ UNIV›
by blast
lemma ‹g p ⊆ UNIV›
using trigger (* raises: *)
proof (induct p)
case (T x) (* exception THM 0 raised (line 741 of "thm.ML"): assume: variables *)
then show ?case
by simp
qed
end
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment