Hi all,
I (or more precisely @Hanna Lachnitt ) is automatically generating theorems like the one below:
lemma H:
fixes t s :: int
shows "(s ≤ t) = ((0::int) ≤ t - s)"
by auto
Is there any way to make sure that the order given by the fixes is respected? (I also tried ⋀
, with the same result)
thm H[of t] (*how should t instantiate t here?*)
As we do ML instantiation I would prefer avoiding the H[where t=t]
version.
In the document, there is an attribute named params
, for which I suspect could be useful. However, I have neither used it myself nor have I observed its usage within the standard library or AFP... I believe some Isabelle/ML hacks could solve the task, though I am not sure how to do it off the top of my head.
which document do you mean?
https://isabelle.in.tum.de/library/Doc/Isar_Ref/Proof.html?
Last updated: Dec 21 2024 at 12:33 UTC