Skip to content

Commit

Permalink
sed -ie "s/RhsPattern/ExpressionTerm/g"
Browse files Browse the repository at this point in the history
  • Loading branch information
h0nzZik committed Jan 30, 2024
1 parent aeb5db6 commit 2f21c3c
Show file tree
Hide file tree
Showing 4 changed files with 7 additions and 7 deletions.
2 changes: 1 addition & 1 deletion minuska/theories/naive_interpreter.v
Original file line number Diff line number Diff line change
Expand Up @@ -100,7 +100,7 @@ Definition rewrite_with
Lemma evaluate_rhs_pattern_correct
{Σ : StaticModel}

(φ : RhsPattern)
(φ : ExpressionTerm)
(ρ : Valuation)
(g : GroundTerm)
:
Expand Down
4 changes: 2 additions & 2 deletions minuska/theories/spec_semantics.v
Original file line number Diff line number Diff line change
Expand Up @@ -666,7 +666,7 @@ Instance Satisfies_asb_expr


#[export]
Instance Satisfies__GroundTerm__RhsPattern
Instance Satisfies__GroundTerm__ExpressionTerm
{Σ : StaticModel}
{V var : Type}
{_varED : EqDecision var}
Expand All @@ -680,7 +680,7 @@ Instance Satisfies__GroundTerm__RhsPattern
Satisfies
V
GroundTerm
RhsPattern
ExpressionTerm
var
.
Proof. apply _. Defined.
Expand Down
4 changes: 2 additions & 2 deletions minuska/theories/spec_syntax.v
Original file line number Diff line number Diff line change
Expand Up @@ -147,7 +147,7 @@ Inductive SideCondition {Σ : StaticModel} :=
| sc_constraint (c : AtomicProposition)
.

Definition RhsPattern {Σ : StaticModel} :=
Definition ExpressionTerm {Σ : StaticModel} :=
Term' symbol Expression
.

Expand All @@ -158,7 +158,7 @@ Record RewritingRule {Σ : StaticModel}
:= mkRewritingRule
{
fr_from : SymbolicTerm ;
fr_to : RhsPattern ;
fr_to : ExpressionTerm ;
fr_scs : list SideCondition ;
}.

Expand Down
4 changes: 2 additions & 2 deletions minuska/theories/syntax_properties.v
Original file line number Diff line number Diff line change
Expand Up @@ -105,8 +105,8 @@ Section eqdec.
Defined.

#[export]
Instance RhsPattern_eqdec {Σ : StaticModel}
: EqDecision RhsPattern
Instance ExpressionTerm_eqdec {Σ : StaticModel}
: EqDecision ExpressionTerm
.
Proof.
ltac1:(solve_decision).
Expand Down

0 comments on commit 2f21c3c

Please sign in to comment.