From b79d0a04787d9234cf580841bf58e592fe4ab3ee Mon Sep 17 00:00:00 2001 From: Sylvain Boulmé Date: Fri, 28 May 2021 15:24:16 +0200 Subject: starting to extend RTLtoBTL with Liveness checking (on BTL side) --- scheduling/BTLmatchRTL.v | 12 ------------ 1 file changed, 12 deletions(-) (limited to 'scheduling/BTLmatchRTL.v') diff --git a/scheduling/BTLmatchRTL.v b/scheduling/BTLmatchRTL.v index 23ff6681..8994579d 100644 --- a/scheduling/BTLmatchRTL.v +++ b/scheduling/BTLmatchRTL.v @@ -223,18 +223,6 @@ Record match_function dupmap f f': Prop := { preserv_fnstacksize: fn_stacksize f = RTL.fn_stacksize f' }. -Inductive match_fundef: BTL.fundef -> RTL.fundef -> Prop := - | match_Internal dupmap f f': match_function dupmap f f' -> match_fundef (Internal f) (Internal f') - | match_External ef: match_fundef (External ef) (External ef). - -Inductive match_stackframes: stackframe -> RTL.stackframe -> Prop := - | match_stackframe_intro - dupmap res f sp pc rs f' pc' - (TRANSF: match_function dupmap f f') - (DUPLIC: dupmap!pc = Some pc') - : match_stackframes (BTL.Stackframe res f sp pc rs) (RTL.Stackframe res f' sp pc' rs). - - (** * Shared verifier between RTL -> BTL and BTL -> RTL *) Local Open Scope error_monad_scope. -- cgit