Skip to content

Commit

Permalink
Fix definition broken by HOL's change to Inductive syntax
Browse files Browse the repository at this point in the history
  • Loading branch information
mn200 committed Nov 7, 2023
1 parent a121a00 commit aeb8c0f
Showing 1 changed file with 6 additions and 6 deletions.
12 changes: 6 additions & 6 deletions compiler/backend/proofs/clos_opProofScript.sml
Expand Up @@ -698,21 +698,21 @@ Inductive red_rel:
ElemAt t1; Constant (ConstInt i); Constant (ConstStr s);
Constant (ConstWord64 w)] ⇒
red_rel [Op t op xs] ys)
[∧]
(red_rel [] [])
[∧]
(∀x. red_rel [x] [x])
[∧]
(∀v t. red_rel [Var t v] [])
[red_rel_multi:]
(∀x y zs x1 x2.
red_rel [x] x1 ∧ red_rel (y::zs) x2 ⇒
red_rel (x::y::zs) (x1 ++ x2))
red_rel (x::y::zs) (x1 ++ x2))
[red_rel_Let:]
(∀xs x x1 t.
red_rel xs x1 ∧ red_rel [x] [] ⇒
red_rel [Let t xs x] x1) ∧
red_rel [Let t xs x] x1)
[∧]
(∀x y z x1 x2 x3.
red_rel [x] x1 ∧ red_rel [y] x2 ∧ red_rel [z] x3 ⇒
red_rel [If t x y z] (x1 ++ x2 ++ x3))
Expand Down

0 comments on commit aeb8c0f

Please sign in to comment.