Does anyone have a small example where the infamous ENTER MATCH
message is triggered?
From the mailing list:
theory SimpleStuff imports Main
begin
typedecl i
consts a::i b::i
axiomatization where
A1: "¬(a = b)" and
A2: "∀x::i. x = a ∨ x = b"
theorem T1: "∃(F::(i⇒bool)⇒i). ∀T::i. (∃(S::i⇒bool). F S = T)"
apply fastforce
Turns out that fastforce
just finds the proof when you prevent it from printing...
Last updated: Dec 21 2024 at 12:33 UTC