Skip to content

Commit

Permalink
Reinstate old behaviour when rewrites compete
Browse files Browse the repository at this point in the history
If we have ⊢ x = e1 in the argument list and x = e2 as an assumption,
the theorem in the assumptions used to be chosen first by simp and
friends. The commit in cfa24e2 flipped this choice, but this flips
it back again. Of course, users shouldn't really be relying on this,
but at least one CakeML proof did, and in this case, there seems no
need to punish this.
  • Loading branch information
mn200 committed Oct 3, 2024
1 parent 8871e08 commit 4ee759f
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/marker/markerLib.sml
Original file line number Diff line number Diff line change
Expand Up @@ -696,7 +696,7 @@ fun filter_then asms aslPs thltac (gl as (asl0,g)) =
val asl = apply_aslPs (free_varsl (g::asl0)) aslPs
(filter (not o is_label) asl0)
in
thltac (asms @ map ASSUME asl) gl
thltac (map ASSUME asl @ asms) gl
end

fun process_taclist_then {arg} thltac (gl as (asl,g)) =
Expand Down

0 comments on commit 4ee759f

Please sign in to comment.