Apply scripts are a style of doing proofs in the theorem prover Isabelle; an alternative is structured Isar proofs.
Questions tagged [apply-script]
3 questions
1
vote
1 answer
Isabelle: Use of the "induct" or "induct_tac" methods
Let's say I have a lemma about a simple inductively-defined set:
inductive_set foo :: "'a ⇒ 'a list set" for x :: 'a where
"[] ∈ foo x" | "[x] ∈ foo x"
lemma "⋀x y. y ∈ foo x ⟹ qux x y ⟹ baz x y"
(It's important to me that the "⋀x y" bit stays,…

John Wickerson
- 1,204
- 12
- 23
1
vote
1 answer
Canonical way to get a more specific lemma
Say I have a lemma mylem: foo ?a = bar ?a, and I need to apply it on a goal that has two occurrences of foo, e.g. baz (foo (f p q)) (foo (g r s)), but only at one of these positions. I know of two ways of doing that without having to write out all…

Joachim Breitner
- 25,395
- 6
- 78
- 139
0
votes
2 answers
Isabelle: Opposite of "intro impI"
If my goal state is foo ==> bar --> qux, I know that I can use the statement
apply (intro impI)
to yield the goal state foo ==> bar ==> qux. What about the other direction? Which command will send me back to the goal state foo ==> bar --> qux?…

John Wickerson
- 1,204
- 12
- 23