summaryrefslogtreecommitdiff
path: root/backend/InterfGraphProperties.v
blob: 09e1b59fdd21db77f396333e81af0db99cf0e0c2 (plain)
1
2
3
4
5
6
7
8
Require Import InterfGraph.
Require Import Coloring.

Lemma set_reg_reg_diff_ext : forall x f live live0,
SetRegReg.In x (interf_reg_reg (interf_graph f live live0)) -> fst x <> snd x.

Proof.
Admitted.