blob: 1b57e5b514f9ed7aeb2daffeca43fa8e94bb1776 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
|
Require Import Crypto.Compilers.Syntax.
Require Import Crypto.Compilers.Named.Context.
Require Import Crypto.Util.Tactics.BreakMatch.
Require Import Crypto.Util.Decidable.
Section with_context.
Context {base_type_code Name var} (Context : @Context base_type_code Name var)
(base_type_code_dec : DecidableRel (@eq base_type_code))
(Name_dec : DecidableRel (@eq Name)).
Fixpoint find_Name n
{T : flat_type base_type_code}
: interp_flat_type (fun _ => Name) T -> option base_type_code
:= match T with
| Tbase t' => fun n' : Name => if dec (n = n') then Some t' else None
| Unit => fun _ => None
| Prod A B
=> fun ab : interp_flat_type _ A * interp_flat_type _ B
=> match @find_Name n B (snd ab), @find_Name n A (fst ab) with
| Some tb, _ => Some tb
| None, Some ta => Some ta
| None, None => None
end
end.
Fixpoint find_Name_and_val {var'} t (n : Name)
{T : flat_type base_type_code}
: interp_flat_type (fun _ => Name) T -> interp_flat_type var' T -> option (var' t) -> option (var' t)
:= match T with
| Tbase t' => fun (n' : Name) v default
=> if dec (n = n')
then cast_if_eq t' t v
else default
| Unit => fun _ _ default => default
| Prod A B
=> fun (ab : interp_flat_type _ A * interp_flat_type _ B)
(a'b' : interp_flat_type _ A * interp_flat_type _ B)
default
=> @find_Name_and_val
var' t n B (snd ab) (snd a'b')
(@find_Name_and_val
var' t n A (fst ab) (fst a'b')
default)
end.
Class ContextOk :=
{ lookupb_extendb_same
: forall (ctx : Context) n t v, lookupb t (extendb ctx n (t:=t) v) n = Some v;
lookupb_extendb_different
: forall (ctx : Context) n n' t t' v, n <> n' -> lookupb t' (extendb ctx n (t:=t) v) n'
= lookupb t' ctx n';
lookupb_extendb_wrong_type
: forall (ctx : Context) n t t' v, t <> t' -> lookupb t' (extendb ctx n (t:=t) v) n = None;
lookupb_removeb_different
: forall (ctx : Context) n n' t t', n <> n' -> lookupb t' (removeb t ctx n) n'
= lookupb t' ctx n';
lookupb_removeb_same
: forall (ctx : Context) n t t', lookupb t' (removeb t ctx n) n = None;
lookupb_empty
: forall n t, lookupb t (@empty _ _ _ Context) n = None;
lookupb_unique_type
: forall (ctx : Context) n t t', lookupb t' ctx n <> None -> lookupb t ctx n <> None -> t = t' }.
Definition context_equiv (a b : Context)
:= forall n t, lookupb t a n = lookupb t b n.
End with_context.
|