1 (********************************************************************)
3 (* The Why3 Verification Platform
/ The Why3 Development Team
*)
4 (* Copyright
2010-2023 -- Inria
- CNRS
- Paris
-Saclay University
*)
6 (* This software is distributed under the terms of the GNU Lesser
*)
7 (* General Public License version
2.1, with the special exception
*)
8 (* on linking described in file LICENSE.
*)
10 (********************************************************************)
12 (* This file is generated by Why3
's Coq-realize driver *)
13 (* Beware! Only edit allowed sections below *)
14 Require Import BuiltIn.
28 Definition p : set.Fset.fset t -> Prop.
36 (forall (s:set.Fset.fset t), set.Fset.is_empty s -> p s) ->
37 (forall (s:set.Fset.fset t), p s -> (forall (t1:t), p (set.Fset.add t1 s))) ->
38 forall (s:set.Fset.fset t), p s.
41 (* TODO make something interesting *)
42 unfold p. constructor.