data:image/s3,"s3://crabby-images/02ace/02ace956f9868cf2a1a780bd2c0a517cd3a46077" alt="JAR search and dependency download from the Maven repository"
gapt.proofs.context.update.ProofDefinitionDeclaration.scala Maven / Gradle / Ivy
Go to download
Show more of this group Show more artifacts with this name
Show all versions of gapt_3 Show documentation
Show all versions of gapt_3 Show documentation
General Architecture for Proof Theory
The newest version!
package gapt.proofs.context.update
import gapt.expr.Apps
import gapt.expr.Const
import gapt.expr.Expr
import gapt.proofs.SequentConnector
import gapt.proofs.context.Context
import gapt.proofs.context.ProofDefinition
import gapt.proofs.context.facet.ProofDefinitions
import gapt.proofs.context.facet.ProofNames
import gapt.proofs.context.State
import gapt.proofs.lk.LKProof
case class ProofDefinitionDeclaration(lhs: Expr, referencedProof: LKProof) extends Update {
override def apply(ctx: Context): State = {
ctx.check(referencedProof)
val Apps(c: Const, vs) = lhs: @unchecked
vs.foreach(ctx.check(_))
val declSeq = ctx.get[ProofNames].lookup(lhs)
.getOrElse(throw new IllegalArgumentException(s"Proof name ${lhs.toSigRelativeString(ctx)} is not defined"))
require(
referencedProof.conclusion.isSubMultisetOf(declSeq),
"End-sequent of proof definition does not match declaration.\n" +
"Given sequent: " + referencedProof.endSequent.toSigRelativeString(ctx) + "\n" +
"Expected sequent: " + declSeq.toSigRelativeString(ctx) + "\n" +
"Extraneous formulas: " +
referencedProof.endSequent.diff(declSeq).toSigRelativeString(ctx)
)
val conn = SequentConnector.guessInjection(fromLower = referencedProof.conclusion, toUpper = declSeq)
val defn = ProofDefinition(lhs, conn, referencedProof)
ctx.state.update[ProofDefinitions](_ + defn)
}
}
© 2015 - 2025 Weber Informatics LLC | Privacy Policy