From: Sven Schneider <sven.schneider.pub@gmx.de>
Hi all,
I have some old 2014 theory files that I might want to update to the
current version.
Apparently something has changed and I am unable to find anything in the
NEWS about it.
Is there a minimal workaround that requires minimal effort?
There are very many instances of this sort in the proofs...
Best regards
example
==========================
theory Test
imports
Main
begin
lemma TEST: "foo"
apply(subgoal_tac "?X")
==========================
output
=============
"Unbound schematic variable: ?X"
=============
From: Makarius <makarius@sketis.net>
The proper way to do it is via "eigen-context" like this:
apply (subgoal_tac "X" for X)
Unbound schematic variables violate the Isabelle/Isar context
discipline. The more tools are properly localized, the less they can
sneak into proof texts.
Here is also a relavant NEWS entry from Isabelle2015:
Makarius
Last updated: Nov 21 2024 at 12:39 UTC