File tree Expand file tree Collapse file tree 2 files changed +15
-1
lines changed
Expand file tree Collapse file tree 2 files changed +15
-1
lines changed Original file line number Diff line number Diff line change @@ -1120,7 +1120,7 @@ let rec t_hi_conseq notmod f1 f2 f3 tc =
11201120 t_intros_i [m;h0] @! t_cutdef
11211121 (ptlocal ~args: [pamemory m; palocal h0] hi)
11221122 mpre @! EcLowGoal. t_trivial;
1123- t_mytrivial;
1123+ t_mytrivial @! t_intros_i [m; h0] @! t_apply_hyp h0 ;
11241124 t_apply_hyp hh];
11251125 tac pre posta @+ [
11261126 t_apply_hyp hi;
Original file line number Diff line number Diff line change 1+ require import Real.
2+
3+ module Foo = {proc foo () = {}}.
4+
5+ lemma foo_ll : islossless Foo.foo by islossless.
6+
7+ op [opaque] p = predT<:int >.
8+
9+ lemma foo_h: hoare [ Foo.foo : true ==> forall j, p j].
10+ proof. by proc; auto => /> j; rewrite /p. qed.
11+
12+ lemma foo_p: phoare[ Foo.foo : true ==> forall j, p j] = 1 %r.
13+ by conseq foo_ll foo_h.
14+ qed.
You can’t perform that action at this time.
0 commit comments