Skip to content

Commit

Permalink
Browse files Browse the repository at this point in the history
  • Loading branch information
liyishuai committed Jan 5, 2024
1 parent 6ae41d2 commit 235f6f2
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/Instances.v
Original file line number Diff line number Diff line change
Expand Up @@ -725,21 +725,21 @@ Proof.
move: H2 => [[H2 | [H2 | H2]] H3];
destruct m => //=; apply Hgen => //=;
inversion H2; subst; auto; simpl in *.
+ apply (@semReturnSize Generators.G ProducerGen ProducerSemanticsGen (option A) _) in H3; inversion H3.
+ apply semLiftProdSize in H3; eauto with typeclass_instances. inversion H3 as [x [H0 H1]].
+ apply (@semReturnSize Generators.G ProducerGen ProducerSemanticsGen (option A) None s (Some a)) in H3; inversion H3.
+ apply (@semLiftProdSize _ ProducerGen _ _ _ Some (@arbitrary _ G) s (Some a)) in H3; eauto with typeclass_instances. inversion H3 as [x [H0 H1]].
inversion H1; subst; auto.
- destruct m eqn:Hm; simpl in *; move => HP; subst.
+ apply semFrequencySize; simpl.
exists (7, liftM Some arbitrary); split; auto.
* right; left; auto.
* simpl. apply semLiftProdSize; simpl;
* simpl. apply (@semLiftProdSize _ ProducerGen _ _ _ Some (@arbitrary _ G) s (Some a)); simpl;
eauto with typeclass_instances.
apply imset_in; apply Hgen; auto.
+ apply semFrequencySize; simpl.
exists (1, ret None); split; auto.
* left; auto.
* simpl.
apply (@semReturnSize Generators.G ProducerGen ProducerSemanticsGen). constructor.
apply (@semReturnSize Generators.G ProducerGen ProducerSemanticsGen (option A) None s None). constructor.
Qed.

Lemma arbPair_correctSize
Expand Down

0 comments on commit 235f6f2

Please sign in to comment.