object TacticCommands extends TacticCommands
- Alphabetic
- By Inheritance
- TacticCommands
- TacticCommands
- AnyRef
- Any
- Hide All
- Show All
- Public
- All
Value Members
-
final
def
!=(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
-
final
def
##(): Int
- Definition Classes
- AnyRef → Any
-
final
def
==(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
-
def
allL(terms: Expr*): ForallLeftTactic
Applies the
ForallLeft
tactic to the current subgoal: The goalApplies the
ForallLeft
tactic to the current subgoal: The goal∀x1,...,∀xn.A, Γ :- Δ
is reduced to
A[x1\t1,...,xn\tn], ∀x1,...,∀xn.A, Γ :- Δ.
This will only work if there is exactly one universal formula in the antecedent!
- terms
The terms
t1,...,tn
.
- Definition Classes
- TacticCommands
-
def
allL(applyToLabel: String, terms: Expr*): ForallLeftTactic
Applies the
ForallLeft
tactic to the current subgoal: The goalApplies the
ForallLeft
tactic to the current subgoal: The goal∀x1,...,∀xn.A, Γ :- Δ
is reduced to
A[x1\t1,...,xn\tn], ∀x1,...,∀xn.A, Γ :- Δ
.- applyToLabel
The label of the formula
∀x1,...,∀xn.A
.- terms
The terms
t1,...,tn
.
- Definition Classes
- TacticCommands
-
def
allR: ForallRightTactic
Applies the
ForallRight
tactic to the current subgoal: The goalApplies the
ForallRight
tactic to the current subgoal: The goalΓ :- Δ, ∀x.A
is reduced to
Γ :- Δ, A
.This will only work if there is exactly one universal formula in the succedent!
- Definition Classes
- TacticCommands
-
def
allR(applyToLabel: String): ForallRightTactic
Applies the
ForallRight
tactic to the current subgoal: The goalApplies the
ForallRight
tactic to the current subgoal: The goalΓ :- Δ, ∀x.A
is reduced to
Γ :- Δ, A
.- applyToLabel
The label of the formula
∀x.A
.
- Definition Classes
- TacticCommands
-
def
allR(eigenVariable: Var): ForallRightTactic
Applies the
ForallRight
tactic to the current subgoal: The goalApplies the
ForallRight
tactic to the current subgoal: The goalΓ :- Δ, ∀x.A
is reduced to
Γ :- Δ, A[x\α]
.This will only work if there is exactly one universal formula in the succedent!
- eigenVariable
The variable
α
.
- Definition Classes
- TacticCommands
-
def
allR(applyToLabel: String, eigenVariable: Var): ForallRightTactic
Applies the
ForallRight
tactic to the current subgoal: The goalApplies the
ForallRight
tactic to the current subgoal: The goalΓ :- Δ, ∀x.A
is reduced to
Γ :- Δ, A[x\α]
.- applyToLabel
The label of the formula
∀x.A
.- eigenVariable
The variable
α
.
- Definition Classes
- TacticCommands
-
def
analyticInduction(implicit ctx: MutableContext): AnalyticInductionTactic
- Definition Classes
- TacticCommands
-
def
andL: AndLeftTactic
Applies the
AndLeft
tactic to the current subgoal: The goalApplies the
AndLeft
tactic to the current subgoal: The goalA ∧ B, Γ :- Δ
is reduced to
A, B, Γ :- Δ
.This will only work if there is exactly one conjunctive formula in the antecedent!
- Definition Classes
- TacticCommands
-
def
andL(applyToLabel: String): AndLeftTactic
Applies the
AndLeft
tactic to the current subgoal: The goalApplies the
AndLeft
tactic to the current subgoal: The goalA ∧ B, Γ :- Δ
is reduced to
A, B, Γ :- Δ
.- applyToLabel
The label of the formula
A ∧ B
.
- Definition Classes
- TacticCommands
-
def
andR: AndRightTactic
Applies the
AndRight
tactic to the current subgoal: The goalApplies the
AndRight
tactic to the current subgoal: The goalΓ :- Δ, A ∧ B
is reduced to
Γ :- Δ, A
andΓ :- Δ, B
.This will only work if there is exactly one conjunctive formula in the succedent!
- Definition Classes
- TacticCommands
-
def
andR(applyToLabel: String): AndRightTactic
Applies the
AndRight
tactic to the current subgoal: The goalApplies the
AndRight
tactic to the current subgoal: The goalΓ :- Δ, A ∧ B
is reduced to
Γ :- Δ, A
andΓ :- Δ, B
.- applyToLabel
The label of the formula
A ∧ B
.
- Definition Classes
- TacticCommands
-
final
def
asInstanceOf[T0]: T0
- Definition Classes
- Any
-
def
axiomBot: BottomAxiomTactic.type
Applies the
BottomAxiom
tactic to the current subgoal: A subgoal of the form⊥, Γ :- Δ
will be closed.Applies the
BottomAxiom
tactic to the current subgoal: A subgoal of the form⊥, Γ :- Δ
will be closed.- Definition Classes
- TacticCommands
-
def
axiomLog: LogicalAxiomTactic.type
Applies the
LogicalAxiom
tactic to the current subgoal: A subgoal of the formA, Γ :- Δ, A
will be closed.Applies the
LogicalAxiom
tactic to the current subgoal: A subgoal of the formA, Γ :- Δ, A
will be closed.- Definition Classes
- TacticCommands
-
def
axiomRefl: ReflexivityAxiomTactic.type
Applies the
ReflexivityAxiom
tactic to the current subgoal: A subgoal of the formΓ :- Δ, s = s
will be closed.Applies the
ReflexivityAxiom
tactic to the current subgoal: A subgoal of the formΓ :- Δ, s = s
will be closed.- Definition Classes
- TacticCommands
-
def
axiomTop: TopAxiomTactic.type
Applies the
TopAxiom
tactic to the current subgoal: A subgoal of the formΓ :- Δ, ⊤
will be closed.Applies the
TopAxiom
tactic to the current subgoal: A subgoal of the formΓ :- Δ, ⊤
will be closed.- Definition Classes
- TacticCommands
-
def
chain(h: String): ChainTactic
- Definition Classes
- TacticCommands
-
def
clone(): AnyRef
- Attributes
- protected[java.lang]
- Definition Classes
- AnyRef
- Annotations
- @native() @throws( ... )
-
def
currentGoal: Tactic[OpenAssumption]
Retrieves the current subgoal.
Retrieves the current subgoal.
- Definition Classes
- TacticCommands
-
def
cut(label: String, cutFormula: Formula): CutTactic
Applies the
Cut
tactic to the current subgoal: The goalApplies the
Cut
tactic to the current subgoal: The goalΓ :- Δ
is reduced to
Γ :- Δ, C
andC, Γ :- Δ
.- label
The label of
C
.- cutFormula
The formula
C
.
- Definition Classes
- TacticCommands
-
def
decompose: Tactical[Unit]
Decomposes the current subgoal by applying all "simple" rules as often as possible.
Decomposes the current subgoal by applying all "simple" rules as often as possible. These rules are: -
¬:l
and¬:r
-∧:l
-∨:r
-⊃:r
-∀:r
-∃:l
- Definition Classes
- TacticCommands
-
def
destruct(label: String): Tactical[Any]
- Definition Classes
- TacticCommands
-
final
def
eq(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef
-
def
eql(eq: String, fm: String): EqualityTactic
Applies the
Equality
tactic to the current subgoal: Given an equations = t
and a formulaA
, some occurrences ofs
in A are replaced byt
or vice versa.Applies the
Equality
tactic to the current subgoal: Given an equations = t
and a formulaA
, some occurrences ofs
in A are replaced byt
or vice versa. The exact behavior can be controlled with additional commands:-
fromLeftToRight
: Occurrences ofs
will be replaced byt
. -fromRightToLeft
: Occurrences oft
will be replaced bys
. -yielding(f)
: The tactic will attempt to replace occurences in such a way that the end result isf
.If neither
fromLeftToRight
norfromRightToLeft
is used, the direction of replacement needs to be unambiguous, i.e.s
andt
may not both occur inA
.- eq
The label of
s = t
.- fm
The label of
A
.
- Definition Classes
- TacticCommands
-
def
equals(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
-
def
escargot(implicit ctx: MutableContext): ResolutionProverTactic
Calls
escargot
on the current subgoal.Calls
escargot
on the current subgoal.- Definition Classes
- TacticCommands
-
def
exL: ExistsLeftTactic
Applies the
ExistsLeft
tactic to the current subgoal: The goalApplies the
ExistsLeft
tactic to the current subgoal: The goal∃x.A, Γ :- Δ
is reduced to
A, Γ :- Δ
.This will only work if there is exactly one existential formula in the antecedent!
- Definition Classes
- TacticCommands
-
def
exL(applyToLabel: String): ExistsLeftTactic
Applies the
ExistsLeft
tactic to the current subgoal: The goalApplies the
ExistsLeft
tactic to the current subgoal: The goal∃x.A, Γ :- Δ
is reduced to
A, Γ :- Δ
.- applyToLabel
The label of the formula
∃x.A
.
- Definition Classes
- TacticCommands
-
def
exL(eigenVariable: Var): ExistsLeftTactic
Applies the
ExistsLeft
tactic to the current subgoal: The goalApplies the
ExistsLeft
tactic to the current subgoal: The goal∃x.A, Γ :- Δ
is reduced to
A[x\α], Γ :- Δ
.This will only work if there is exactly one existential formula in the antecedent!
- eigenVariable
The variable
α
.
- Definition Classes
- TacticCommands
-
def
exL(applyToLabel: String, eigenVariable: Var): ExistsLeftTactic
Applies the
ExistsLeft
tactic to the current subgoal: The goalApplies the
ExistsLeft
tactic to the current subgoal: The goal∃x.A, Γ :- Δ
is reduced to
A[x\α], Γ :- Δ
.- applyToLabel
The label of the formula
∃x.A
.- eigenVariable
The variable
α
.
- Definition Classes
- TacticCommands
-
def
exR(terms: Expr*): ExistsRightTactic
Applies the
ExistsRight
tactic to the current subgoal: The goalApplies the
ExistsRight
tactic to the current subgoal: The goalΓ :- Δ, ∃x1...∃xn.A
is reduced to
Γ :- Δ, ∃x1...∃xn.A, A[x1\t1,...,xn\tn]
.This will only work if there is exactly one existential formula in the succedent!
- terms
The terms
t1,...,tn
.
- Definition Classes
- TacticCommands
-
def
exR(applyToLabel: String, terms: Expr*): ExistsRightTactic
Applies the
ExistsRight
tactic to the current subgoal: The goalApplies the
ExistsRight
tactic to the current subgoal: The goalΓ :- Δ, ∃x1...∃xn.A
is reduced to
Γ :- Δ, ∃x1...∃xn.A, A[x1\t1,...,xn\tn]
.- applyToLabel
The label of the formula
∃x1...∃xn.A
.- terms
The terms
t1,...,tn
.
- Definition Classes
- TacticCommands
-
def
fail: Tactical[Nothing] { def apply(proofState: at.logic.gapt.proofs.gaptic.ProofState): scala.util.Left[at.logic.gapt.proofs.gaptic.TacticalFailure,Nothing] }
Tactic that immediately fails.
Tactic that immediately fails.
- Definition Classes
- TacticCommands
-
def
finalize(): Unit
- Attributes
- protected[java.lang]
- Definition Classes
- AnyRef
- Annotations
- @throws( classOf[java.lang.Throwable] )
-
def
foTheory(implicit ctx: Context): Tactical[Unit]
Solves the current subgoal as a first-order consequence of the background theory.
Solves the current subgoal as a first-order consequence of the background theory. This closes the goal.
- ctx
A at.logic.gapt.proofs.Context. The current subgoal must be contained in its background theory.
- Definition Classes
- TacticCommands
-
def
focus(indexOfSubGoal: OpenAssumptionIndex): FocusTactical
Moves the specified goal to the front of the goal list.
Moves the specified goal to the front of the goal list.
- indexOfSubGoal
The index of the goal.
- Definition Classes
- TacticCommands
-
def
focus(indexOfSubGoal: Int): FocusTactical
Moves the specified goal to the front of the goal list.
Moves the specified goal to the front of the goal list.
- indexOfSubGoal
The index of the goal.
- Definition Classes
- TacticCommands
-
def
forget(pred: (String, Formula) ⇒ Boolean): Tactical[Unit]
- Definition Classes
- TacticCommands
-
def
forget(ls: String*): Tactical[Unit]
Lets you "forget" a sequence of formulas, i.e.
Lets you "forget" a sequence of formulas, i.e. the tactics version of the weakening rule. The formulas with labels
L1,...,Ln
will be removed from the current goal.- ls
The labels
L1
,...,Ln
.
- Definition Classes
- TacticCommands
-
final
def
getClass(): Class[_]
- Definition Classes
- AnyRef → Any
- Annotations
- @native()
-
def
hashCode(): Int
- Definition Classes
- AnyRef → Any
- Annotations
- @native()
-
def
haveInstance(formula: Formula, polarity: Polarity): Tactical[String]
Instantiates prenex quantifiers to obtain a formula in a given polarity.
Instantiates prenex quantifiers to obtain a formula in a given polarity.
- Definition Classes
- TacticCommands
-
def
haveInstances(sequent: HOLSequent): Tactical[Sequent[String]]
- Definition Classes
- TacticCommands
-
def
impL: ImpLeftTactic
Applies the
ImpLeft
tactic to the current subgoal: The goalApplies the
ImpLeft
tactic to the current subgoal: The goalA → B, Γ :- Δ
is reduced to
Γ :- Δ, A
andB, Γ :- Δ
.This will only work if there is exactly one implicative formula in the antecedent!
- Definition Classes
- TacticCommands
-
def
impL(applyToLabel: String): ImpLeftTactic
Applies the
ImpLeft
tactic to the current subgoal: The goalApplies the
ImpLeft
tactic to the current subgoal: The goalA → B, Γ :- Δ
is reduced to
Γ :- Δ, A
andB, Γ :- Δ
.- applyToLabel
The label of the formula
A → B
.
- Definition Classes
- TacticCommands
-
def
impR: ImpRightTactic
Applies the
ImpRight
tactic to the current subgoal: The goalApplies the
ImpRight
tactic to the current subgoal: The goalΓ :- Δ, A → B
is reduced to
A, Γ :- Δ, B
.This will only work if there is exactly one implicative formula in the succedent!
- Definition Classes
- TacticCommands
-
def
impR(applyToLabel: String): ImpRightTactic
Applies the
ImpRight
tactic to the current subgoal: The goalApplies the
ImpRight
tactic to the current subgoal: The goalΓ :- Δ, A → B
is reduced to
A, Γ :- Δ, B
.- applyToLabel
The label of the formula
A → B
.
- Definition Classes
- TacticCommands
-
def
include(label: String, proof: LKProof): Tactical[Unit]
Uses an LKProof as a lemma.
Uses an LKProof as a lemma.
If
proof
ends inΓ :- φ
, then the current goalΓ, Π :- Λ
is reduced to
Γ, Π, φ :- Λ
- label
the label for φ in the subgoal
- proof
The proof to insert as a lemma by a cut.
- Definition Classes
- TacticCommands
-
def
induction(on: Var, label: String)(implicit ctx: Context): InductionTactic
Applies the
Induction
tactic to the current subgoal: The goalApplies the
Induction
tactic to the current subgoal: The goalΓ, :- Δ, ∀x.A
is reduced to
n
new subgoals, wheren
is the number of constructors of the type ofx
.- label
The label of the formula
∀x.A
.- ctx
A at.logic.gapt.proofs.Context. It must contain an inductive definition of the type of
x
.
- Definition Classes
- TacticCommands
-
def
induction(on: Var)(implicit ctx: Context): InductionTactic
Applies the
Induction
tactic to the current subgoal: The goalApplies the
Induction
tactic to the current subgoal: The goalΓ, :- Δ, ∀x.A
is reduced to
n
new subgoals, wheren
is the number of constructors of the type ofx
.This will only work if there is exactly one universal formula in the succedent!
- ctx
A at.logic.gapt.proofs.Context. It must contain an inductive definition of the type of
x
.
- Definition Classes
- TacticCommands
-
def
insert(proof: LKProof): InsertTactic
Inserts an LKProof for the current subgoal.
Inserts an LKProof for the current subgoal.
- proof
The proof to be inserted. Its end-sequent must subsume the current goal.
- Definition Classes
- TacticCommands
-
def
introUnivsExcept(i: Int): Tactical[Unit]
- Definition Classes
- TacticCommands
-
final
def
isInstanceOf[T0]: Boolean
- Definition Classes
- Any
-
final
def
ne(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef
-
def
negL: NegLeftTactic
Applies the
NegLeft
tactic to the current subgoal: The goalApplies the
NegLeft
tactic to the current subgoal: The goal¬A, Γ :- Δ
is reduced to
Γ :- Δ, A
.This will only work if there is exactly one negated formula in the antecedent!
- Definition Classes
- TacticCommands
-
def
negL(applyToLabel: String): NegLeftTactic
Applies the
NegLeft
tactic to the current subgoal: The goalApplies the
NegLeft
tactic to the current subgoal: The goal¬A, Γ :- Δ
is reduced to
Γ :- Δ, A
.- applyToLabel
The label of the formula
¬A
.
- Definition Classes
- TacticCommands
-
def
negR: NegRightTactic
Applies the
NegRight
tactic to the current subgoal: The goalApplies the
NegRight
tactic to the current subgoal: The goalΓ :- Δ, A
is reduced to
A, Γ :- Δ
.This will only work if there is exactly one negated formula in the succedent!
- Definition Classes
- TacticCommands
-
def
negR(applyToLabel: String): NegRightTactic
Applies the
NegRight
tactic to the current subgoal: The goalApplies the
NegRight
tactic to the current subgoal: The goalΓ :- Δ, ¬A
is reduced to
A, Γ :- Δ
.- applyToLabel
The label of the formula
¬A
.
- Definition Classes
- TacticCommands
-
final
def
notify(): Unit
- Definition Classes
- AnyRef
- Annotations
- @native()
-
final
def
notifyAll(): Unit
- Definition Classes
- AnyRef
- Annotations
- @native()
-
def
now: Tactical[Unit]
- Definition Classes
- TacticCommands
-
def
orL: OrLeftTactic
Applies the
OrLeft
tactic to the current subgoal: The goalApplies the
OrLeft
tactic to the current subgoal: The goalA ∨ B, Γ :- Δ
is reduced to
A, Γ :- Δ
andB, Γ :- Δ
.This will only work if there is exactly one disjunctive formula in the antecedent!
- Definition Classes
- TacticCommands
-
def
orL(applyToLabel: String): OrLeftTactic
Applies the
OrLeft
tactic to the current subgoal: The goalApplies the
OrLeft
tactic to the current subgoal: The goalA ∨ B, Γ :- Δ
is reduced to
A, Γ :- Δ
andB, Γ :- Δ
.- applyToLabel
The label of the formula
A ∨ B
.
- Definition Classes
- TacticCommands
-
def
orR: OrRightTactic
Applies the
OrRight
tactic to the current subgoal: The goalApplies the
OrRight
tactic to the current subgoal: The goalΓ :- Δ, A ∨ B
is reduced to
Γ :- Δ, A, B
.This will only work if there is exactly one disjunctive formula in the succedent!
- Definition Classes
- TacticCommands
-
def
orR(applyToLabel: String): OrRightTactic
Applies the
OrRight
tactic to the current subgoal: The goalApplies the
OrRight
tactic to the current subgoal: The goalΓ :- Δ, A ∨ B
is reduced to
Γ :- Δ, A, B
.- applyToLabel
The label of the formula
A ∨ B
.
- Definition Classes
- TacticCommands
-
def
prop: Tactic[Unit]
Calls the builtin tableau prover on the current subgoal.
Calls the builtin tableau prover on the current subgoal. If the goal is a tautology, a proof will automatically be found and inserted.
- Definition Classes
- TacticCommands
-
def
prover9(implicit ctx: MutableContext): ResolutionProverTactic
Calls
prover9
on the current subgoal.Calls
prover9
on the current subgoal.- Definition Classes
- TacticCommands
-
def
quasiprop: Tactic[Unit]
- Definition Classes
- TacticCommands
-
def
ref(proofName: String)(implicit ctx: Context): ProofLinkTactic
Applies the
LogicalAxiom
tactic to the current subgoal: A subgoal of the formA, Γ :- Δ, A
will be closed.Applies the
LogicalAxiom
tactic to the current subgoal: A subgoal of the formA, Γ :- Δ, A
will be closed.- Definition Classes
- TacticCommands
-
def
refl: ReflexivityAxiomTactic.type
Synonym for axiomRefl.
Synonym for axiomRefl.
- Definition Classes
- TacticCommands
-
def
renameLabel(oldLabel: String): RenameTactic
Changes the provided label.
Changes the provided label. Syntax:
renameLabel("foo") to "bar"
- oldLabel
The label to be renamed.
- Definition Classes
- TacticCommands
-
def
repeat[T](t: Tactical[T]): RepeatTactic[T]
Repeats a tactical until it fails.
-
def
resolutionProver(prover: Prover)(implicit ctx: MutableContext): ResolutionProverTactic
- Definition Classes
- TacticCommands
-
def
rewrite: RewriteTactic
Rewrites the formula specified by target using (possibly universally quantified) equations.
Rewrites the formula specified by target using (possibly universally quantified) equations.
rewrite.many ltr "equation1" in "target" rewrite.many ltr ("equation1", "eq2") rtl ("eq3", "eq4") in "target" subst (hov"x" -> le"f(f(c))")
ltr
: rewrite left-to-right using this equationrtl
: rewrite right-to-left using this equationmany
: rewrite as long as possible (default is to only rewrite once)- Definition Classes
- TacticCommands
-
def
skip: Tactical[Unit]
Does nothing.
Does nothing.
- Definition Classes
- TacticCommands
-
final
def
synchronized[T0](arg0: ⇒ T0): T0
- Definition Classes
- AnyRef
-
def
theory(implicit ctx: Context): Tactical[Unit]
Declares the current subgoal as a theory axiom, i.e.
Declares the current subgoal as a theory axiom, i.e. a sequent that is contained in the background theory. This closes the goal.
- ctx
A at.logic.gapt.proofs.Context. The current subgoal must be contained in its background theory.
- Definition Classes
- TacticCommands
-
def
toString(): String
- Definition Classes
- AnyRef → Any
-
def
treeGrammarInduction(implicit ctx: Context): TreeGrammarInductionTactic
- Definition Classes
- TacticCommands
-
def
trivial: Tactical[Unit]
Attempts to apply the tactics
axiomTop
,axiomBot
,axiomRefl
, andaxiomLog
.Attempts to apply the tactics
axiomTop
,axiomBot
,axiomRefl
, andaxiomLog
.- Definition Classes
- TacticCommands
-
def
unfold(definitions: String*)(implicit ctx: Context): UnfoldTacticHelper
Replaces a defined constant with its definition.
Replaces a defined constant with its definition. Syntax:
unfold("def1", "def2",...,"defn") in ("label1", "label2",...,"labelk")
NB: This will only replace the first definition it finds in each supplied formula. If you want to unfold all definitions, use
repeat
.- definitions
The definitions
def1
,...,defn
.- ctx
A at.logic.gapt.proofs.Context. The definitions you want to unfold need to be present in
ctx
.
- Definition Classes
- TacticCommands
-
final
def
wait(): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws( ... )
-
final
def
wait(arg0: Long, arg1: Int): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws( ... )
-
final
def
wait(arg0: Long): Unit
- Definition Classes
- AnyRef
- Annotations
- @native() @throws( ... )
Deprecated Value Members
-
def
sorry: Tactical[Unit]
Leaves a hole in the current proof by inserting a dummy proof of the empty sequent.
Leaves a hole in the current proof by inserting a dummy proof of the empty sequent.
- Definition Classes
- TacticCommands
- Annotations
- @deprecated
- Deprecated
(Since version the dawn of time) Proof not finished!
This is the API documentation for GAPT.
The main package is at.logic.gapt.