File: Timing.v

package info (click to toggle)
coq-quickchick 2.1.1-2
  • links: PTS, VCS
  • area: main
  • in suites: experimental
  • size: 2,432 kB
  • sloc: ml: 4,367; ansic: 789; makefile: 388; sh: 27; python: 4; lisp: 2; perl: 2
file content (134 lines) | stat: -rw-r--r-- 4,521 bytes parent folder | download | duplicates (4)
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
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
90
91
92
93
94
95
96
97
98
99
100
101
102
103
104
105
106
107
108
109
110
111
112
113
114
115
116
117
118
119
120
121
122
123
124
125
126
127
128
129
130
131
132
133
134
From QuickChick Require Import QuickChick.

Require Import List. Import ListNotations.

From QuickChick.ifcbasic Require Import Machine Printing Generation Indist DerivedGen.
From QuickChick.ifcbasic Require GenExec.

Require Import Coq.Strings.String.
Local Open Scope string.

Definition SSNI_manual (t : table) (v : @Variation State) : Checker  :=
  let '(V st1 st2) := v in
  let '(St _ _ _ (_@l1)) := st1 in
  let '(St _ _ _ (_@l2)) := st2 in
  if indist st1 st2 then
    match l1, l2 with
      | L,L  =>
        match exec t st1, exec t st2 with
          | Some st1', Some st2' =>
            checker (indist st1' st2')
          | _, _ => checker rejected
        end
      | H, H =>
        match exec t st1, exec t st2 with
          | Some st1', Some st2' =>
            if is_atom_low (st_pc st1') && is_atom_low (st_pc st2') then
              checker (indist st1' st2') 
            else if is_atom_low (st_pc st1') then
              (checker (indist st2 st2'))
            else
              (checker (indist st1 st1'))
          | _, _ => checker rejected
        end
      | H,_ =>
        match exec t st1 with
          | Some st1' =>
            checker (indist st1 st1')
          | _ => checker rejected
        end
      | _,H =>
        match exec t st2 with
          | Some st2' =>
            checker  (indist st2 st2')
          | _ => checker rejected
        end
    end
  else checker rejected.

Instance CheckableOptBool : Checkable (option bool) :=
  { checker x :=
      match x with
      | Some true  => checker true
      | Some false => checker false
      | None => checker rejected
      end }.

Definition SSNI_derived (t : table) (v : @Variation State) : Checker  :=
  let '(V st1 st2) := v in
  let '(St _ _ _ (_@l1)) := st1 in
  let '(St _ _ _ (_@l2)) := st2 in
  match @decOpt (IndistState st1 st2) _ 5 with
  | Some true =>
    match l1, l2 with
      | L,L  =>
        match exec t st1, exec t st2 with
        | Some st1', Some st2' =>
(*          whenFail ("Initial states: " ++ nl ++ show_pair st1 st2 ++ nl
                                       ++ "Final states: " ++ nl ++ show_pair st1' st2' ++nl)*)
            (checker (@decOpt (IndistState st1' st2') _ 5))
          | _, _ => checker rejected
        end
      | H, H =>
        match exec t st1, exec t st2 with
          | Some st1', Some st2' =>
            if is_atom_low (st_pc st1') && is_atom_low (st_pc st2') then
            whenFail ("Initial states: " ++ nl ++ show_pair st1 st2 ++ nl
                        ++ "Final states: " ++ nl ++ show_pair st1' st2' ++nl) 
              
            (checker (@decOpt (IndistState st1' st2') _ 5))
            else if is_atom_low (st_pc st1') then
                   whenFail ("States: " ++ nl ++ show_pair st2 st2' ++ nl )
                   
                   (checker (@decOpt (IndistState st2 st2') _ 5))
                 else
                    whenFail ("States: " ++ nl ++ show_pair st1 st1' ++ nl )
            (checker (@decOpt (IndistState st1 st1') _ 5))
          | _, _ => checker rejected
        end
      | H,_ =>
        match exec t st1 with
        | Some st1' =>
          whenFail ("States: " ++ nl ++ show_pair st1 st1' ++ nl )
          
            (checker (@decOpt (IndistState st1 st1') _ 5))
          | _ => checker rejected
        end
      | _,H =>
        match exec t st2 with
        | Some st2' =>
          whenFail ("States: " ++ nl ++ show_pair st2 st2' ++ nl )
          
            (checker (@decOpt (IndistState st2 st2') _ 5))
          | _ => checker rejected
        end
    end
  | _ => checker rejected
  end.

Axiom withTime : Checker -> Checker.
Extract Constant withTime =>
  "(fun c -> Printf.printf ""%.8f\n"" (Sys.time ()); c)".

Definition prop_manual : Checker :=
  forAllShrink gen_variation_state (fun _ => nil)
               (fun v => SSNI_manual default_table v).

Definition prop_derived : Checker :=
  forAllShrink gen_variation_state (fun _ => nil)
               (fun v => SSNI_derived default_table v).

Extract Constant defNumTests => "20000".
QuickChick prop_manual.
QuickChick prop_derived.
(*
Definition prop_test : Checker :=
  forAllShrink gen_variation_state (fun _ => nil)
               (fun v =>
                  let r0 := trace ("Next" ++ nl) (checker true) in
                  let r2 := withTime (SSNI_derived default_table v) in
                  let r1 := withTime (SSNI_manual default_table v) in
                  withTime (conjoin [r0;r2;r1])).

QuickChick prop_test.
*)